Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 665dede

Browse files
refactor(data/int/basic): weaken hypotheses for int.induction_on
1 parent 07aa1e3 commit 665dede

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/data/int/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -95,7 +95,7 @@ theorem le_sub_one_iff {a b : ℤ} : a ≤ b - 1 ↔ a < b :=
9595
le_sub_iff_add_le
9696

9797
@[elab_as_eliminator] protected lemma induction_on {p : ℤ → Prop}
98-
(i : ℤ) (hz : p 0) (hp : ∀i, p i → p (i + 1)) (hn : ∀i, p i → p (i - 1)) : p i :=
98+
(i : ℤ) (hz : p 0) (hp : ∀i : ℕ, p i → p (i + 1)) (hn : ∀i : ℕ, p (-i) → p (-i - 1)) : p i :=
9999
begin
100100
induction i,
101101
{ induction i,

0 commit comments

Comments
 (0)