Skip to content

Commit

Permalink
Merge pull request #35 from abdoo8080/patch-1
Browse files Browse the repository at this point in the history
Delete profile messages.
  • Loading branch information
PratherConid authored Nov 24, 2024
2 parents 91e5820 + d0b5f5d commit d9af64d
Showing 1 changed file with 0 additions and 4 deletions.
4 changes: 0 additions & 4 deletions Auto/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -476,7 +476,6 @@ def runAuto
@[tactic auto]
def evalAuto : Tactic
| `(auto | auto $instr $hints $[$uords]*) => withMainContext do
let startTime ← IO.monoMsNow
-- Suppose the goal is `∀ (x₁ x₂ ⋯ xₙ), G`
-- First, apply `intros` to put `x₁ x₂ ⋯ xₙ` into the local context,
-- now the goal is just `G`
Expand All @@ -492,7 +491,6 @@ def evalAuto : Tactic
let (lemmas, inhFacts) ← collectAllLemmas hints uords (goalBinders.push ngoal)
let declName? ← Elab.Term.getDeclName?
let proof ← runAuto declName? lemmas inhFacts
IO.println s!"Auto found proof. Time spent by auto : {(← IO.monoMsNow) - startTime}ms"
absurd.assign proof
| .useSorry =>
let proof ← Meta.mkAppM ``sorryAx #[Expr.const ``False [], Expr.const ``false []]
Expand Down Expand Up @@ -562,7 +560,6 @@ def runNativeProverWithAuto
@[tactic mononative]
def evalMonoNative : Tactic
| `(mononative | mononative $hints $[$uords]*) => withMainContext do
let startTime ← IO.monoMsNow
-- Suppose the goal is `∀ (x₁ x₂ ⋯ xₙ), G`
-- First, apply `intros` to put `x₁ x₂ ⋯ xₙ` into the local context,
-- now the goal is just `G`
Expand All @@ -574,7 +571,6 @@ def evalMonoNative : Tactic
withMainContext do
let (lemmas, inhFacts) ← collectAllLemmas hints uords (goalBinders.push ngoal)
let proof ← monoInterface lemmas inhFacts Solver.Native.queryNative
IO.println s!"Auto found proof. Time spent by auto : {(← IO.monoMsNow) - startTime}ms"
absurd.assign proof
| _ => throwUnsupportedSyntax

Expand Down

0 comments on commit d9af64d

Please sign in to comment.