Documentation

SphereEversion.ToMathlib.Data.Nat.Basic

theorem exists_by_induction {α : Type u_1} {P : αProp} (h₀ : (a : α), P 0 a) (ih : ∀ (n : ) (a : α), P n a (a' : α), P (n + 1) a') :
(f : α), ∀ (n : ), P n (f n)
theorem exists_by_induction' {α : Type u_1} (P : αProp) (Q : ααProp) (h₀ : (a : α), P 0 a) (ih : ∀ (n : ) (a : α), P n a (a' : α), P (n + 1) a' Q n a a') :
(f : α), ∀ (n : ), P n (f n) Q n (f n) (f (n + 1))