Documentation

Mathlib.Data.Countable.Basic

Countable types #

In this file we provide basic instances of the Countable typeclass defined elsewhere.

Definition in terms of Function.Embedding #

theorem Function.Embedding.countable {α : Sort u} {β : Sort v} [Countable β] (f : α β) :
theorem Function.Embedding.uncountable {α : Sort u} {β : Sort v} [Uncountable α] (f : α β) :

Operations on Type*s #

instance instCountableSum {α : Type u} {β : Type v} [Countable α] [Countable β] :
Countable (α β)
instance Sum.uncountable_inl {α : Type u} {β : Type v} [Uncountable α] :
instance Sum.uncountable_inr {α : Type u} {β : Type v} [Uncountable β] :
@[simp]
theorem untopD_coe_enat (d n : ) :
WithTop.untopD d n = n
instance instCountableProd {α : Type u} {β : Type v} [Countable α] [Countable β] :
Countable (α × β)
instance instUncountableProdOfNonempty {α : Type u} {β : Type v} [Uncountable α] [Nonempty β] :
Uncountable (α × β)
instance instUncountableProdOfNonempty_1 {α : Type u} {β : Type v} [Nonempty α] [Uncountable β] :
Uncountable (α × β)
theorem countable_left_of_prod_of_nonempty {α : Type u} {β : Type v} [Nonempty β] (h : Countable (α × β)) :
theorem countable_right_of_prod_of_nonempty {α : Type u} {β : Type v} [Nonempty α] (h : Countable (α × β)) :
theorem countable_prod_swap {α : Type u} {β : Type v} [Countable (α × β)] :
Countable (β × α)
instance instCountableSigma {α : Type u} {π : αType w} [Countable α] [∀ (a : α), Countable (π a)] :
theorem Sigma.uncountable {α : Type u} {π : αType w} (a : α) [Uncountable (π a)] :
instance instUncountableSigmaOfNonempty {α : Type u} {π : αType w} [Nonempty α] [∀ (a : α), Uncountable (π a)] :
@[instance 500]
instance SetCoe.countable {α : Type u} [Countable α] (s : Set α) :

Operations on Sort*s #

instance instCountablePSum {α : Sort u} {β : Sort v} [Countable α] [Countable β] :
Countable (α ⊕' β)
instance instCountablePProd {α : Sort u} {β : Sort v} [Countable α] [Countable β] :
Countable (α ×' β)
instance instCountablePSigma {α : Sort u} {π : αSort w} [Countable α] [∀ (a : α), Countable (π a)] :
instance instCountableForallOfFinite {α : Sort u} {π : αSort w} [Finite α] [∀ (a : α), Countable (π a)] :
Countable ((a : α) → π a)