Documentation

Mathlib.Deprecated.Cardinal.Finite

Deprecated material on PartENat.card. #

@[deprecated ENat.card]
def PartENat.card (α : Type u_1) :

PartENat.card α is the cardinality of α as an extended natural number. If α is infinite, PartENat.card α = ⊤.

Equations
Instances For
    @[simp]
    theorem PartENat.card_sum (α : Type u_1) (β : Type u_2) :
    theorem PartENat.card_congr {α : Type u_1} {β : Type u_2} (f : α β) :
    @[simp]
    theorem PartENat.card_image_of_injOn {α : Type u} {β : Type v} {f : αβ} {s : Set α} (h : Set.InjOn f s) :
    theorem PartENat.card_image_of_injective {α : Type u} {β : Type v} (f : αβ) (s : Set α) (h : Function.Injective f) :
    @[deprecated ENat.card_eq_coe_natCard]
    theorem PartENat.card_eq_coe_natCard (α : Type u_1) [Finite α] :
    @[deprecated PartENat.card_eq_coe_natCard]
    theorem PartENat.card_eq_coe_nat_card (α : Type u_1) [Finite α] :

    Alias of PartENat.card_eq_coe_natCard.