Skip to content

Commit

Permalink
Unused variable
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed May 7, 2024
1 parent 7254574 commit 3509232
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Data/Nat/Div.lean
Original file line number Diff line number Diff line change
Expand Up @@ -102,7 +102,7 @@ protected theorem modCore_eq_mod (x y : Nat) : Nat.modCore x y = x % y := by
exact if_neg fun ⟨hlt, hle⟩ => Nat.lt_irrefl _ (Nat.lt_of_lt_of_le hlt hle)
| 1, 0 => rw [Nat.modCore]; rfl
| 1, 1 => rw [Nat.modCore, Nat.modCore]; rfl
| 1, (y+2) => rw [Nat.modCore]; rfl
| 1, (_+2) => rw [Nat.modCore]; rfl
| (_ + 2), _ => rfl

theorem mod_eq (x y : Nat) : x % y = if 0 < y ∧ y ≤ x then (x - y) % y else x := by
Expand Down

0 comments on commit 3509232

Please sign in to comment.