Zulip Chat Archive
Stream: Is there code for X?
Topic: Banach–Alaoglu theorem
Adam Topaz (Aug 08 2022 at 14:24):
Dear functional analysts of mathlib --
How far are we from having the Banach–Alaoglu theorem? I'm not at all familiar with the functional analysis part of mathlib, but it seems that we have at least some of the necessary lemmas, e.g. docs#continuous_linear_map.is_closed_image_coe_closed_ball
Moritz Doll (Aug 08 2022 at 14:25):
We have it for normed spaces: docs#continuous_linear_map.is_compact_image_coe_closed_ball
Adam Topaz (Aug 08 2022 at 14:25):
Ha! just the lemma below :)
Moritz Doll (Aug 08 2022 at 14:25):
for topological vector spaces we are not that far, but as far as I know nobody is working on it
Adam Topaz (Aug 08 2022 at 14:25):
Thanks I'll try to see if I can use this in my use case
Adam Topaz (Aug 08 2022 at 14:26):
The issue is that the norm on the weak dual I am using is not the usual one, so I'm not completely sure it would work.
Adam Topaz (Aug 08 2022 at 15:00):
Actually, do we know that the weak dual is a closed as a subset of the cartesian product?
Adam Topaz (Aug 08 2022 at 15:01):
More precisely, I'm working with a normed space over and looking at its weak dual .
Jireh Loreaux (Aug 08 2022 at 17:46):
I'm not sure what your topology is on that second space.
Adam Topaz (Aug 08 2022 at 17:48):
Just the product topology.
Adam Topaz (Aug 08 2022 at 17:49):
Namely I'm just looking at the map .
Adam Topaz (Aug 08 2022 at 17:50):
And has the weak topology
Jireh Loreaux (Aug 08 2022 at 17:54):
I think docs#weak_bilin.coe_fn_continuous should get you where you want to go, but I'm not at my machine right now.
Adam Topaz (Aug 08 2022 at 17:55):
Oh, continuity is easy to prove, but I think this is actually a closed immersion, and that's what I'm after.
Jireh Loreaux (Aug 08 2022 at 17:56):
Adam Topaz (Aug 08 2022 at 17:57):
that's not a closed embedding, unfortunately :(
Jireh Loreaux (Aug 08 2022 at 17:58):
Sorry, out of time, I'm headed into a meeting. If this is still unanswered in a few hours I'll try to do it.
Adam Topaz (Aug 08 2022 at 18:06):
No rush! Thanks for the help :)
Anatole Dedecker (Aug 08 2022 at 18:41):
Wait is that really true? That would mean that a pointwise limit of continuous linear functionals is linear (which is trivial: docs#linear_map_of_tendsto) and continuous (which is false in general I believe). That would work if V is complete though, thanks to docs#continuous_linear_map_of_tendsto
Adam Topaz (Aug 08 2022 at 18:47):
Yes you're right. Fortunately, I'm in a situation with V
being complete (alternatively, I'm happy to use just the algebraic dual in my particular context, since I have another way of restricting to continuous functionals).
Jireh Loreaux (Aug 08 2022 at 19:50):
docs#continuous_linear_map_of_tendsto is about sequences (actually, it could generalize to pointwise bounded families tending to some function pointwise), but the weak⋆ topology isn't first countable, so sequences won't be enough.
Adam, what statement do you need exactly? After Anatole's comment and a few minutes thinking about it, I'm not sure this is a closed immersion. However, your mention of Banach-Alaoglu at the beginning of the thread makes me suspect you only need something weaker. For example, if you just need to know that the unit ball of the dual is closed (in the product topology), then that's much easier, and this is a thing which comes up commonly in functional analysis.
Adam Topaz (Aug 08 2022 at 19:55):
Here is the precise situation -- I have a compact Hausdorff totally disconnected space , and I'm considering with the sup norm.
I'm looking at the weak dual . Choose some and consider the set of all such that where is the indicator function on and form a clopen partition of . What I'm trying to show is that is compact. It's not quite a closed ball in the usual sense, but as far as I can tell it is indeed a closed subset which is bounded in the usual sense by .
This is needed for one of the final examples we're trying to do for LTE.
Adam Topaz (Aug 08 2022 at 20:01):
So in some sense I would like to use docs#weak_dual.is_compact_of_bounded_of_closed to prove compactness of this .
Is this a sound strategy? I'm not at all a functional analyst ;-/
Adam Topaz (Aug 08 2022 at 20:06):
If you have some other way to show that the functor sending a profinite space to the space of -signed Radon measures bounded by commutes with cofiltered limits, then I'm all ears :)
Jireh Loreaux (Aug 08 2022 at 20:10):
To show this is compact in the product topology, the steps are:
- Show that it is bounded in the norm topology on the dual and closed in the weak⋆ topology, both of which seem doable.
- apply docs#weak_dual.is_compact_of_bounded_of_closed to get that it is compact in the weak⋆ topology
- apply docs#weak_bilin.coe_fn_continuous to get that the image (under the "identity" function) is compact in the product topology. (this is why I originally mentioned this result, because I thought you wanted something to this effect.)
Jireh Loreaux (Aug 08 2022 at 20:10):
In other words, yes, your approach seems reasonable, but I did not check the viability of (1) carefully.
Adam Topaz (Aug 08 2022 at 20:11):
I'm quite sure I have a path forward with (1).
Adam Topaz (Aug 08 2022 at 20:12):
Thanks for the help! Even just discussing this out loud is helpful for me :)
Moritz Doll (Aug 08 2022 at 20:21):
@Jireh Loreaux do you really mean docs#weak_bilin.coe_fn_continuous or do you rather mean docs#weak_bilin.embedding ?
Adam Topaz (Aug 08 2022 at 20:22):
Just to clarify, I don't actually need to map to the product topology, so I think just (1) and (2) would suffice for my application.
Jireh Loreaux (Aug 08 2022 at 20:27):
Moritz, continuity suffices right? I mean, continuous images of compact sets are compact, so I don't think you would need it to be an embedding (although it is nevertheless in this case).
Moritz Doll (Aug 08 2022 at 20:28):
yes, of course. I was misinterpreting the map (and the docstring for docs#weak_bilin.embedding wrote the map as I wanted to see it).
Jireh Loreaux (Aug 08 2022 at 20:29):
I know, I had to think about it too when I first read it.
Moritz Doll (Aug 08 2022 at 20:29):
maybe I should add another docstring to docs#weak_bilin.coe_fn_continuous
Jireh Loreaux (Aug 08 2022 at 20:30):
cc @Kalle Kytölä I thought you might want to see Adam using your work on Banach-Alaoglu for normed spaces. See, it's useful even though it's not in full generality!
Jireh Loreaux (Aug 08 2022 at 20:32):
Moritz, while you're at it, there's no embedding specific to docs#weak_dual, whereas there does exist docs#weak_dual.coe_fn_continuous. If you think it's worth it, you could add the embedding too.
Adam Topaz (Aug 09 2022 at 19:55):
Quick update: The strategy (1) + (2) above worked perfectly :) See
https://github.com/leanprover-community/lean-liquid/blob/7284f07b6f14019d5cf7ebd7134fe9648b80bf47/src/examples/Radon/main.lean#L173
Thanks all for the help!
Last updated: Dec 20 2023 at 11:08 UTC