Skip to content

Commit

Permalink
doc(topology/algebra/*): explanation of relation between `uniform_gro…
Browse files Browse the repository at this point in the history
…up` and `topological_group` (#13151)

Adding some comments on how to use `uniform_group` and `topological_group`.
  • Loading branch information
mcdoll committed Apr 5, 2022
1 parent 429c6e3 commit 21c48e1
Show file tree
Hide file tree
Showing 2 changed files with 16 additions and 2 deletions.
8 changes: 6 additions & 2 deletions src/topology/algebra/group.lean
Expand Up @@ -11,7 +11,7 @@ import topology.sets.compacts
import topology.algebra.constructions

/-!
# Theory of topological groups
# Topological groups
This file defines the following typeclasses:
Expand Down Expand Up @@ -330,7 +330,11 @@ class topological_add_group (G : Type u) [topological_space G] [add_group G]
extends has_continuous_add G, has_continuous_neg G : Prop

/-- A topological group is a group in which the multiplication and inversion operations are
continuous. -/
continuous.
When you declare an instance that does not already have a `uniform_space` instance,
you should also provide an instance of `uniform_space` and `uniform_group` using
`topological_group.to_uniform_space` and `topological_group_is_uniform`. -/
@[to_additive]
class topological_group (G : Type*) [topological_space G] [group G]
extends has_continuous_mul G, has_continuous_inv G : Prop
Expand Down
10 changes: 10 additions & 0 deletions src/topology/algebra/uniform_group.lean
Expand Up @@ -12,6 +12,16 @@ import tactic.abel
/-!
# Uniform structure on topological groups
This file defines uniform groups and its additive counterpart. These typeclasses should be
preferred over using `[topological_space α] [topological_group α]` since every topological
group naturally induces a uniform structure.
## Main declarations
* `uniform_group` and `uniform_add_group`: Multiplicative and additive uniform groups, that
i.e., groups with uniformly continuous `(*)` and `(⁻¹)` / `(+)` and `(-)`.
## Main results
* `topological_add_group.to_uniform_space` and `topological_add_group_is_uniform` can be used to
construct a canonical uniformity for a topological add group.
Expand Down

0 comments on commit 21c48e1

Please sign in to comment.