Skip to content

Commit 0620221

Browse files
committed
feat: Add grind_pattern on Nat.mod_eq_of_lt
1 parent 088f8b0 commit 0620221

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/Init/Data/Nat/Div/Basic.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -179,6 +179,9 @@ theorem mod_eq_of_lt {a b : Nat} (h : a < b) : a % b = a :=
179179
if_neg h'
180180
(mod_eq a b).symm ▸ this
181181

182+
grind_pattern mod_eq_of_lt => a % b where
183+
guard (a < b)
184+
182185
@[simp] theorem one_mod_eq_zero_iff {n : Nat} : 1 % n = 0 ↔ n = 1 := by
183186
match n with
184187
| 0 => simp

0 commit comments

Comments
 (0)