Documentation

Mathlib.SetTheory.Cardinal.ToNat

Projection from cardinal numbers to natural numbers #

In this file we define Cardinal.toNat to be the natural projection Cardinal → ℕ, sending all infinite cardinals to zero. We also prove basic lemmas about this definition.

This function sends finite cardinals to the corresponding natural, and infinite cardinals to 0.

Equations
Instances For
    @[simp]
    theorem Cardinal.toNat_ofENat (n : ℕ∞) :
    Cardinal.toNat n = n.toNat
    @[simp]

    Two finite cardinals are equal iff they are equal their Cardinal.toNat projections are equal.

    @[deprecated Cardinal.toNat_le_toNat]
    @[deprecated Cardinal.toNat_lt_toNat]
    @[deprecated Cardinal.toNat_natCast]
    theorem Cardinal.toNat_cast (n : ) :

    Alias of Cardinal.toNat_natCast.

    @[simp]
    theorem Cardinal.toNat_ofNat (n : ) [n.AtLeastTwo] :

    toNat has a right-inverse: coercion.

    theorem Cardinal.toNat_eq_iff {c : Cardinal.{u}} {n : } (hn : n 0) :
    Cardinal.toNat c = n c = n

    A version of toNat_eq_iff for literals

    @[deprecated map_prod]
    theorem Cardinal.toNat_finset_prod {α : Type u} (s : Finset α) (f : αCardinal.{u_1}) :
    Cardinal.toNat (∏ is, f i) = is, Cardinal.toNat (f i)