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 83ad3a2 commit 4df5cf4Copy full SHA for 4df5cf4
tests/lean/run/grind_order_eq.lean
@@ -0,0 +1,11 @@
1
+open Lean Grind Std
2
+
3
+example [LE α] [IsPartialOrder α] (a b : α) (f : α → Nat) : a ≤ b → b ≤ c → c ≤ a → f a = f b := by
4
+ grind (splits := 0)
5
6
+example [CommRing α] [LE α] [LT α] [LawfulOrderLT α] [IsPartialOrder α] [OrderedRing α]
7
+ (a b : α) (f : α → Int) : a ≤ b + 1 → b ≤ a - 1 → f a = f (2 + b - 1) := by
8
+ grind -mbtc -lia -linarith (splits := 0)
9
10
+example (a b : Int) (f : Int → Int) : a ≤ b + 1 → b ≤ a - 1 → f a = f (2 + b - 1) := by
11
0 commit comments