The category of uniform spaces
We construct the category of uniform spaces, show that the complete separated uniform spaces form a reflective subcategory, and hence possess all limits that uniform spaces do.
TODO: show that uniform spaces actually have all limits!
A (bundled) uniform space.
Equations
The information required to build morphisms for UniformSpace
.
Equations
- x.uniform_space = x.str
Construct a bundled UniformSpace
from the underlying type and the typeclass.
Equations
- UniformSpace.of α = {α := α, str := _inst_1}
Equations
Equations
- X.has_coe_to_fun Y = {F := λ (_x : X ⟶ Y), ↥X → ↥Y, coe := (category_theory.forget UniformSpace).map Y}
The forgetful functor from uniform spaces to topological spaces.
Equations
- UniformSpace.has_forget_to_Top = {forget₂ := {obj := λ (X : UniformSpace), Top.of ↥X, map := λ (X Y : UniformSpace) (f : X ⟶ Y), {to_fun := ⇑f, continuous_to_fun := _}, map_id' := UniformSpace.has_forget_to_Top._proof_2, map_comp' := UniformSpace.has_forget_to_Top._proof_3}, forget_comp := UniformSpace.has_forget_to_Top._proof_4}
- α : Type ?
- is_uniform_space : uniform_space c.α
- is_complete_space : complete_space c.α
- is_separated : separated_space c.α
A (bundled) complete separated uniform space.
Equations
- CpltSepUniformSpace.has_coe_to_sort = {S := Type u, coe := CpltSepUniformSpace.α}
Equations
Construct a bundled UniformSpace
from the underlying type and the appropriate typeclasses.
Equations
Equations
- CpltSepUniformSpace.inhabited = {default := CpltSepUniformSpace.of empty CpltSepUniformSpace.inhabited._proof_2}
The category instance on CpltSepUniformSpace
.
The concrete category instance on CpltSepUniformSpace
.
The functor turning uniform spaces into complete separated uniform spaces.
Equations
- UniformSpace.completion_functor = {obj := λ (X : UniformSpace), CpltSepUniformSpace.of (uniform_space.completion ↥X), map := λ (X Y : UniformSpace) (f : X ⟶ Y), ⟨uniform_space.completion.map f.val, _⟩, map_id' := UniformSpace.completion_functor._proof_8, map_comp' := UniformSpace.completion_functor._proof_9}
The inclusion of a uniform space into its completion.
Equations
- X.completion_hom = ⟨coe coe_to_lift, _⟩
The mate of a morphism from a UniformSpace
to a CpltSepUniformSpace
.
Equations
The completion functor is left adjoint to the forgetful functor.
Equations
- UniformSpace.adj = category_theory.adjunction.mk_of_hom_equiv {hom_equiv := λ (X : UniformSpace) (Y : CpltSepUniformSpace), {to_fun := λ (f : UniformSpace.completion_functor.obj X ⟶ Y), X.completion_hom ≫ f, inv_fun := λ (f : X ⟶ (category_theory.forget₂ CpltSepUniformSpace UniformSpace).obj Y), UniformSpace.extension_hom f, left_inv := _, right_inv := _}, hom_equiv_naturality_left_symm' := UniformSpace.adj._proof_3, hom_equiv_naturality_right' := UniformSpace.adj._proof_4}