mathlib3 documentation

topology.algebra.open_subgroup

Open subgroups of a topological groups #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This files builds the lattice open_subgroup G of open subgroups in a topological group G, and its additive version open_add_subgroup. This lattice has a top element, the subgroup of all elements, but no bottom element in general. The trivial subgroup which is the natural candidate bottom has no reason to be open (this happens only in discrete groups).

Note that this notion is especially relevant in a non-archimedean context, for instance for p-adic groups.

Main declarations #

TODO #

@[protected, instance]
Equations
@[protected, instance]
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_add_subgroup.mem_coe_opens {G : Type u_1} [add_group G] [topological_space G] {U : open_add_subgroup G} {g : G} :
g U g U
@[simp, norm_cast]
theorem open_subgroup.mem_coe_opens {G : Type u_1} [group G] [topological_space G] {U : open_subgroup G} {g : G} :
g U g U
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_subgroup.mem_coe_subgroup {G : Type u_1} [group G] [topological_space G] {U : open_subgroup G} {g : G} :
g U g U
@[ext]
theorem open_subgroup.ext {G : Type u_1} [group G] [topological_space G] {U V : open_subgroup G} (h : (x : G), x U x V) :
U = V
@[ext]
theorem open_add_subgroup.ext {G : Type u_1} [add_group G] [topological_space G] {U V : open_add_subgroup G} (h : (x : G), x U x V) :
U = V
@[protected]
@[protected]
@[protected, instance]
Equations
@[simp]
theorem open_subgroup.mem_top {G : Type u_1} [group G] [topological_space G] (x : G) :
@[simp]
theorem open_add_subgroup.mem_top {G : Type u_1} [add_group G] [topological_space G] (x : G) :
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
@[protected, instance]
Equations
def open_subgroup.prod {G : Type u_1} [group G] [topological_space G] {H : Type u_2} [group H] [topological_space H] (U : open_subgroup G) (V : open_subgroup H) :

The product of two open subgroups as an open subgroup of the product group.

Equations

The product of two open subgroups as an open subgroup of the product group.

Equations
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_subgroup.coe_prod {G : Type u_1} [group G] [topological_space G] {H : Type u_2} [group H] [topological_space H] (U : open_subgroup G) (V : open_subgroup H) :
(U.prod V) = U ×ˢ V
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_subgroup.coe_subgroup_prod {G : Type u_1} [group G] [topological_space G] {H : Type u_2} [group H] [topological_space H] (U : open_subgroup G) (V : open_subgroup H) :
(U.prod V) = U.prod V
@[protected, instance]
Equations
@[simp, norm_cast]
theorem open_subgroup.coe_inf {G : Type u_1} [group G] [topological_space G] {U V : open_subgroup G} :
(U V) = U V
@[simp, norm_cast]
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_subgroup.coe_subgroup_inf {G : Type u_1} [group G] [topological_space G] {U V : open_subgroup G} :
(U V) = U V
@[simp, norm_cast]
theorem open_subgroup.coe_opens_inf {G : Type u_1} [group G] [topological_space G] {U V : open_subgroup G} :
(U V) = U V
@[simp, norm_cast]
@[simp]
theorem open_subgroup.mem_inf {G : Type u_1} [group G] [topological_space G] {U V : open_subgroup G} {x : G} :
x U V x U x V
@[simp]
theorem open_add_subgroup.mem_inf {G : Type u_1} [add_group G] [topological_space G] {U V : open_add_subgroup G} {x : G} :
x U V x U x V
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_subgroup.coe_subgroup_le {G : Type u_1} [group G] [topological_space G] {U V : open_subgroup G} :
U V U V

The preimage of an open_add_subgroup along a continuous add_monoid homomorphism is an open_add_subgroup.

Equations
def open_subgroup.comap {G : Type u_1} [group G] [topological_space G] {N : Type u_2} [group N] [topological_space N] (f : G →* N) (hf : continuous f) (H : open_subgroup N) :

The preimage of an open_subgroup along a continuous monoid homomorphism is an open_subgroup.

Equations
@[simp, norm_cast]
@[simp, norm_cast]
theorem open_subgroup.coe_comap {G : Type u_1} [group G] [topological_space G] {N : Type u_2} [group N] [topological_space N] (H : open_subgroup N) (f : G →* N) (hf : continuous f) :
@[simp, norm_cast]
@[simp]
theorem open_subgroup.mem_comap {G : Type u_1} [group G] [topological_space G] {N : Type u_2} [group N] [topological_space N] {H : open_subgroup N} {f : G →* N} {hf : continuous f} {x : G} :
@[simp]
theorem open_add_subgroup.mem_comap {G : Type u_1} [add_group G] [topological_space G] {N : Type u_2} [add_group N] [topological_space N] {H : open_add_subgroup N} {f : G →+ N} {hf : continuous f} {x : G} :
theorem open_subgroup.comap_comap {G : Type u_1} [group G] [topological_space G] {N : Type u_2} [group N] [topological_space N] {P : Type u_3} [group P] [topological_space P] (K : open_subgroup P) (f₂ : N →* P) (hf₂ : continuous f₂) (f₁ : G →* N) (hf₁ : continuous f₁) :
open_subgroup.comap f₁ hf₁ (open_subgroup.comap f₂ hf₂ K) = open_subgroup.comap (f₂.comp f₁) _ K
theorem open_add_subgroup.comap_comap {G : Type u_1} [add_group G] [topological_space G] {N : Type u_2} [add_group N] [topological_space N] {P : Type u_3} [add_group P] [topological_space P] (K : open_add_subgroup P) (f₂ : N →+ P) (hf₂ : continuous f₂) (f₁ : G →+ N) (hf₁ : continuous f₁) :
theorem subgroup.is_open_of_mem_nhds {G : Type u_1} [group G] [topological_space G] [has_continuous_mul G] (H : subgroup G) {g : G} (hg : H nhds g) :
theorem subgroup.is_open_mono {G : Type u_1} [group G] [topological_space G] [has_continuous_mul G] {H₁ H₂ : subgroup G} (h : H₁ H₂) (h₁ : is_open H₁) :
theorem add_subgroup.is_open_mono {G : Type u_1} [add_group G] [topological_space G] [has_continuous_add G] {H₁ H₂ : add_subgroup G} (h : H₁ H₂) (h₁ : is_open H₁) :

If a subgroup of an additive topological group has 0 in its interior, then it is open.

If a subgroup of a topological group has 1 in its interior, then it is open.

@[protected, instance]
Equations
@[simp, norm_cast]
theorem submodule.is_open_mono {R : Type u_1} {M : Type u_2} [comm_ring R] [add_comm_group M] [topological_space M] [topological_add_group M] [module R M] {U P : submodule R M} (h : U P) (hU : is_open U) :
theorem ideal.is_open_of_open_subideal {R : Type u_1} [comm_ring R] [topological_space R] [topological_ring R] {U I : ideal R} (h : U I) (hU : is_open U) :