Documentation

Mathlib.Topology.Algebra.Group.Pointwise

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.

theorem subset_interior_smul {α : Type u} {β : Type v} [TopologicalSpace β] [Group α] [MulAction α β] [ContinuousConstSMul α β] {s : Set α} {t : Set β} [TopologicalSpace α] :
theorem subset_interior_vadd {α : Type u} {β : Type v} [TopologicalSpace β] [AddGroup α] [AddAction α β] [ContinuousConstVAdd α β] {s : Set α} {t : Set β} [TopologicalSpace α] :
theorem IsClosed.smul_left_of_isCompact {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] [Group α] [MulAction α β] [ContinuousInv α] [ContinuousSMul α β] {s : Set α} {t : Set β} (ht : IsClosed t) (hs : IsCompact s) :
theorem IsClosed.vadd_left_of_isCompact {α : Type u} {β : Type v} [TopologicalSpace α] [TopologicalSpace β] [AddGroup α] [AddAction α β] [ContinuousNeg α] [ContinuousVAdd α β] {s : Set α} {t : Set β} (ht : IsClosed t) (hs : IsCompact s) :

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:

theorem IsOpen.mul_left {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul α α] {s t : Set α} :
IsOpen tIsOpen (s * t)
theorem IsOpen.add_left {α : Type u} [TopologicalSpace α] [AddGroup α] [ContinuousConstVAdd α α] {s t : Set α} :
IsOpen tIsOpen (s + t)
theorem subset_interior_mul_right {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul α α] {s t : Set α} :
s * interior t interior (s * t)
theorem subset_interior_mul {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul α α] {s t : Set α} :
theorem singleton_mul_mem_nhds {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul α α] {s : Set α} (a : α) {b : α} (h : s nhds b) :
{a} * s nhds (a * b)
theorem singleton_add_mem_nhds {α : Type u} [TopologicalSpace α] [AddGroup α] [ContinuousConstVAdd α α] {s : Set α} (a : α) {b : α} (h : s nhds b) :
{a} + s nhds (a + b)
theorem singleton_mul_mem_nhds_of_nhds_one {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul α α] {s : Set α} (a : α) (h : s nhds 1) :
{a} * s nhds a
theorem singleton_add_mem_nhds_of_nhds_zero {α : Type u} [TopologicalSpace α] [AddGroup α] [ContinuousConstVAdd α α] {s : Set α} (a : α) (h : s nhds 0) :
{a} + s nhds a
theorem IsOpen.mul_right {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul αᵐᵒᵖ α] {s t : Set α} (hs : IsOpen s) :
IsOpen (s * t)
theorem IsOpen.add_right {α : Type u} [TopologicalSpace α] [AddGroup α] [ContinuousConstVAdd αᵃᵒᵖ α] {s t : Set α} (hs : IsOpen s) :
IsOpen (s + t)
theorem mul_singleton_mem_nhds {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul αᵐᵒᵖ α] {s : Set α} (a : α) {b : α} (h : s nhds b) :
s * {a} nhds (b * a)
theorem add_singleton_mem_nhds {α : Type u} [TopologicalSpace α] [AddGroup α] [ContinuousConstVAdd αᵃᵒᵖ α] {s : Set α} (a : α) {b : α} (h : s nhds b) :
s + {a} nhds (b + a)
theorem mul_singleton_mem_nhds_of_nhds_one {α : Type u} [TopologicalSpace α] [Group α] [ContinuousConstSMul αᵐᵒᵖ α] {s : Set α} (a : α) (h : s nhds 1) :
s * {a} nhds a
theorem add_singleton_mem_nhds_of_nhds_zero {α : Type u} [TopologicalSpace α] [AddGroup α] [ContinuousConstVAdd αᵃᵒᵖ α] {s : Set α} (a : α) (h : s nhds 0) :
s + {a} nhds a
theorem IsOpen.div_left {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {s t : Set G} (ht : IsOpen t) :
IsOpen (s / t)
theorem IsOpen.sub_left {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {s t : Set G} (ht : IsOpen t) :
IsOpen (s - t)
theorem IsOpen.div_right {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {s t : Set G} (hs : IsOpen s) :
IsOpen (s / t)
theorem IsOpen.sub_right {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {s t : Set G} (hs : IsOpen s) :
IsOpen (s - t)
theorem IsOpen.mul_closure {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {s : Set G} (hs : IsOpen s) (t : Set G) :
s * closure t = s * t
theorem IsOpen.add_closure {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {s : Set G} (hs : IsOpen s) (t : Set G) :
s + closure t = s + t
theorem IsOpen.closure_mul {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {t : Set G} (ht : IsOpen t) (s : Set G) :
closure s * t = s * t
theorem IsOpen.closure_add {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {t : Set G} (ht : IsOpen t) (s : Set G) :
closure s + t = s + t
theorem IsOpen.div_closure {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {s : Set G} (hs : IsOpen s) (t : Set G) :
s / closure t = s / t
theorem IsOpen.sub_closure {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {s : Set G} (hs : IsOpen s) (t : Set G) :
s - closure t = s - t
theorem IsOpen.closure_div {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {t : Set G} (ht : IsOpen t) (s : Set G) :
closure s / t = s / t
theorem IsOpen.closure_sub {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {t : Set G} (ht : IsOpen t) (s : Set G) :
closure s - t = s - t
theorem IsClosed.mul_left_of_isCompact {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {s t : Set G} (ht : IsClosed t) (hs : IsCompact s) :
IsClosed (s * t)
theorem IsTopologicalGroup.t2Space_of_one_sep {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] (H : ∀ (x : G), x 1Unhds 1, xU) :
theorem IsTopologicalAddGroup.t2Space_of_zero_sep {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] (H : ∀ (x : G), x 0Unhds 0, xU) :
theorem exists_closed_nhds_one_inv_eq_mul_subset {G : Type w} [TopologicalSpace G] [Group G] [IsTopologicalGroup G] {U : Set G} (hU : U nhds 1) :
Vnhds 1, IsClosed V V⁻¹ = V 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.

theorem exists_closed_nhds_zero_neg_eq_add_subset {G : Type w} [TopologicalSpace G] [AddGroup G] [IsTopologicalAddGroup G] {U : Set G} (hU : U nhds 0) :
Vnhds 0, IsClosed V -V = V 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.