Documentation

Mathlib.Analysis.Normed.Group.Subgroup

Subgroups of normed (semi)groups #

In this file, we prove that subgroups of a normed (semi)group are also normed (semi)groups.

Tags #

normed group

Subgroups of normed groups #

A subgroup of a seminormed group is also a seminormed group, with the restriction of the norm.

Equations

A subgroup of a seminormed group is also a seminormed group, with the restriction of the norm.

Equations
@[simp]
theorem Subgroup.coe_norm {E : Type u_1} [SeminormedGroup E] {s : Subgroup E} (x : s) :

If x is an element of a subgroup s of a seminormed group E, its norm in s is equal to its norm in E.

@[simp]
theorem AddSubgroup.coe_norm {E : Type u_1} [SeminormedAddGroup E] {s : AddSubgroup E} (x : s) :

If x is an element of a subgroup s of a seminormed group E, its norm in s is equal to its norm in E.

theorem Subgroup.norm_coe {E : Type u_1} [SeminormedGroup E] {s : Subgroup E} (x : s) :

If x is an element of a subgroup s of a seminormed group E, its norm in s is equal to its norm in E.

This is a reversed version of the simp lemma Subgroup.coe_norm for use by norm_cast.

theorem AddSubgroup.norm_coe {E : Type u_1} [SeminormedAddGroup E] {s : AddSubgroup E} (x : s) :

If x is an element of a subgroup s of a seminormed group E, its norm in s is equal to its norm in E.

This is a reversed version of the simp lemma AddSubgroup.coe_norm for use by norm_cast.

Subgroup classes of normed groups #

@[instance 75]
instance SubgroupClass.seminormedGroup {E : Type u_1} [SeminormedGroup E] {S : Type u_2} [SetLike S E] [SubgroupClass S E] (s : S) :

A subgroup of a seminormed group is also a seminormed group, with the restriction of the norm.

Equations
@[instance 75]

A subgroup of a seminormed additive group is also a seminormed additive group, with the restriction of the norm.

Equations
@[simp]
theorem SubgroupClass.coe_norm {E : Type u_1} [SeminormedGroup E] {S : Type u_2} [SetLike S E] [SubgroupClass S E] (s : S) (x : s) :

If x is an element of a subgroup s of a seminormed group E, its norm in s is equal to its norm in E.

@[simp]
theorem AddSubgroupClass.coe_norm {E : Type u_1} [SeminormedAddGroup E] {S : Type u_2} [SetLike S E] [AddSubgroupClass S E] (s : S) (x : s) :

If x is an element of an additive subgroup s of a seminormed additive group E, its norm in s is equal to its norm in E.

@[instance 75]
instance SubgroupClass.normedGroup {E : Type u_1} [NormedGroup E] {S : Type u_2} [SetLike S E] [SubgroupClass S E] (s : S) :
Equations
@[instance 75]
instance AddSubgroupClass.normedAddGroup {E : Type u_1} [NormedAddGroup E] {S : Type u_2} [SetLike S E] [AddSubgroupClass S E] (s : S) :
Equations
@[instance 75]
instance SubgroupClass.normedCommGroup {E : Type u_1} [NormedCommGroup E] {S : Type u_2} [SetLike S E] [SubgroupClass S E] (s : S) :
Equations