Skip to content

Commit

Permalink
remove logInfo for Branch finishing proof
Browse files Browse the repository at this point in the history
  • Loading branch information
joneugster committed Apr 8, 2024
1 parent 7cedfc5 commit ce71bc8
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion server/GameServer/Commands.lean
Original file line number Diff line number Diff line change
Expand Up @@ -577,7 +577,8 @@ elab (name := GameServer.Tactic.Branch) "Branch" t:tacticSeq : tactic => do
-- Show an info whether the branch proofs all remaining goals.
let gs ← Tactic.getUnsolvedGoals
if gs.isEmpty then
trace[debug] "This branch finishes the proof."
-- trace[debug] "This branch finishes the proof."
pure ()
else
trace[debug] "This branch leaves open goals."

Expand Down

0 comments on commit ce71bc8

Please sign in to comment.