Documentation

Mathlib.Topology.Algebra.ClosedSubgroup

Closed subgroups of a topological group #

This files builds the SemilatticeInf ClosedSubgroup G of closed subgroups in a topological group G, and its additive version ClosedAddSubgroup.

Main definitions and results #

structure ClosedSubgroup (G : Type u) [Group G] [TopologicalSpace G] extends Subgroup G :

The type of closed subgroups of a topological group.

Instances For
    theorem ClosedSubgroup.ext {G : Type u} {inst✝ : Group G} {inst✝¹ : TopologicalSpace G} {x y : ClosedSubgroup G} (carrier : (↑x).carrier = (↑y).carrier) :
    x = y
    structure ClosedAddSubgroup (G : Type u) [AddGroup G] [TopologicalSpace G] extends AddSubgroup G :

    The type of closed subgroups of an additive topological group.

    Instances For
      theorem ClosedAddSubgroup.ext {G : Type u} {inst✝ : AddGroup G} {inst✝¹ : TopologicalSpace G} {x y : ClosedAddSubgroup G} (carrier : (↑x).carrier = (↑y).carrier) :
      x = y
      Equations
      Equations
      Equations
      Equations
      Equations
      Equations
      theorem Subgroup.normalCore_isClosed {G : Type u} [Group G] [TopologicalSpace G] [ContinuousMul G] (H : Subgroup G) (h : IsClosed H) :
      IsClosed H.normalCore
      theorem Subgroup.isOpen_of_isClosed_of_finiteIndex {G : Type u} [Group G] [TopologicalSpace G] [ContinuousMul G] (H : Subgroup G) [H.FiniteIndex] (h : IsClosed H) :
      IsOpen H