Documentation

Mathlib.Topology.Algebra.Group.Quotient

Topology on the quotient group #

In this file we define topology on G ⧸ N, where N is a subgroup of G, and prove basic properties of this topology.

@[simp]
theorem QuotientGroup.dense_image_mk {G : Type u_1} [TopologicalSpace G] [Group G] [ContinuousMul G] {N : Subgroup G} {s : Set G} :
Dense (mk '' s) Dense (s * N)
instance QuotientGroup.instT1Space {G : Type u_1} [TopologicalSpace G] [Group G] [ContinuousMul G] {N : Subgroup G} [hN : IsClosed N] :
T1Space (G N)

The quotient of a topological group G by a closed subgroup N is T1.

When G is normal, this implies (because G ⧸ N is a topological group) that the quotient is T3 (see QuotientGroup.instT3Space).

Back to the general case, we will show later that the quotient is in fact T2 since N acts on G properly.

instance QuotientAddGroup.instT1Space {G : Type u_1} [TopologicalSpace G] [AddGroup G] [ContinuousAdd G] {N : AddSubgroup G} [hN : IsClosed N] :
T1Space (G N)

The quotient of a topological additive group G by a closed subgroup N is T1.

When G is normal, this implies (because G ⧸ N is a topological additive group) that the quotient is T3 (see QuotientAddGroup.instT3Space).

Back to the general case, we will show later that the quotient is in fact T2 since N acts on G properly.

A quotient of a locally compact group is locally compact.

theorem QuotientGroup.nhds_eq {G : Type u_1} [TopologicalSpace G] [Group G] [ContinuousMul G] (N : Subgroup G) (x : G) :

Neighborhoods in the quotient are precisely the map of neighborhoods in the prequotient.

theorem QuotientAddGroup.nhds_eq {G : Type u_1} [TopologicalSpace G] [AddGroup G] [ContinuousAdd G] (N : AddSubgroup G) (x : G) :

Neighborhoods in the quotient are precisely the map of neighborhoods in the prequotient.

The quotient of a second countable topological group by a subgroup is second countable.

The quotient of a second countable additive topological group by a subgroup is second countable.

instance QuotientGroup.instT3Space {G : Type u_1} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] (N : Subgroup G) [N.Normal] [hN : IsClosed N] :
T3Space (G N)