Skip to content

Commit

Permalink
add IO.monoMsNow time stamp
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Jan 12, 2025
1 parent 384d308 commit 8650ab9
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 0 deletions.
1 change: 1 addition & 0 deletions Auto/EvaluateAuto/TestAuto.lean
Original file line number Diff line number Diff line change
Expand Up @@ -129,6 +129,7 @@ def runAutoOnConsts (config : EvalAutoConfig) (names : Array Name) : CoreM Unit
if let .some fhandle := logFileHandle? then
fhandle.putStrLn ""
fhandle.putStrLn s!"Testing || {name} : {← (Lean.Meta.ppExpr ci.type).run'}"
fhandle.putStrLn s!"IO.monoMsNow : {← IO.monoMsNow}"
fhandle.flush
let result : Result ← withCurrHeartbeats <|
withReader (fun ctx => {ctx with maxHeartbeats := config.maxHeartbeats * 1000}) <|
Expand Down
1 change: 1 addition & 0 deletions Auto/EvaluateAuto/TestTactics.lean
Original file line number Diff line number Diff line change
Expand Up @@ -225,6 +225,7 @@ where
if let .some fhandle := logFileHandle? then
fhandle.putStrLn ""
fhandle.putStrLn s!"Testing tactic {idx} || {ci.name} : {← (Lean.Meta.ppExpr ci.type).run'}"
fhandle.putStrLn s!"IO.monoMsNow : {← IO.monoMsNow}"
fhandle.flush
let result ← (do
if nonterms.contains (tactic, ci.name) then
Expand Down

0 comments on commit 8650ab9

Please sign in to comment.