Countable types #
In this file we provide basic instances of the Countable
typeclass defined elsewhere.
Definition in terms of Function.Embedding
#
Operations on Type*
s #
theorem
instUncountableProdOfNonempty
{α : Type u}
{β : Type v}
[Uncountable α]
[Nonempty β]
:
Uncountable (α × β)
theorem
instUncountableProdOfNonempty_1
{α : Type u}
{β : Type v}
[Nonempty α]
[Uncountable β]
:
Uncountable (α × β)
theorem
Sigma.uncountable
{α : Type u}
{π : α → Type w}
(a : α)
[Uncountable (π a)]
:
Uncountable (Sigma π)
theorem
instUncountableSigmaOfNonempty
{α : Type u}
{π : α → Type w}
[Nonempty α]
[∀ (a : α), Uncountable (π a)]
:
Uncountable (Sigma π)