Uniform structure on topological groups
topological_add_group.to_uniform_space
andtopological_add_group_is_uniform
can be used to construct a canonical uniformity for a topological add group.extension of ℤ-bilinear maps to complete groups (useful for ring completions)
add_group_with_zero_nhd
: construct the topological structure from a group with a neighbourhood around zero. Then withtopological_add_group.to_uniform_space
one can derive auniform_space
.
- uniform_continuous_sub : uniform_continuous (λ (p : α × α), p.fst - p.snd)
A uniform (additive) group is a group in which the addition and negation are uniformly continuous.
Equations
Equations
Equations
- topological_add_group.to_uniform_space G = {to_topological_space := _inst_2, to_core := {uniformity := filter.comap (λ (p : G × G), p.snd - p.fst) (nhds 0), refl := _, symm := _, comp := _}, is_open_uniformity := _}
- add_left : ∀ (a a' : α) (b : β), f (a + a', b) = f (a, b) + f (a', b)
- add_right : ∀ (a : α) (b b' : β), f (a, b + b') = f (a, b) + f (a, b')
Instances
Equations
- _ = _
Bourbaki GT III.6.5 Theorem I: ℤ-bilinear continuous maps from dense images into a complete Hausdorff group extend by continuity. Note: Bourbaki assumes that α and β are also complete Hausdorff, but this is not necessary.