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 19e1fe5 commit 2143f85Copy full SHA for 2143f85
src/Init/Data/Int/LemmasAux.lean
@@ -62,7 +62,17 @@ theorem natCast_succ_pos (n : Nat) : 0 < (n.succ : Int) := natCast_pos.2 n.succ_
62
63
@[simp high] theorem natCast_nonpos_iff {n : Nat} : (n : Int) ≤ 0 ↔ n = 0 := by omega
64
65
-@[simp, norm_cast] theorem cast_id {n : Int} : Int.cast n = n := rfl
+@[simp, norm_cast, grind =] theorem cast_id {n : Int} : Int.cast n = n := rfl
66
+
67
+end Int
68
69
+namespace Nat
70
71
+@[simp, norm_cast, grind =] theorem cast_id (n : Nat) : Nat.cast n = n := rfl
72
73
+end Nat
74
75
+namespace Int
76
77
@[simp] theorem ble'_eq_true (a b : Int) : (Int.ble' a b = true) = (a ≤ b) := by
78
cases a <;> cases b <;> simp [Int.ble'] <;> omega
0 commit comments