Pointwise operations on sets in topological groups #
Topological operations on pointwise sums and products #
A few results about interior and closure of the pointwise addition/multiplication of sets in groups
with continuous addition/multiplication. See also Submonoid.top_closure_mul_self_eq
in
Topology.Algebra.Monoid
.
One may expect a version of IsClosed.smul_left_of_isCompact
where t
is compact and s
is
closed, but such a lemma can't be true in this level of generality. For a counterexample, consider
ℚ
acting on ℝ
by translation, and let s : Set ℚ := univ
, t : set ℝ := {0}
. Then s
is
closed and t
is compact, but s +ᵥ t
is the set of all rationals, which is definitely not
closed in ℝ
.
To fix the proof, we would need to make two additional assumptions:
- for any
x ∈ t
,s • {x}
is closed - for any
x ∈ t
, there is a continuous functiong : s • {x} → s
such that, for ally ∈ s • {x}
, we havey = (g y) • x
These are fairly specific hypotheses so we don't state this version of the lemmas, but an interesting fact is that these two assumptions are verified in the case of anIsTopologicalAddTorsor
. We prove this special case inIsClosed.vadd_right_of_isCompact
.
Given a neighborhood U
of the identity, one may find a neighborhood V
of the identity which
is closed, symmetric, and satisfies V * V ⊆ U
.
Given a neighborhood U
of the identity, one may find a neighborhood V
of the
identity which is closed, symmetric, and satisfies V + V ⊆ U
.
If a point in a topological group has a compact neighborhood, then the group is locally compact.
If a function defined on a topological group has a support contained in a compact set, then either the function is trivial or the group is locally compact.
If a function defined on a topological additive group has a support contained in a compact set, then either the function is trivial or the group is locally compact.
If a function defined on a topological group has compact support, then either the function is trivial or the group is locally compact.
If a function defined on a topological additive group has compact support, then either the function is trivial or the group is locally compact.