mathlib3 documentation

set_theory.cardinal.schroeder_bernstein

Schröder-Bernstein theorem, well-ordering of cardinals #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file proves the Schröder-Bernstein theorem (see schroeder_bernstein), the well-ordering of cardinals (see min_injective) and the totality of their order (see total).

Notes #

Cardinals are naturally ordered by α ≤ β ↔ ∃ f : a → β, injective f:

Cardinals are defined and further developed in the file set_theory.cardinal.

theorem function.embedding.schroeder_bernstein {α : Type u} {β : Type v} {f : α β} {g : β α} (hf : function.injective f) (hg : function.injective g) :

The Schröder-Bernstein Theorem: Given injections α → β and β → α, we can get a bijection α → β.

theorem function.embedding.antisymm {α : Type u} {β : Type v} :
β) α) nonempty β)

The Schröder-Bernstein Theorem: Given embeddings α ↪ β and β ↪ α, there exists an equivalence α ≃ β.

theorem function.embedding.min_injective {ι : Type u} (β : ι Type v) [I : nonempty ι] :
(i : ι), nonempty (Π (j : ι), β i β j)

The cardinals are well-ordered. We express it here by the fact that in any set of cardinals there is an element that injects into the others. See cardinal.linear_order for (one of) the lattice instances.

theorem function.embedding.total (α : Type u) (β : Type v) :
nonempty β) nonempty α)

The cardinals are totally ordered. See cardinal.linear_order for (one of) the lattice instance.