Documentation

Mathlib.Analysis.Normed.Group.HomCompletion

Completion of normed group homs #

Given two (semi) normed groups G and H and a normed group hom f : NormedAddGroupHom G H, we build and study a normed group hom f.completion : NormedAddGroupHom (completion G) (completion H) such that the diagram

                   f
     G       ----------->     H

     |                        |
     |                        |
     |                        |
     V                        V

completion G -----------> completion H
            f.completion

commutes. The map itself comes from the general theory of completion of uniform spaces, but here we want a normed group hom, study its operator norm and kernel.

The vertical maps in the above diagrams are also normed group homs constructed in this file.

Main definitions and results: #

The normed group hom induced between completions.

Equations
Instances For
    theorem NormedAddGroupHom.completion_coe {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] (f : NormedAddGroupHom G H) (g : G) :
    f.completion g = (f g)

    Completion of normed group homs as a normed group hom.

    Equations
    Instances For
      @[simp]
      theorem normedAddGroupHomCompletionHom_apply {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] (f : NormedAddGroupHom G H) :
      normedAddGroupHomCompletionHom f = f.completion
      theorem NormedAddGroupHom.completion_comp {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] {K : Type u_3} [SeminormedAddCommGroup K] (f : NormedAddGroupHom G H) (g : NormedAddGroupHom H K) :
      g.completion.comp f.completion = (g.comp f).completion
      theorem NormedAddGroupHom.completion_neg {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] (f : NormedAddGroupHom G H) :
      (-f).completion = -f.completion
      theorem NormedAddGroupHom.completion_add {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] (f g : NormedAddGroupHom G H) :
      (f + g).completion = f.completion + g.completion
      theorem NormedAddGroupHom.completion_sub {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] (f g : NormedAddGroupHom G H) :
      (f - g).completion = f.completion - g.completion

      The map from a normed group to its completion, as a normed group hom.

      Equations
      Instances For
        @[simp]
        theorem NormedAddCommGroup.toCompl_apply {G : Type u_1} [SeminormedAddCommGroup G] (a✝ : G) :
        toCompl a✝ = a✝
        theorem NormedAddGroupHom.ker_completion {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] {f : NormedAddGroupHom G H} {C : } (h : f.SurjectiveOnWith f.range C) :
        f.completion.ker = closure (NormedAddCommGroup.toCompl.comp (incl f.ker)).range

        If H is complete, the extension of f : NormedAddGroupHom G H to a NormedAddGroupHom (completion G) H.

        Equations
        Instances For
          @[simp]
          theorem NormedAddGroupHom.extension_coe {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] [T0Space H] [CompleteSpace H] (f : NormedAddGroupHom G H) (v : G) :
          f.extension v = f v
          theorem NormedAddGroupHom.extension_unique {G : Type u_1} [SeminormedAddCommGroup G] {H : Type u_2} [SeminormedAddCommGroup H] [T0Space H] [CompleteSpace H] (f : NormedAddGroupHom G H) {g : NormedAddGroupHom (UniformSpace.Completion G) H} (hg : ∀ (v : G), f v = g v) :
          f.extension = g