Documentation

Mathlib.Topology.Compactness.CompactlyCoherentSpace

Compactly coherent spaces and the k-ification #

In this file we will define compactly coherent spaces and prove basic properties about them. This is a weaker version of CompactlyGeneratedSpace. These notions agree on Hausdorff spaces. They are both referred to as compactly generated spaces in the literature.

Main definitions #

Main results #

References #

Compactly coherent spaces #

A space is a compactly coherent space if the topology is generated by the compact sets.

Instances

    A set A in a compactly coherent space is open iff for every compact set K, the intersection K ∩ A is open in K.

    A set A in a compactly coherent space is closed iff for every compact set K, the intersection K ∩ A is closed in K.

    theorem CompactlyCoherentSpace.of_isOpen {X : Type u} [TopologicalSpace X] (h : ∀ (A : Set X), (∀ (K : Set X), IsCompact KIsOpen (Subtype.val ⁻¹' A))IsOpen A) :

    If every set A is open if for every compact K the intersection K ∩ A is open in K, then the space is a compactly coherent space.

    theorem CompactlyCoherentSpace.of_isClosed {X : Type u} [TopologicalSpace X] (h : ∀ (A : Set X), (∀ (K : Set X), IsCompact KIsClosed (Subtype.val ⁻¹' A))IsClosed A) :

    If every set A is closed if for every compact K the intersection K ∩ A is closed in K, then the space is a compactly coherent space.

    Every weakly locally compact space is a compactly coherent space.

    @[deprecated CompactlyCoherentSpace.of_weaklyLocallyCompactSpace (since := "2025-05-30")]

    Alias of CompactlyCoherentSpace.of_weaklyLocallyCompactSpace.


    Every weakly locally compact space is a compactly coherent space.

    Every sequential space is a compactly coherent space.

    @[deprecated CompactlyCoherentSpace.of_sequentialSpace (since := "2025-05-30")]

    Alias of CompactlyCoherentSpace.of_sequentialSpace.


    Every sequential space is a compactly coherent space.

    In a compactly coherent space X, a set s is open iff f ⁻¹' s is open for every continuous map from a compact space.

    theorem CompactlyCoherentSpace.of_isOpen_forall_compactSpace {X : Type u} [TopologicalSpace X] (h : ∀ (s : Set X), (∀ (K : Type u) [inst : TopologicalSpace K] [CompactSpace K] (f : KX), Continuous fIsOpen (f ⁻¹' s))IsOpen s) :

    A topological space X is compactly coherent if a set s is open when f ⁻¹' s? is open for every continuous map f : K → X, where K is compact.