Documentation

Mathlib.Topology.Compactness.LocallyCompact

Locally compact spaces #

We define the following classes of topological spaces:

  • exists_compact_mem_nhds : ∀ (x : X), s, IsCompact s s nhds x

    Every point of a weakly locally compact space admits a compact neighborhood.

We say that a topological space is a weakly locally compact space, if each point of this space admits a compact neighborhood.

Instances
    theorem exists_compact_superset {X : Type u_1} [TopologicalSpace X] [WeaklyLocallyCompactSpace X] {K : Set X} (hK : IsCompact K) :
    K', IsCompact K' K interior K'

    In a weakly locally compact space, every compact set is contained in the interior of a compact set.

    In a weakly locally compact space, the filters 𝓝 x and cocompact X are disjoint for all X.

    • local_compact_nhds : ∀ (x : X) (n : Set X), n nhds xs, s nhds x s n IsCompact s

      In a locally compact space, every neighbourhood of every point contains a compact neighbourhood of that same point.

    There are various definitions of "locally compact space" in the literature, which agree for Hausdorff spaces but not in general. This one is the precise condition on X needed for the evaluation map C(X, Y) × X → Y to be continuous for all Y when C(X, Y) is given the compact-open topology.

    See also WeaklyLocallyCompactSpace, a typeclass that only assumes that each point has a compact neighborhood.

    Instances
      theorem compact_basis_nhds {X : Type u_1} [TopologicalSpace X] [LocallyCompactSpace X] (x : X) :
      Filter.HasBasis (nhds x) (fun s => s nhds x IsCompact s) fun s => s
      theorem local_compact_nhds {X : Type u_1} [TopologicalSpace X] [LocallyCompactSpace X] {x : X} {n : Set X} (h : n nhds x) :
      s, s nhds x s n IsCompact s
      theorem locallyCompactSpace_of_hasBasis {X : Type u_1} [TopologicalSpace X] {ι : XType u_4} {p : (x : X) → ι xProp} {s : (x : X) → ι xSet X} (h : ∀ (x : X), Filter.HasBasis (nhds x) (p x) (s x)) (hc : ∀ (x : X) (i : ι x), p x iIsCompact (s x i)) :
      instance Pi.locallyCompactSpace_of_finite {ι : Type u_3} {X : ιType u_4} [(i : ι) → TopologicalSpace (X i)] [∀ (i : ι), LocallyCompactSpace (X i)] [Finite ι] :
      LocallyCompactSpace ((i : ι) → X i)

      In general it suffices that all but finitely many of the spaces are compact, but that's not straightforward to state and use.

      Equations
      instance Pi.locallyCompactSpace {ι : Type u_3} {X : ιType u_4} [(i : ι) → TopologicalSpace (X i)] [∀ (i : ι), LocallyCompactSpace (X i)] [∀ (i : ι), CompactSpace (X i)] :
      LocallyCompactSpace ((i : ι) → X i)

      For spaces that are not Hausdorff.

      Equations
      theorem exists_compact_subset {X : Type u_1} [TopologicalSpace X] [LocallyCompactSpace X] {x : X} {U : Set X} (hU : IsOpen U) (hx : x U) :
      K, IsCompact K x interior K K U

      A reformulation of the definition of locally compact space: In a locally compact space, every open set containing x has a compact subset containing x in its interior.

      theorem exists_compact_between {X : Type u_1} [TopologicalSpace X] [hX : LocallyCompactSpace X] {K : Set X} {U : Set X} (hK : IsCompact K) (hU : IsOpen U) (h_KU : K U) :
      L, IsCompact L K interior L L U

      In a locally compact space, for every containment K ⊆ U of a compact set K in an open set U, there is a compact neighborhood L such that K ⊆ L ⊆ U: equivalently, there is a compact L such that K ⊆ interior L and L ⊆ U.