Documentation

Mathlib.Analysis.Normed.Group.Quotient

Quotients of seminormed groups #

For any SeminormedAddCommGroup M and any S : AddSubgroup M, we provide a SeminormedAddCommGroup, the group quotient M ⧸ S. If S is closed, we provide NormedAddCommGroup (M ⧸ S) (regardless of whether M itself is separated). The two main properties of these structures are the underlying topology is the quotient topology and the projection is a normed group homomorphism which is norm non-increasing (better, it has operator norm exactly one unless S is dense in M). The corresponding universal property is that every normed group hom defined on M which vanishes on S descends to a normed group hom defined on M ⧸ S.

This file also introduces a predicate IsQuotient characterizing normed group homs that are isomorphic to the canonical projection onto a normed group quotient.

In addition, this file also provides normed structures for quotients of modules by submodules, and of (commutative) rings by ideals. The SeminormedAddCommGroup and NormedAddCommGroup instances described above are transferred directly, but we also define instances of NormedSpace, SeminormedCommRing, NormedCommRing and NormedAlgebra under appropriate type class assumptions on the original space. Moreover, while QuotientAddGroup.completeSpace works out-of-the-box for quotients of NormedAddCommGroups by AddSubgroups, we need to transfer this instance in Submodule.Quotient.completeSpace so that it applies to these other quotients.

Main definitions #

We use M and N to denote seminormed groups and S : AddSubgroup M. All the following definitions are in the AddSubgroup namespace. Hence we can access AddSubgroup.normedMk S as S.normedMk.

Main results #

Implementation details #

For any SeminormedAddCommGroup M and any S : AddSubgroup M we define a norm on M ⧸ S by ‖x‖ = sInf (norm '' {m | mk' S m = x}). This formula is really an implementation detail, it shouldn't be needed outside of this file setting up the theory.

Since M ⧸ S is automatically a topological space (as any quotient of a topological space), one needs to be careful while defining the SeminormedAddCommGroup instance to avoid having two different topologies on this quotient. This is not purely a technological issue. Mathematically there is something to prove. The main point is proved in the auxiliary lemma quotient_nhd_basis that has no use beyond this verification and states that zero in the quotient admits as basis of neighborhoods in the quotient topology the sets {x | ‖x‖ < ε} for positive ε.

Once this mathematical point is settled, we have two topologies that are propositionally equal. This is not good enough for the type class system. As usual we ensure definitional equality using forgetful inheritance, see Note [forgetful inheritance]. A (semi)-normed group structure includes a uniform space structure which includes a topological space structure, together with propositional fields asserting compatibility conditions. The usual way to define a SeminormedAddCommGroup is to let Lean build a uniform space structure using the provided norm, and then trivially build a proof that the norm and uniform structure are compatible. Here the uniform structure is provided using TopologicalAddGroup.toUniformSpace which uses the topological structure and the group structure to build the uniform structure. This uniform structure induces the correct topological structure by construction, but the fact that it is compatible with the norm is not obvious; this is where the mathematical content explained in the previous paragraph kicks in.

noncomputable instance normOnQuotient {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) :
Norm (M S)

The definition of the norm on the quotient by an additive subgroup.

Equations
theorem AddSubgroup.quotient_norm_eq {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) :
x = sInf (norm '' {m : M | m = x})
theorem QuotientAddGroup.norm_eq_infDist {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) :
x = Metric.infDist 0 {m : M | m = x}
theorem QuotientAddGroup.norm_mk {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M) :

An alternative definition of the norm on the quotient group: the norm of ((x : M) : M ⧸ S) is equal to the distance from x to S.

theorem image_norm_nonempty {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) :
Set.Nonempty (norm '' {m : M | (QuotientAddGroup.mk' S) m = x})
theorem bddBelow_image_norm {M : Type u_1} [SeminormedAddCommGroup M] (s : Set M) :
BddBelow (norm '' s)
theorem isGLB_quotient_norm {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) :
IsGLB (norm '' {m : M | (QuotientAddGroup.mk' S) m = x}) x
theorem quotient_norm_neg {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) :

The norm on the quotient satisfies ‖-x‖ = ‖x‖.

theorem quotient_norm_sub_rev {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) (y : M S) :
x - y = y - x

The norm of the projection is smaller or equal to the norm of the original element.

theorem quotient_norm_mk_le' {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) (m : M) :

The norm of the projection is smaller or equal to the norm of the original element.

theorem quotient_norm_mk_eq {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) (m : M) :
(QuotientAddGroup.mk' S) m = sInf ((fun (x : M) => m + x) '' S)

The norm of the image under the natural morphism to the quotient.

theorem quotient_norm_nonneg {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) (x : M S) :

The quotient norm is nonnegative.

The quotient norm is nonnegative.

The norm of the image of m : M in the quotient by S is zero if and only if m belongs to the closure of S.

theorem QuotientAddGroup.norm_lt_iff {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} {x : M S} {r : } :
x < r ∃ (m : M), m = x m < r
theorem norm_mk_lt {M : Type u_1} [SeminormedAddCommGroup M] {S : AddSubgroup M} (x : M S) {ε : } (hε : 0 < ε) :
∃ (m : M), (QuotientAddGroup.mk' S) m = x m < x + ε

For any x : M ⧸ S and any 0 < ε, there is m : M such that mk' S m = x and ‖m‖ < ‖x‖ + ε.

theorem norm_mk_lt' {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) (m : M) {ε : } (hε : 0 < ε) :
∃ s ∈ S, m + s < (QuotientAddGroup.mk' S) m + ε

For any m : M and any 0 < ε, there is s ∈ S such that ‖m + s‖ < ‖mk' S m‖ + ε.

theorem quotient_norm_add_le {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) (x : M S) (y : M S) :

The quotient norm satisfies the triangle inequality.

theorem norm_mk_zero {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) :

The quotient norm of 0 is 0.

theorem norm_mk_eq_zero {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) (hS : IsClosed S) (m : M) (h : (QuotientAddGroup.mk' S) m = 0) :
m S

If (m : M) has norm equal to 0 in M ⧸ S for a closed subgroup S of M, then m ∈ S.

theorem quotient_nhd_basis {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) :
Filter.HasBasis (nhds 0) (fun (ε : ) => 0 < ε) fun (ε : ) => {x : M S | x < ε}

The seminormed group structure on the quotient by an additive subgroup.

Equations

The quotient in the category of normed groups.

Equations
noncomputable def AddSubgroup.normedMk {M : Type u_1} [SeminormedAddCommGroup M] (S : AddSubgroup M) :

The morphism from a seminormed group to the quotient by a subgroup.

Equations
Instances For

    The operator norm of the projection is at most 1.

    The operator norm of the projection is 1 if the subspace is not dense.

    The operator norm of the projection is 0 if the subspace is dense.

    IsQuotient f, for f : M ⟶ N means that N is isomorphic to the quotient of M by the kernel of f.

    Instances For
      noncomputable def NormedAddGroupHom.lift {M : Type u_1} [SeminormedAddCommGroup M] {N : Type u_3} [SeminormedAddCommGroup N] (S : AddSubgroup M) (f : NormedAddGroupHom M N) (hf : sS, f s = 0) :

      Given f : NormedAddGroupHom M N such that f s = 0 for all s ∈ S, where, S : AddSubgroup M is closed, the induced morphism NormedAddGroupHom (M ⧸ S) N.

      Equations
      Instances For
        theorem NormedAddGroupHom.lift_mk {M : Type u_1} [SeminormedAddCommGroup M] {N : Type u_3} [SeminormedAddCommGroup N] (S : AddSubgroup M) (f : NormedAddGroupHom M N) (hf : sS, f s = 0) (m : M) :
        theorem NormedAddGroupHom.IsQuotient.norm_lift {M : Type u_1} {N : Type u_2} [SeminormedAddCommGroup M] [SeminormedAddCommGroup N] {f : NormedAddGroupHom M N} (hquot : NormedAddGroupHom.IsQuotient f) {ε : } (hε : 0 < ε) (n : N) :
        ∃ (m : M), f m = n m < n + ε
        theorem NormedAddGroupHom.lift_norm_le {M : Type u_1} [SeminormedAddCommGroup M] {N : Type u_3} [SeminormedAddCommGroup N] (S : AddSubgroup M) (f : NormedAddGroupHom M N) (hf : sS, f s = 0) {c : NNReal} (fb : f c) :

        Submodules and ideals #

        In what follows, the norm structures created above for quotients of (semi)NormedAddCommGroups by AddSubgroups are transferred via definitional equality to quotients of modules by submodules, and of rings by ideals, thereby preserving the definitional equality for the topological group and uniform structures worked for above. Completeness is also transferred via this definitional equality.

        In addition, instances are constructed for NormedSpace, SeminormedCommRing, NormedCommRing and NormedAlgebra under the appropriate hypotheses. Currently, we do not have quotients of rings by two-sided ideals, hence the commutativity hypotheses are required.

        Equations
        • =
        theorem Submodule.Quotient.norm_mk_lt {M : Type u_1} [SeminormedAddCommGroup M] {R : Type u_3} [Ring R] [Module R M] {S : Submodule R M} (x : M S) {ε : } (hε : 0 < ε) :
        ∃ (m : M), Submodule.Quotient.mk m = x m < x + ε

        For any x : M ⧸ S and any 0 < ε, there is m : M such that Submodule.Quotient.mk m = x and ‖m‖ < ‖x‖ + ε.

        instance Submodule.Quotient.instBoundedSMul {M : Type u_1} [SeminormedAddCommGroup M] {R : Type u_3} [Ring R] [Module R M] (S : Submodule R M) (𝕜 : Type u_4) [SeminormedCommRing 𝕜] [Module 𝕜 M] [BoundedSMul 𝕜 M] [SMul 𝕜 R] [IsScalarTower 𝕜 R M] :
        BoundedSMul 𝕜 (M S)
        Equations
        • =
        instance Submodule.Quotient.normedSpace {M : Type u_1} [SeminormedAddCommGroup M] {R : Type u_3} [Ring R] [Module R M] (S : Submodule R M) (𝕜 : Type u_4) [NormedField 𝕜] [NormedSpace 𝕜 M] [SMul 𝕜 R] [IsScalarTower 𝕜 R M] :
        NormedSpace 𝕜 (M S)
        Equations
        theorem Ideal.Quotient.norm_mk_lt {R : Type u_3} [SeminormedCommRing R] {I : Ideal R} (x : R I) {ε : } (hε : 0 < ε) :
        ∃ (r : R), (Ideal.Quotient.mk I) r = x r < x + ε
        instance Ideal.Quotient.normedAlgebra {R : Type u_3} [SeminormedCommRing R] (I : Ideal R) (𝕜 : Type u_4) [NormedField 𝕜] [NormedAlgebra 𝕜 R] :
        NormedAlgebra 𝕜 (R I)
        Equations