mathlib3 documentation

analysis.normed.group.SemiNormedGroup.completion

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 #

Projects #

  1. Construct the category of complete seminormed groups, say CompleteSemiNormedGroup and promote the Completion functor below to a functor landing in this category.
  2. 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
Instances for SemiNormedGroup.Completion

The canonical morphism from a seminormed group V to its completion.

Equations

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
@[protected, instance]
Equations

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