Documentation

Mathlib.Topology.Compactness.SigmaCompact

Sigma-compactness in topological spaces #

Main definitions #

def IsSigmaCompact {α : Type u} [TopologicalSpace α] (s : Set α) :

A subset s ⊆ α is called σ-compact if it is the union of countably many compact sets.

Equations
Instances For
    theorem IsCompact.isSigmaCompact {α : Type u} [TopologicalSpace α] {s : Set α} (hs : IsCompact s) :

    Compact sets are σ-compact.

    @[simp]

    The empty set is σ-compact.

    theorem isSigmaCompact_iUnion_of_isCompact {α : Type u} [TopologicalSpace α] {ι : Type u_3} [hι : Countable ι] (s : ιSet α) (hcomp : ∀ (i : ι), IsCompact (s i)) :
    IsSigmaCompact (⋃ i, s i)

    Countable unions of compact sets are σ-compact.

    theorem isSigmaCompact_sUnion_of_isCompact {α : Type u} [TopologicalSpace α] {S : Set (Set α)} (hc : Set.Countable S) (hcomp : ∀ (s : Set α), s SIsCompact s) :

    Countable unions of compact sets are σ-compact.

    theorem isSigmaCompact_iUnion {α : Type u} [TopologicalSpace α] {ι : Type u_3} [Countable ι] (s : ιSet α) (hcomp : ∀ (i : ι), IsSigmaCompact (s i)) :
    IsSigmaCompact (⋃ i, s i)

    Countable unions of σ-compact sets are σ-compact.

    theorem isSigmaCompact_sUnion {α : Type u} [TopologicalSpace α] (S : Set (Set α)) (hc : Set.Countable S) (hcomp : ∀ (s : S), IsSigmaCompact s) :

    Countable unions of σ-compact sets are σ-compact.

    theorem isSigmaCompact_biUnion {α : Type u} [TopologicalSpace α] {ι : Type u_3} {s : Set ι} {S : ιSet α} (hc : Set.Countable s) (hcomp : ∀ (i : ι), i sIsSigmaCompact (S i)) :
    IsSigmaCompact (⋃ i ∈ s, S i)

    Countable unions of σ-compact sets are σ-compact.

    theorem IsSigmaCompact.of_isClosed_subset {α : Type u} [TopologicalSpace α] {s : Set α} {t : Set α} (ht : IsSigmaCompact t) (hs : IsClosed s) (h : s t) :

    A closed subset of a σ-compact set is σ-compact.

    theorem IsSigmaCompact.image_of_continuousOn {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} (hs : IsSigmaCompact s) (hf : ContinuousOn f s) :

    If s is σ-compact and f is continuous on s, f(s) is σ-compact.

    theorem IsSigmaCompact.image {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} (hf : Continuous f) {s : Set α} (hs : IsSigmaCompact s) :

    If s is σ-compact and f continuous, f(s) is σ-compact.

    theorem Inducing.isSigmaCompact_iff {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} (hf : Inducing f) :

    If f : X → Y is Inducing, the image f '' s of a set s is σ-compact if and only s is σ-compact.

    theorem Embedding.isSigmaCompact_iff {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} {s : Set α} (hf : Embedding f) :

    If f : X → Y is an Embedding, the image f '' s of a set s is σ-compact if and only s is σ-compact.

    theorem Subtype.isSigmaCompact_iff {α : Type u} [TopologicalSpace α] {p : αProp} {s : Set { a // p a }} :

    Sets of subtype are σ-compact iff the image under a coercion is.

    A σ-compact space is a space that is the union of a countable collection of compact subspaces. Note that a locally compact separable T₂ space need not be σ-compact. The sequence can be extracted using compactCovering.

    Instances

      A topological space is σ-compact iff univ is σ-compact.

      In a σ-compact space, univ is σ-compact.

      theorem SigmaCompactSpace_iff_exists_compact_covering {α : Type u} [TopologicalSpace α] :
      SigmaCompactSpace α K, (∀ (n : ), IsCompact (K n)) ⋃ n, K n = Set.univ

      A topological space is σ-compact iff there exists a countable collection of compact subspaces that cover the entire space.

      theorem SigmaCompactSpace.exists_compact_covering {α : Type u} [TopologicalSpace α] [h : SigmaCompactSpace α] :
      K, (∀ (n : ), IsCompact (K n)) ⋃ n, K n = Set.univ
      theorem isSigmaCompact_range {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] {f : αβ} (hf : Continuous f) [SigmaCompactSpace α] :

      If X is σ-compact, im f is σ-compact.

      A subset s is σ-compact iff s (with the subspace topology) is a σ-compact space.

      theorem SigmaCompactSpace.of_countable {α : Type u} [TopologicalSpace α] (S : Set (Set α)) (Hc : Set.Countable S) (Hcomp : ∀ (s : Set α), s SIsCompact s) (HU : ⋃₀ S = Set.univ) :

      A choice of compact covering for a σ-compact space, chosen to be monotone.

      Equations
      Instances For
        theorem iUnion_compactCovering (α : Type u) [TopologicalSpace α] [SigmaCompactSpace α] :
        ⋃ n, compactCovering α n = Set.univ
        theorem compactCovering_subset (α : Type u) [TopologicalSpace α] [SigmaCompactSpace α] ⦃m : ⦃n : (h : m n) :
        theorem LocallyFinite.countable_univ {α : Type u} [TopologicalSpace α] [SigmaCompactSpace α] {ι : Type u_3} {f : ιSet α} (hf : LocallyFinite f) (hne : ∀ (i : ι), Set.Nonempty (f i)) :
        Set.Countable Set.univ

        If α is a σ-compact space, then a locally finite family of nonempty sets of α can have only countably many elements, Set.Countable version.

        noncomputable def LocallyFinite.encodable {α : Type u} [TopologicalSpace α] [SigmaCompactSpace α] {ι : Type u_3} {f : ιSet α} (hf : LocallyFinite f) (hne : ∀ (i : ι), Set.Nonempty (f i)) :

        If f : ι → Set α is a locally finite covering of a σ-compact topological space by nonempty sets, then the index type ι is encodable.

        Equations
        Instances For
          theorem countable_cover_nhdsWithin_of_sigma_compact {α : Type u} [TopologicalSpace α] [SigmaCompactSpace α] {f : αSet α} {s : Set α} (hs : IsClosed s) (hf : ∀ (x : α), x sf x nhdsWithin x s) :
          t x, Set.Countable t s ⋃ x ∈ t, f x

          In a topological space with sigma compact topology, if f is a function that sends each point x of a closed set s to a neighborhood of x within s, then for some countable set t ⊆ s, the neighborhoods f x, x ∈ t, cover the whole set s.

          theorem countable_cover_nhds_of_sigma_compact {α : Type u} [TopologicalSpace α] [SigmaCompactSpace α] {f : αSet α} (hf : ∀ (x : α), f x nhds x) :
          s, Set.Countable s ⋃ x ∈ s, f x = Set.univ

          In a topological space with sigma compact topology, if f is a function that sends each point x to a neighborhood of x, then for some countable set s, the neighborhoods f x, x ∈ s, cover the whole space.

          structure CompactExhaustion (X : Type u_3) [TopologicalSpace X] :
          Type u_3

          An exhaustion by compact sets of a topological space is a sequence of compact sets K n such that K n ⊆ interior (K (n + 1)) and ⋃ n, K n = univ.

          If X is a locally compact sigma compact space, then CompactExhaustion.choice X provides a choice of an exhaustion by compact sets. This choice is also available as (default : CompactExhaustion X).

          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            @[simp]
            theorem CompactExhaustion.toFun_eq_coe {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) :
            K.toFun = K
            theorem CompactExhaustion.subset_interior_succ {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) (n : ) :
            K n interior (K (n + 1))
            theorem CompactExhaustion.subset {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) ⦃m : ⦃n : (h : m n) :
            K m K n
            theorem CompactExhaustion.subset_succ {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) (n : ) :
            K n K (n + 1)
            theorem CompactExhaustion.subset_interior {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) ⦃m : ⦃n : (h : m < n) :
            K m interior (K n)
            theorem CompactExhaustion.iUnion_eq {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) :
            ⋃ n, K n = Set.univ
            theorem CompactExhaustion.exists_mem {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) (x : α) :
            n, x K n
            noncomputable def CompactExhaustion.find {α : Type u} [TopologicalSpace α] (K : CompactExhaustion α) (x : α) :

            The minimal n such that x ∈ K n.

            Equations
            Instances For

              Prepend the empty set to a compact exhaustion K n.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For

                A choice of an exhaustion by compact sets of a weakly locally compact σ-compact space.

                Equations
                Instances For
                  Equations