Definition and notation for extended natural numbers #
Extended natural numbers ℕ∞ = WithTop ℕ
.
Equations
- «termℕ∞» = Lean.ParserDescr.node `«termℕ∞» 1024 (Lean.ParserDescr.symbol "ℕ∞")
Instances For
Recursor for ENat
using the preferred forms ⊤
and ↑a
.
Equations
- ENat.recTopCoe top coe none = top
- ENat.recTopCoe top coe (some a) = coe a
Instances For
@[simp]
theorem
ENat.recTopCoe_top
{C : ℕ∞ → Sort u_1}
(d : C ⊤)
(f : (a : ℕ) → C ↑a)
:
ENat.recTopCoe d f ⊤ = d
@[simp]
theorem
ENat.recTopCoe_coe
{C : ℕ∞ → Sort u_1}
(d : C ⊤)
(f : (a : ℕ) → C ↑a)
(x : ℕ)
:
ENat.recTopCoe d f ↑x = f x