Skip to content

Commit

Permalink
Fix AesopTest.HeartbeatLimit
Browse files Browse the repository at this point in the history
  • Loading branch information
JLimperg committed Aug 6, 2024
1 parent 2ca67d8 commit 6786aef
Showing 1 changed file with 5 additions and 10 deletions.
15 changes: 5 additions & 10 deletions AesopTest/HeartbeatLimit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,23 +8,18 @@ import Aesop
import Batteries.Linter.UnreachableTactic

set_option aesop.check.all true
set_option aesop.smallErrorMessages true
set_option linter.unreachableTactic false

@[aesop safe constructors]
inductive Even : Nat → Prop
| zero : Even 0
| plusTwo : Even n → Even (n + 2)

-- FIXME this is producing a different message under v4.11.0-rc1

-- /--
-- error: (deterministic) timeout at `whnf`, maximum number of heartbeats (1) has been reached
-- use `set_option maxHeartbeats <num>` to set the limit
-- use `set_option diagnostics true` to get diagnostic information
-- -/
-- #guard_msgs in
-- example : Even 10 := by
-- aesop (config := { maxRuleHeartbeats := 1, terminal := true })
/-- error: tactic 'aesop' failed, failed to prove the goal after exhaustive search. -/
#guard_msgs in
example : Even 10 := by
aesop (config := { maxRuleHeartbeats := 1, terminal := true })

example : Even 10 := by
aesop
Expand Down

0 comments on commit 6786aef

Please sign in to comment.