Hausdorff–Alexandroff Theorem #
In this file, we prove the Hausdorff–Alexandroff theorem, which states that every nonempty compact metric space is a continuous image of the Cantor set.
Main theorems #
exists_nat_bool_continuous_surjective_of_compact: Hausdorff–Alexandroff Theorem.
Proof Outline #
First, note that the Cantor set is homeomorphic to ℕ → Bool, as shown in
cantorSetHomeomorphNatToBool. Therefore, in this file, we work only with the space
ℕ → Bool and refer to it as the "Cantor space".
The proof consists of three steps. Let X be a compact metric space.
- Every compact metric space is homeomorphic to a closed subset of the Hilbert cube.
This is already proved in
exists_closed_embedding_to_hilbert_cube. Using this result, we may assume thatXis a closed subset of the Hilbert cube. - We construct a continuous surjection
cantorToHilbertfrom the Cantor space to the Hilbert cube. - Taking the preimage of
Xunder this surjection, it remains to prove that any closed subset of the Cantor space is the continuous image of the Cantor space.
A continuous surjection from the Cantor space to the Hilbert cube.
Equations
- cantorToHilbert x = Pi.map (fun (x : ℕ) (b : ℕ → Bool) => Real.fromBinary b) (cantorSpaceHomeomorphNatToCantorSpace x)
Instances For
theorem
exists_nat_bool_continuous_surjective_of_compact
(X : Type u_1)
[Nonempty X]
[MetricSpace X]
[CompactSpace X]
:
∃ (f : (ℕ → Bool) → X), Continuous f ∧ Function.Surjective f
Hausdorff–Alexandroff theorem: every nonempty compact metric space is a continuous image of the Cantor set.