Documentation

Mathlib.Topology.Separation.CompletelyRegular

Completely regular topological spaces. #

This file defines CompletelyRegularSpace and T35Space.

Main definitions #

Main results #

Completely regular spaces #

T₃.₅ spaces #

Implementation notes #

The present definition CompletelyRegularSpace is a slight modification of the one given in [russell1974]. There it's assumed that any point x ∈ Kᶜ is separated from the closed set K by a continuous real valued function f (as opposed to f being unit-interval-valued). This can be converted to the present definition by replacing a real-valued f by h ∘ g ∘ f, with g : x ↦ max(x, 0) and h : x ↦ min(x, 1). Some sources (e.g. [russell1974]) also assume that a completely regular space is T₁. Here a completely regular space that is also T₁ is called a T₃.₅ space.

References #

A space is completely regular if points can be separated from closed sets via continuous functions to the unit interval.

Instances
    theorem completelyRegularSpace_iff (X : Type u) [TopologicalSpace X] :
    CompletelyRegularSpace X ∀ (x : X) (K : Set X), IsClosed KxK∃ (f : XunitInterval), Continuous f f x = 0 Set.EqOn f 1 K
    theorem completelyRegularSpace_iff_isOpen {X : Type u} [TopologicalSpace X] :
    CompletelyRegularSpace X ∀ (x : X) (K : Set X), IsOpen Kx K∃ (f : XunitInterval), Continuous f f x = 0 Set.EqOn f 1 K
    theorem CompletelyRegularSpace.completely_regular_isOpen {X : Type u} [TopologicalSpace X] [CompletelyRegularSpace X] (x : X) (K : Set X) :
    IsOpen Kx K∃ (f : XunitInterval), Continuous f f x = 0 Set.EqOn f 1 K
    theorem completelyRegularSpace_iInf {ι : Type u_1} {X : Type u_2} {t : ιTopologicalSpace X} (ht : ∀ (i : ι), CompletelyRegularSpace X) :
    instance instCompletelyRegularSpaceForall {ι : Type u_1} {X : ιType u_2} [t : (i : ι) → TopologicalSpace (X i)] [ht : ∀ (i : ι), CompletelyRegularSpace (X i)] :
    CompletelyRegularSpace ((i : ι) → X i)

    A T₃.₅ space is a completely regular space that is also T₀.

    Instances
      theorem Topology.IsEmbedding.t35Space {X : Type u} [TopologicalSpace X] {Y : Type v} [TopologicalSpace Y] [T35Space Y] {f : XY} (hf : IsEmbedding f) :
      instance instT35SpaceSubtype {X : Type u} [TopologicalSpace X] {p : XProp} [T35Space X] :
      instance instT35SpaceForall {ι : Type u_1} {X : ιType u_2} [t : (i : ι) → TopologicalSpace (X i)] [ht : ∀ (i : ι), T35Space (X i)] :
      T35Space ((i : ι) → X i)
      instance instT35SpaceProd {X : Type u_1} {Y : Type u_2} [tX : TopologicalSpace X] [tY : TopologicalSpace Y] [htX : T35Space X] [htY : T35Space Y] :
      T35Space (X × Y)
      @[deprecated separatesPoints_continuous_of_t35Space (since := "2025-04-13")]

      Alias of separatesPoints_continuous_of_t35Space.

      @[deprecated separatesPoints_continuous_of_t35Space_Icc (since := "2025-04-13")]

      Alias of separatesPoints_continuous_of_t35Space_Icc.

      @[deprecated injective_stoneCechUnit_of_t35Space (since := "2025-04-13")]

      Alias of injective_stoneCechUnit_of_t35Space.