Documentation

Mathlib.Topology.MetricSpace.HausdorffAlexandroff

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 #

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.

  1. 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 that X is a closed subset of the Hilbert cube.
  2. We construct a continuous surjection cantorToHilbert from the Cantor space to the Hilbert cube.
  3. Taking the preimage of X under this surjection, it remains to prove that any closed subset of the Cantor space is the continuous image of the Cantor space.
noncomputable def Real.fromBinary :
(Bool)unitInterval

Convert a sequence of binary digits to a real number from unitInterval.

Equations
Instances For
    noncomputable def cantorToHilbert (x : Bool) :

    A continuous surjection from the Cantor space to the Hilbert cube.

    Equations
    Instances For
      theorem exists_retractionCantorSet {X : Set (Bool)} (h_closed : IsClosed X) (h_nonempty : X.Nonempty) :
      ∃ (f : (Bool)Bool), Continuous f Set.range f = X

      Hausdorff–Alexandroff theorem: every nonempty compact metric space is a continuous image of the Cantor set.