Skip to content

Commit f2501be

Browse files
committed
test
1 parent 65541c8 commit f2501be

File tree

1 file changed

+12
-0
lines changed

1 file changed

+12
-0
lines changed

tests/lean/run/grind_linarith_2.lean

Lines changed: 12 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -64,3 +64,15 @@ example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
6464
example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
6565
: c = a → a + b ≤ 33 ≤ b + c → a + b = 3 := by
6666
grind
67+
68+
/--
69+
trace: [grind.linarith.model] a := 7/2
70+
[grind.linarith.model] b := 1
71+
[grind.linarith.model] c := 2
72+
[grind.linarith.model] d := 3
73+
-/
74+
#guard_msgs (drop error, trace) in
75+
set_option trace.grind.linarith.model true in
76+
example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c d : α)
77+
: b ≥ 0 → c > b → d > b → a ≠ b + c → a > b + c → a < b + d → False := by
78+
grind

0 commit comments

Comments
 (0)