Skip to content

Commit 030aad1

Browse files
committed
chore: offset for simp weakening
1 parent 6b873c6 commit 030aad1

File tree

1 file changed

+2
-1
lines changed

1 file changed

+2
-1
lines changed

src/Init/Data/Int/DivMod/Lemmas.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1353,6 +1353,7 @@ theorem tdiv_ofNat_eq_zero_iff_natAbs_lt_or_eq_zero {a : Int} {b : Nat} :
13531353
· simpa using this _
13541354
· obtain ⟨n, hn⟩ := exists_eq_neg_ofNat (show -[a+1] ≤ 0 by omega)
13551355
simp [hn, this]
1356+
apply this
13561357
intro a
13571358
rw [Int.tdiv_eq_ediv_of_nonneg (by omega)]
13581359
norm_cast
@@ -1374,7 +1375,7 @@ than the absolute value of the denominator, or the denominator is zero.
13741375
· obtain ⟨b, rfl⟩ := eq_ofNat_of_zero_le (show 0 ≤ b by omega)
13751376
norm_cast
13761377
apply Int.tdiv_ofNat_eq_zero_iff_natAbs_lt_or_eq_zero
1377-
1378+
13781379
/-! ### tmod -/
13791380

13801381
-- `tmod` analogues of `emod` lemmas from `Bootstrap.lean`

0 commit comments

Comments
 (0)