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 6b8291a commit 8b6ec8aCopy full SHA for 8b6ec8a
src/Init/Data/Range/Polymorphic/NatLemmas.lean
@@ -573,10 +573,12 @@ theorem induct_rcc_right (motive : Nat → Nat → Prop)
573
(base : ∀ a b, b < a → motive a b)
574
(step : ∀ a b, a ≤ b → motive a b → motive a (b + 1))
575
(a b : Nat) : motive a b := by
576
- apply induct_rco_right (fun a b => motive a (b + 1))
577
induction h : b + 1 - a generalizing a b
578
· apply base; omega
579
· rename_i d ih
+ match b with
580
+ | 0 =>
581
+ have : a = 0 := by omega
582
583
obtain ⟨b, rfl⟩ := Nat.exists_eq_succ_of_ne_zero (show b ≠ 0 by omega)
584
apply step
0 commit comments