Documentation

Mathlib.Topology.Separation.Profinite

Separation properties: profinite spaces #

A T1 space with a clopen basis is totally separated.

theorem nhds_basis_clopen {X : Type u_1} [TopologicalSpace X] [T2Space X] [CompactSpace X] [TotallyDisconnectedSpace X] (x : X) :
(nhds x).HasBasis (fun (s : Set X) => x s IsClopen s) id
theorem compact_exists_isClopen_in_isOpen {X : Type u_1} [TopologicalSpace X] [T2Space X] [CompactSpace X] [TotallyDisconnectedSpace X] {x : X} {U : Set X} (is_open : IsOpen U) (memU : x U) :
∃ (V : Set X), IsClopen V x V V U

Every member of an open set in a compact Hausdorff totally disconnected space is contained in a clopen set contained in the open set.

A locally compact Hausdorff totally disconnected space has a basis with clopen elements.

A locally compact Hausdorff space is totally disconnected if and only if it is totally separated.

@[deprecated loc_compact_t2_tot_disc_iff_tot_sep]

Alias of loc_compact_t2_tot_disc_iff_tot_sep.


A locally compact Hausdorff space is totally disconnected if and only if it is totally separated.

@[instance 100]

A totally disconnected compact Hausdorff space is totally separated.