File tree Expand file tree Collapse file tree 1 file changed +26
-0
lines changed
Expand file tree Collapse file tree 1 file changed +26
-0
lines changed Original file line number Diff line number Diff line change @@ -38,3 +38,29 @@ set_option trace.grind.debug.linarith.search.assign true in
3838example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c d : α)
3939 : b ≥ 0 → c > b → d > b → a ≠ b + c → a > b + c → a < b + d → False := by
4040 grind
41+
42+ example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c d : α)
43+ : a ≤ b → a ≥ c + d → d = 0 → b = c → a = b := by
44+ grind
45+
46+ example [IntModule α] [LinearOrder α] [IntModule.IsOrdered α] (a b c d : α)
47+ : a ≤ b → a ≥ c + d → d ≤ 0 → d ≥ 0 → b = c → a = b := by
48+ grind
49+
50+ open Linarith RArray
51+ set_option trace.grind.debug.proof true in
52+ example [IntModule α] [LinearOrder α] [IntModule.IsOrdered α] (a b c d : α)
53+ : a ≤ b → a - c ≥ 0 + d → d ≤ 0 → d ≥ 0 → b = c → a ≠ b → False := by
54+ grind
55+
56+ example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
57+ : a + 2 *b = 0 → c + b = -b → a = c := by
58+ grind
59+
60+ example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
61+ : a + 2 *b = 0 → a = c → c + b = -b := by
62+ grind
63+
64+ example [CommRing α] [LinearOrder α] [Ring.IsOrdered α] (a b c : α)
65+ : c = a → a + b ≤ 3 → 3 ≤ b + c → a + b = 3 := by
66+ grind
You can’t perform that action at this time.
0 commit comments