Documentation

Mathlib.Topology.NatEmbedding

Infinite Hausdorff topological spaces #

In this file we prove several properties of infinite Hausdorff topological spaces.

theorem exists_seq_infinite_isOpen_pairwise_disjoint (X : Type u_1) [TopologicalSpace X] [T2Space X] [Infinite X] :
∃ (U : Set X), (∀ (n : ), (U n).Infinite) (∀ (n : ), IsOpen (U n)) Pairwise (Function.onFun Disjoint U)

In an infinite Hausdorff topological space, there exists a sequence of pairwise disjoint infinite open sets.

If X is an infinite Hausdorff topological space, then there exists a topological embedding f : ℕ → X.

Note: this theorem is true for an infinite KC-space but the proof in that case is different.

If X is an infinite Hausdorff topological space, then there exists an infinite set s : Set X that has the induced topology is the discrete topology.