Documentation

Mathlib.Topology.Algebra.IsUniformGroup.DiscreteSubgroup

Discrete subgroups of topological groups #

Note that the instance Subgroup.isClosed_of_discrete does not live here, in order that it can be used in other files without requiring lots of group-theoretic imports.

def Subgroup.subgroupOfContinuousMulEquivOfLe {G : Type u_1} [Group G] [TopologicalSpace G] {H K : Subgroup G} (hHK : H K) :
(H.subgroupOf K) ≃ₜ* H

If G has a topology, and H ≤ K are subgroups, then H as a subgroup of K is isomorphic, as a topological group, to H as a subgroup of G. This is subgroupOfEquivOfLe upgraded to a ContinuousMulEquiv.

Equations
Instances For

    If G has a topology, and H ≤ K are subgroups, then H as a subgroup of K is isomorphic, as a topological group, to H as a subgroup of G. This is addSubgroupOfEquivOfLe upgraded to a ContinuousAddEquiv.

    Equations
    Instances For
      @[simp]

      If G is a topological group and H a finite-index subgroup, then G is topologically discrete iff H is.