Zulip Chat Archive
Stream: general
Topic: Trying to understand nhdsSet
Trevor Murphy (Dec 17 2025 at 21:21):
I'm learning about filters through some basic exercises on normed topological vector spaces over the reals. One question that arose for me was this: can I show the following
example {X : Type*} [SeminormedAddCommGroup X] [NormedSpace โ X]
{U V : Set X} : ๐หข (U + V) = ๐หข U + ๐หข V := sorry
If not, are there hypotheses I can add to U and/or V that make it true in a nontrivial way? Intuitively I'm pretty sure that the "โค" direction is true in general, though I'm still struggling to formalize a proof. But I'm really struggling to think about the "โฅ" direction. I can't think of a counterexample, but I also get easily confused when trying to unravel the definitions.
Is somebody able to point me in a useful direction?
Kevin Buzzard (Dec 17 2025 at 21:48):
Can you edit your post to make it a #mwe ? So far I tried adding import Mathlib and open scoped Topology but your code still doesn't compile so I don't even know what the question says.
Kevin Buzzard (Dec 17 2025 at 21:53):
Oh finally got it: is this your question?
import Mathlib
open scoped Topology Pointwise
example {X : Type*} [SeminormedAddCommGroup X] [NormedSpace โ X]
{U V : Set X} : ๐หข (U + V) = ๐หข U + ๐หข V := sorry
Can you give a mathematics proof of what you're claiming here? i.e. are you asking a mathematics question or a Lean question?
Trevor Murphy (Dec 17 2025 at 22:17):
Ah sorry for the confusion. There's a math question and a lean question. Here's the lean part first:
The claim ๐หข (U + V) โค ๐หข U + ๐หข V holds generally. Let W be any set in ๐หข U + ๐หข V, and let U' and V' be open sets with U โ U', V โ V', and U' + V' โ W. Then U' + V' is an open set with U + V โ U' + V' โ W, so W is in ๐หข (U + V). I'm stuck translating this into lean because I don't understand the nhdsSet API well enough to pull out the U' and V' that satisfy those conditions.
Trevor Murphy (Dec 17 2025 at 22:23):
Then there's a math question about the reverse inequality. It feels like there should be a counterexample, but I'm just not coming up with it. I was hoping maybe the API and general lean code around nhdsSet could point me in a useful direction but I couldn't figure it out.
Alternatively, it feels like if I assume U and V are nice enough (maybe connected?) then it should be possible to prove the reverse inequality. Again I was hoping to glean some ideas from the conditions and properties of nhdsSet, but I couldn't figure it out.
Kevin Buzzard (Dec 17 2025 at 22:38):
import Mathlib
open scoped Topology Pointwise
example {X : Type*} [SeminormedAddCommGroup X] [NormedSpace โ X]
{U V : Set X} : ๐หข (U + V) โค ๐หข U + ๐หข V := by
-- let W be any set in N(U)+N(V)
intro W hW
-- by definition
-- let A, B be sets with U โ interior(A), V โ interior(B), and A + B โ W
obtain โจA, hA, B, hB, hโฉ := hW
-- let U' and V' be opens with U โ U' โ A and V โ V' โ B
rw [mem_nhdsSet_iff_exists] at hA hB
obtain โจU', hU', hUU', HU'Aโฉ := hA
obtain โจV', hV', hVV', hV'Bโฉ := hB
-- we want to find some open W' with U + V โ W' โ W
rw [mem_nhdsSet_iff_exists]
-- We claim U' + V' works
use U' + V'
-- is an open set with U + V โ U' + V' โ W
-- so we now need to check it's open, it contains U+V and it's contained in W
refine โจ?_, ?_, ?_โฉ
ยท -- U' + V' is open because it's a union of open sets (translate of V')
exact IsOpen.add_left hV'
ยท -- the inclusion U + V โ U' + V' is clear by monotonicity results
mono
ยท -- and the inclusion U' + V' โ W is also clear
apply subset_trans (show U' + V' โ A + B by mono) h
is the inclusion which we have the proof of.
Mirek Olลกรกk (Dec 17 2025 at 22:41):
If I understand the definitions well, this should be a counterexample to the math question:
- A neighborhood of where we take a ball of radius around each integer point.
Trevor Murphy (Dec 17 2025 at 23:01):
Okay! Thanks so much! I'll go work through these
Mirek Olลกรกk (Dec 17 2025 at 23:01):
I don't think connectedness helps much, then I could connect the disconnected points through another dimension. Compactness of should help, then for a given neighborhood of , we can find an -neighborhood inside.
Trevor Murphy (Dec 17 2025 at 23:06):
Ah now I see how that example works. Interesting, thanks for explaining. I'll have a lot to think about on the plane home
Kevin Buzzard (Dec 17 2025 at 23:47):
How about , , and the neighbourhood is simply ?
Last updated: Dec 20 2025 at 21:32 UTC