- to_has_continuous_add : has_continuous_add α
- continuous_neg : continuous (λ (a : α), -a)
A topological (additive) group is a group in which the addition and negation operations are continuous.
Instances
- uniform_add_group.to_topological_add_group
- add_group_with_zero_nhd.topological_add_group
- topological_ring.to_topological_add_group
- normed_top_group
- prod.topological_add_group
- topological_add_group_quotient
- real.topological_add_group
- rat.topological_add_group
- complex.topological_add_group
- tangent_space.topological_add_group
- to_has_continuous_mul : has_continuous_mul α
- continuous_inv : continuous (λ (a : α), a⁻¹)
A topological group is a group in which the multiplication and inversion operations are continuous.
If a function converges to a value in a multiplicative topological group, then its inverse
converges to the inverse of this value. For the version in normed fields assuming additionally
that the limit is nonzero, use tendsto.inv'
.
Equations
Equations
- homeomorph.mul_left a = {to_equiv := {to_fun := (equiv.mul_left a).to_fun, inv_fun := (equiv.mul_left a).inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Equations
- homeomorph.mul_right a = {to_equiv := {to_fun := (equiv.mul_right a).to_fun, inv_fun := (equiv.mul_right a).inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Equations
- homeomorph.inv α = {to_equiv := {to_fun := (equiv.inv α).to_fun, inv_fun := (equiv.inv α).inv_fun, left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Equations
- _ = _
- to_add_comm_group : add_comm_group α
- Z : filter α
- zero_Z : has_pure.pure 0 ≤ add_group_with_zero_nhd.Z α
- sub_Z : filter.tendsto (λ (p : α × α), p.fst - p.snd) ((add_group_with_zero_nhd.Z α).prod (add_group_with_zero_nhd.Z α)) (add_group_with_zero_nhd.Z α)
additive group with a neighbourhood around 0. Only used to construct a topology and uniform space.
This is currently only available for commutative groups, but it can be extended to non-commutative groups too.
Equations
- add_group_with_zero_nhd.topological_space α = topological_space.mk_of_nhds (λ (a : α), filter.map (λ (x : α), x + a) (add_group_with_zero_nhd.Z α))
Equations
Equations
Some results about an open set containing the product of two sets in a topological group.
Given a open neighborhood U
of 0
there is a open neighborhood V
of 0
such that V + V ⊆ U
.
Given a open neighborhood U
of 1
there is a open neighborhood V
of 1
such that VV ⊆ U
.
Given a compact set K
inside an open set U
, there is a open neighborhood V
of 0
such that K + V ⊆ U
.
Given a compact set K
inside an open set U
, there is a open neighborhood V
of 1
such that KV ⊆ U
.
A compact set is covered by finitely many left multiplicative translates of a set with non-empty interior.
A compact set is covered by finitely many left additive translates of a set with non-empty interior.