Zulip Chat Archive
Stream: Is there code for X?
Topic: pointwise ops on nhds
Adam Topaz (Aug 16 2022 at 17:04):
Does anyone know of an efficient way to prove lemmas of the following form?
import order.filter.pointwise
import topology.algebra.ring
open_locale pointwise topological_space
example {G : Type*} [topological_space G] [group G] [topological_group G]
(x y : G) : 𝓝 x * 𝓝 y ≤ 𝓝 (x * y) :=
sorry
Adam Topaz (Aug 16 2022 at 17:04):
ping @Jack McKoen
Yaël Dillies (Aug 16 2022 at 17:07):
Look for a lemma about docs#filter.map₂
Yaël Dillies (Aug 16 2022 at 17:07):
If it desn't exist, look for the set
or finset
version
Anatole Dedecker (Aug 16 2022 at 17:20):
import order.filter.pointwise
import topology.algebra.ring
open filter
open_locale pointwise topological_space
example {G : Type*} [topological_space G] [group G] [topological_group G]
(x y : G) : 𝓝 x * 𝓝 y ≤ 𝓝 (x * y) :=
begin
rw [← map₂_mul, ← map_prod_eq_map₂, ← nhds_prod_eq],
exact continuous_mul.tendsto (x, y)
end
Adam Topaz (Aug 16 2022 at 17:22):
Nice! Thanks!
Last updated: Dec 20 2023 at 11:08 UTC