Skip to content

Commit 7429773

Browse files
committed
chore: fix test
1 parent 11f88a4 commit 7429773

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

tests/lean/run/grind_offset_cnstr.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
module
22
set_option grind.debug true
3-
3+
set_option warn.sorry false
44
/--
55
trace: [grind.offset.internalize.term] a1 ↦ #0
66
[grind.offset.internalize.term] a2 ↦ #1
@@ -274,7 +274,7 @@ trace: [grind.debug.proof] intro_with_eq (p ↔ a2 ≤ a1) (p = (a2 ≤ a1)) (¬
274274
open Lean Grind in
275275
set_option trace.grind.debug.proof true in
276276
theorem ex1 (p : Prop) (a1 a2 a3 : Nat) : (p ↔ a2 ≤ a1) → ¬p → a2 + 3 ≤ a3 → (p ↔ a4 ≤ a3 + 2) → a1 ≤ a4 := by
277-
grind
277+
grind -order
278278

279279
/-! Propagate `cnstr = False` tests -/
280280

0 commit comments

Comments
 (0)