Skip to content

Instantly share code, notes, and snippets.

@drhodes
Created February 10, 2024 14:35
Show Gist options
  • Save drhodes/e5767360f86fadafb25641fc8db48807 to your computer and use it in GitHub Desktop.
Save drhodes/e5767360f86fadafb25641fc8db48807 to your computer and use it in GitHub Desktop.
import Mathlib.Tactic
open Nat
theorem induction0 {P : ℕ → Prop}
(base : P 0) (step : ∀m, P m → P (succ m)) : (∀n, P n) := by
intro k
cases k with
| zero => exact base
| succ m =>
apply step
apply induction0 /- is this recursion valid? -/
exact base
exact step
done
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment