Completions of normed groups #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file contains an API for completions of seminormed groups (basic facts about objects and morphisms).
Main definitions #
SemiNormedGroup.Completion : SemiNormedGroup ⥤ SemiNormedGroup
: the completion of a seminormed group (defined as a functor onSemiNormedGroup
to itself).SemiNormedGroup.Completion.lift (f : V ⟶ W) : (Completion.obj V ⟶ W)
: a normed group hom fromV
to completeW
extends ("lifts") to a seminormed group hom from the completion ofV
toW
.
Projects #
- Construct the category of complete seminormed groups, say
CompleteSemiNormedGroup
and promote theCompletion
functor below to a functor landing in this category. - Prove that the functor
Completion : SemiNormedGroup ⥤ CompleteSemiNormedGroup
is left adjoint to the forgetful functor.
The completion of a seminormed group, as an endofunctor on SemiNormedGroup
.
Equations
- SemiNormedGroup.Completion = {obj := λ (V : SemiNormedGroup), SemiNormedGroup.of (uniform_space.completion ↥V), map := λ (V W : SemiNormedGroup) (f : V ⟶ W), normed_add_group_hom.completion f, map_id' := SemiNormedGroup.Completion._proof_1, map_comp' := SemiNormedGroup.Completion._proof_2}
Instances for SemiNormedGroup.Completion
The canonical morphism from a seminormed group V
to its completion.
Given a normed group hom V ⟶ W
, this defines the associated morphism
from the completion of V
to the completion of W
.
The difference from the definition obtained from the functoriality of completion is in that the
map sending a morphism f
to the associated morphism of completions is itself additive.
Equations
- SemiNormedGroup.category_theory.preadditive = {hom_group := λ (P Q : SemiNormedGroup), infer_instance, add_comp' := SemiNormedGroup.category_theory.preadditive._proof_1, comp_add' := SemiNormedGroup.category_theory.preadditive._proof_2}
Given a normed group hom f : V → W
with W
complete, this provides a lift of f
to
the completion of V
. The lemmas lift_unique
and lift_comp_incl
provide the api for the
universal property of the completion.
Equations
- SemiNormedGroup.Completion.lift f = {to_fun := ⇑(normed_add_group_hom.extension f), map_add' := _, bound' := _}