We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 65541c8 commit f2501beCopy full SHA for f2501be
tests/lean/run/grind_linarith_2.lean
@@ -64,3 +64,15 @@ example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
64
example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
65
: c = a → a + b ≤ 3 → 3 ≤ b + c → a + b = 3 := by
66
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