Zulip Chat Archive

Stream: mathlib4

Topic: Amenable group actions


Anatole Dedecker (Sep 26 2023 at 13:14):

@Matthias U Which definition of amenable groups are you going for? In particular does it assume the group to be locally compact? In any case this is great, please ping me once you have an open PR!

Yaël Dillies (Sep 26 2023 at 13:16):

Anatole, if you want to have a sneak peak, there were 7 open PRs about amenability in mathlib: https://github.com/leanprover-community/mathlib/pulls?q=is%3Apr+amenable+is%3Aopen

Anatole Dedecker (Sep 26 2023 at 13:17):

Oooooh I missed that! (Probably because I didn’t know anything about amenable groups in 2022…)

Matthias U (Sep 26 2023 at 16:38):

Anatole Dedecker said:

Matthias U Which definition of amenable groups are you going for? In particular does it assume the group to be locally compact? In any case this is great, please ping me once you have an open PR!

Sure, I'll let you know. I'm mostly considering finitely generated (discrete) groups, so yes. But I'm happy to discuss possible generalisations, if applicable

Sebastien Gouezel (Sep 26 2023 at 16:40):

It's really important for nonamenability to go beyond discrete groups: essentially all the theory works for locally compact groups (although it is slightly more painful to set up), and this is needed for many applications.

Patrick Massot (Sep 26 2023 at 16:57):

I think Anatole meant that locally compact groups are not enough.

Sebastien Gouezel (Sep 26 2023 at 17:00):

Yes, I got that. My comment was to say that, for sure, discrete groups are not enough.

Notification Bot (Sep 26 2023 at 21:34):

6 messages were moved here from #mathlib4 > github permission by Oliver Nash.

Notification Bot (Sep 26 2023 at 21:34):

A message was moved here from #mathlib4 > github permission by Oliver Nash.

Junyan Xu (Sep 27 2023 at 01:54):

Should this combine with #new-members > Amenable Groups?

Matthias U (Sep 27 2023 at 08:01):

I just created a pull request: https://github.com/leanprover-community/mathlib4/pull/7395 . Looking forward to your comments!

Henrik Böving (Sep 27 2023 at 08:03):

Matthias U said:

I just created a pull request: https://github.com/leanprover-community/mathlib4/pull/7395 . Looking forward to your comments!

you forgot to run

find Mathlib -name "*.lean" | env LC_ALL=C sort | sed 's/\.lean//;s,/,.,g;s/^/import /' > Mathlib.lean

slash update Mathlib.lean with your new file

Matthias U (Sep 27 2023 at 08:17):

Btw, I'm following Bartholdi's survey article: https://arxiv.org/pdf/1705.04091.pdf (see Definitions 2.1 and 2.2 so far).

Anatole Dedecker (Sep 28 2023 at 13:08):

Reposting some comments I wrote on the PR because I think the discussion deserves to happen here:

I don't really know what the right definition of an amenable action is, but I'm worried that this definition won't give the correct definition for amenable (even locally compact) groups. The reason is that you definitely want your mean to be absolutely continuous with respect to any Haar measure on the group (otherwise there's no hope of viewing the mean as a functional on LL^\infty).

Furthermore, it would be nice to have a definition of amenability that works for any topological group, the usual one being the existence of a left invariant mean on right uniformly continuous function. The significant disadvantage of that is that linking this with the usual definition requires a bit more work. This is all explained in the book Sébastien mentioned, and I've written a slightly more precise exposition of it with formalization at the back of my mind, so I'd be happy to help anyone working on that, but I'm not sure we have all the prerequisites for it...

In the meantime, I think I'm okay with writing up the theory in the setting of locally compact groups, but we should keep in mind this future generalization. In particular, I'm against Yaël's proposal to link this with probability measures, because that won't be true in a general setting I think. But I'm not sure what to do regarding amenable actions, I'll try to read about it.

By the way, another painful revelation I had when writing about amenable locally compact groups is that we don't have the right LL^\infty for it: in this context you really want LL^\infty to be the dual of L1L^1, even for non sigma-compact groups, which means that the right thing to quotient by is not equality almost everywhere, but equality locally almost everywhere...

Sebastien Gouezel (Sep 28 2023 at 14:05):

I had never noticed the subtlety between almost everywhere and locally almost everywhere, thanks for pointing it out. For those who are curious, this is the following phenomenon. Consider a measure space with a single point of infinite mass. Then L^1 is trivial, so you expect its dual L^∞ to be also trivial. However, with the usual definition of L^∞ this is a line in this case (you can prescribe the value at the point). But if you mod out by all functions that are zero on finite measure sets (i.e., all functions, since there are no finite measure sets), then you kill everything and you are left with a trivial space, which is good. So one may argue that, when defining L^∞, instead of identifying functions that coincide ae, one should rather identify functions that coincide locally ae, i.e., are ae equal on each set of finite measure.

So what should we do? (1) Redefine L^p (and ae equal functions) to work with functions that coincide locally ae? Or (2) ignore the issue and add sigma-finiteness assumptions when needed (this implies that ae and locally ae coincide)? I'd rather go for (2) since I've never met interesting non-sigma-finite measures, but I would be ready to change my mind if anyone shows a convincing example where the added generality is important.

Sebastien Gouezel (Sep 28 2023 at 14:08):

(With (1), the L^∞ norm of the constant function equal to 1 on a single atom of infinite mass is equal to 0, which feels pretty unusual, to say the least).

Rémy Degenne (Sep 28 2023 at 14:18):

Can you get the same Lp as in (1) by replacing AEStronglyMeasurable by AEFinStronglyMeasurable in the definition of AEEqFun?

Sebastien Gouezel (Sep 28 2023 at 14:48):

I don't think so. On an uncountable space with the counting measure, the constant function 1 is in L^∞ (in the (1) or (2) sense, they coincide here), but it is not AEFinStronglyMeasurable.

Anatole Dedecker (Sep 28 2023 at 16:00):

Well the typical case where you want non sigma-finite measures are Haar measure on non sigma-compact groups. I don't know how much care about it in the general case, but I'm pretty sure that people care about uncountable discrete group at least. Of course the problem doesn't arise in this case, but I'm not sure we want a SecondCountableOrDiscrete typeclass just to go around this problem.

Anatole Dedecker (Sep 28 2023 at 16:05):

My instinct would be to go for (1) (note that this wouldn't actually change the definition for finite p I believe), but I definitely understand that it's a bit of a hassle for a situation which doesn't arise that often. I think we wouldn't lose anything by changing the definition (does anyone know of an example in non-sigma-finite measure where you'd want the current definition), but the risk is making the basic API heavier...

Sebastien Gouezel (Sep 28 2023 at 16:36):

To get an example where the notions differ, it's not really sigma-finiteness that matters. For instance, for the counting measure on an uncountable space, (1) and (2) coincide. The problem is when you have an infinite measure subset that does not contain a subset of finite positive measure. It's not clear to me if this is possible for a Haar measure on a locally compact group?

Kevin Buzzard (Sep 28 2023 at 17:04):

For Haar measure on a locally compact group, if you choose an open neighbourhood of a point within a compact neighbourhood then I think necessarily the open and compact neighbourhoods have nonzero finite measure (because every nonempty open has positive measure and every compact has finite measure; these are general properties of Haar measure).

Sebastien Gouezel (Sep 28 2023 at 17:04):

Here is an example. Consider R×R\mathbb{R} \times \mathbb{R} where the first line has the discrete topology, and the second one the usual topology. Then the Haar measure is a sum of uncountably many Lebesgue measures, one on each vertical line. And this is a locally compact group.

For any countable set ss, then s×{0}s\times \{0\} has zero measure: cover each point in ss by a vertical open interval with measure ϵ2n \epsilon * 2^{-n}, this gives an open set containing ss with measure at most ϵ\epsilon. On the other hand, for any uncountable set ss then s×{0}s\times \{0\} has infinite measure: given an open set which contains it, it contains t×(ϵ,ϵ)t \times (-\epsilon, \epsilon) for some uncountable tt and some positive ϵ\epsilon, so it has infinite measure. By outer regularity, this shows the claim. It follows that the horizontal line is an infinite measure set which contains only infinite measure sets and zero measure sets.

Kevin Buzzard (Sep 28 2023 at 17:11):

So necessarily the infinite measure set must have empty interior, which is indeed what is happening in your example.

Matthias U (Sep 29 2023 at 07:36):

Anatole Dedecker said:

I don't really know what the right definition of an amenable action is, but I'm worried that this definition won't give the correct definition for amenable (even locally compact) groups. The reason is that you definitely want your mean to be absolutely continuous with respect to any Haar measure on the group (otherwise there's no hope of viewing the mean as a functional on LL^\infty).

I tried to read a few things about the general situation: If I understand correctely, the following is true: A (topological) group G (with Haar measure μ\mu) is amenable if and only the left translation action GGG \curvearrowright G admits an invariant mean mm, where as σ\sigma-algebra, we take the Borel σ\sigma-algebra (i.e. the σ\sigma-algebra generated by the open sets of the topology on GG); Here, additionally, we need to demand that the mean mm is absolutely continuous wrt μ\mu (i.e. if AGA\subset G is measurable with μ(A)=0\mu(A) = 0, then we have m(A)=0m(A) = 0).

Reference for this fact: Remark G.1.3 in the appendix of "Kazhdan's Property (T)" by Bekka, de la Harpe, Valette

Sebastien Gouezel (Sep 29 2023 at 09:59):

I have just asked Bachir Bekka about that remark (he happens to have his office next to mine), and he told me to be careful about this remark, because

  • maybe the L(X,μ)L^\infty(X, \mu) in the remark is the usual LL^\infty, contrary to what they use in the rest of the book for LL^\infty on groups.
  • maybe the reference they give for the details (Hewitt-Stromberg) only deals with the sigma-finite case.

I'll have a look at Hewitt-Stromberg.

Sebastien Gouezel (Sep 29 2023 at 10:02):

(And note that the remark will only apply to locally compact groups, as you want to use the characterization in Theorem G.3.1 (v) which holds only for locally compact groups. Bachir argued convincingly that the main property of amenability should be the fixed point property for affine actions on compact convex sets, so the general definition should be the one they give in Definition G.1.4.

Sebastien Gouezel (Sep 29 2023 at 11:51):

Coming back to the distinction between the usual L(μ)L^\infty(\mu) (bounded measurable functions up to ae equivalence) and the more unusual Ll(μ)L_l^\infty(\mu) (bounded measurable functions up to local ae equivalence, i.e., two functions are equivalent iff, for every finite measure set, they coincide ae in this set). I am not sure this distinction is really relevant in the context of amenability of locally compact groups. Indeed, I claim it is equivalent to have an invariant mean on L(μ)L^\infty(\mu) or Ll(μ)L^\infty_l(\mu).

Proof: since there is a map from L(μ)L^\infty(\mu) to Ll(μ)L^\infty_l(\mu), an invariant mean on Ll(μ)L^\infty_l(\mu) gives one on L(μ)L^\infty(\mu). Conversely, assume you have an invariant mean on L(μ)L^\infty(\mu). As uniformly continuous bounded functions embed into L(μ)L^\infty(\mu), this gives an invariant mean on uniformly continuous bounded functions. By (i)=>(v) in Theorem G.3.1 in Bekka-de la Harpe-Valette, this gives an invariant mean on Ll(μ)L^\infty_l(\mu).

@Anatole Dedecker , does it make sense or am I confused somewhere?

Sebastien Gouezel (Sep 29 2023 at 11:57):

(It looks like this line of thought also says that it is equivalent to have an invariant mean on all measurable subsets, or an invariant mean on all measurable subsets which vanishes on all sets of Haar measure 0, or an invariant mean on all measurable subsets which vanishes on all sets of Haar measure locally 0).

Sebastien Gouezel (Sep 29 2023 at 14:34):

To support this, Fremlin (vol 4, Chapter 44) discusses amenable topological groups and amenable locally compact groups at length, without ever using LlL^\infty_l.

Antoine Chambert-Loir (Sep 29 2023 at 21:50):

I support the idea of having more general measure theory than what is usually done in basic treaties. For my own work, for example, where measures live on naturally huge spaces, it was absolutely fundamental to forget about exterior regularity and focus on interior regularity.

Antoine Chambert-Loir (Sep 29 2023 at 21:51):

Fremlin's book (I should say, books) is remarkable. If we manage to formalize it, it would be absolutely great.

Anatole Dedecker (Sep 30 2023 at 13:25):

Sebastien Gouezel said:

Coming back to the distinction between the usual L(μ)L^\infty(\mu) (bounded measurable functions up to ae equivalence) and the more unusual Ll(μ)L_l^\infty(\mu) (bounded measurable functions up to local ae equivalence, i.e., two functions are equivalent iff, for every finite measure set, they coincide ae in this set). I am not sure this distinction is really relevant in the context of amenability of locally compact groups. Indeed, I claim it is equivalent to have an invariant mean on L(μ)L^\infty(\mu) or Ll(μ)L^\infty_l(\mu).

Proof: since there is a map from L(μ)L^\infty(\mu) to Ll(μ)L^\infty_l(\mu), an invariant mean on Ll(μ)L^\infty_l(\mu) gives one on L(μ)L^\infty(\mu). Conversely, assume you have an invariant mean on L(μ)L^\infty(\mu). As uniformly continuous bounded functions embed into L(μ)L^\infty(\mu), this gives an invariant mean on uniformly continuous bounded functions. By (i)=>(v) in Theorem G.3.1 in Bekka-de la Harpe-Valette, this gives an invariant mean on Ll(μ)L^\infty_l(\mu).

Anatole Dedecker , does it make sense or am I confused somewhere?

I'm convinced by the argument, but I think that this could bite us later because existence of a mean on Ll(μ)L^\infty_l(\mu) is really a stronger statement: not only is the map L(μ)Ll(μ)L^\infty(\mu) \to L^\infty_l(\mu) not injective (i.e "we can assume the mean is zero on locally null sets", which is easy to state), it's also not surjective (i.e "we can assume the mean extends to this whole space", which is rather annoying to state without making reference to that bigger state). But I think it should be easy enough to just use the dual of L1L^1 each time we want to refer to Ll(μ)L^\infty_l(\mu), so at least it's not a strict requirement.

Anatole Dedecker (Sep 30 2023 at 13:28):

The situation in Fremlin is confusing to me (somehow I'm always lost when looking up something in Fremlin), because in the proof of theorem 449J (which is his version of G.3.1) he does say "recall that L1 is a Banach algebra under convolution (444Sb), and that L∞ can be
identified with its normed space dual, because μ is a quasi-Radon measure, therefore localizable (415A)". To me that must means that he's assuming something extra on his Haar measures, but I can't find what exactly...

Anatole Dedecker (Sep 30 2023 at 13:30):

The Haar measure in your counterexample above is outer regular wrt open sets and inner regular for open sets wrt compact sets, right?

Sebastien Gouezel (Sep 30 2023 at 13:33):

Anatole Dedecker said:

The Haar measure in your counterexample above is outer regular wrt open sets and inner regular for open sets wrt compact sets, right?

Yes. That's the standard definition of the Haar measure, if I am not mistaken.

Anatole Dedecker (Sep 30 2023 at 13:34):

I agree that it's the standard definition (although regularity is not required in Mathlib, right?)

Anatole Dedecker (Sep 30 2023 at 13:36):

Ah, Fremlin does assume his quasi-Radon measures to be semi-finite, which means exactly that you can't have infinite measure sets containing no nonzero finite measure sets.

Sebastien Gouezel (Sep 30 2023 at 13:40):

But then does it mean he can't construct a Haar measure on every locally compact group?

Anatole Dedecker (Sep 30 2023 at 13:42):

I'm surprised by this too, because he does prove an existence theorem...

Sebastien Gouezel (Sep 30 2023 at 13:52):

It seems Fremlin's definition of Radon measure is not the standard one (he requires inner regularity wrt compact sets for any measurable set, and he doesn't require outer regularity with respect to open sets). So probably his Haar measure is not the usual one...

Anatole Dedecker (Sep 30 2023 at 13:57):

I think the same kind of things happens for the Riesz representation theorem: the french wikipedia page gives two different notions of Radon measure that satisfy the Riesz reprensentation theorem (and there's even a claim that the one we have is not the "right" one)

Anatole Dedecker (Sep 30 2023 at 14:22):

@Antoine Chambert-Loir This is precisely what you claim, right? That inner regularity for all borel sets is more useful than docs#MeasureTheory.Measure.Regular

Anatole Dedecker (Sep 30 2023 at 14:32):

Matthias U said:

Anatole Dedecker said:

I don't really know what the right definition of an amenable action is, but I'm worried that this definition won't give the correct definition for amenable (even locally compact) groups. The reason is that you definitely want your mean to be absolutely continuous with respect to any Haar measure on the group (otherwise there's no hope of viewing the mean as a functional on LL^\infty).

I tried to read a few things about the general situation: If I understand correctely, the following is true: A (topological) group G (with Haar measure μ\mu) is amenable if and only the left translation action GGG \curvearrowright G admits an invariant mean mm, where as σ\sigma-algebra, we take the Borel σ\sigma-algebra (i.e. the σ\sigma-algebra generated by the open sets of the topology on GG); Here, additionally, we need to demand that the mean mm is absolutely continuous wrt μ\mu (i.e. if AGA\subset G is measurable with μ(A)=0\mu(A) = 0, then we have m(A)=0m(A) = 0).

Reference for this fact: Remark G.1.3 in the appendix of "Kazhdan's Property (T)" by Bekka, de la Harpe, Valette

Going back to amenability, yes indeed I think you recover the right notion if you add the absolute continuity, and this is exactly what I claim is the problem with your current definition: there's no absolute continuity. Furthermore, I think it will be nicer to work with means defined on all of LL^\infty instead of indicators to begin with, and prove later than you only care about indicators really.

Anatole Dedecker (Sep 30 2023 at 14:33):

Of course this is assuming we want to use the mean definition at all, instead of going straight to the general case.

Antoine Chambert-Loir (Sep 30 2023 at 14:48):

Anatole Dedecker said:

Antoine Chambert-Loir This is precisely what you claim, right? That inner regularity for all borel sets is more useful than docs#MeasureTheory.Measure.Regular

I just claim that exterior regularity is a good thing when you have it, but not something to expect in general (beyond the world of Polish spaces).

Anatole Dedecker (Sep 30 2023 at 14:58):

(Still about amenability)

Like Sébastien I am convinced that we need to consider the general case at some point and the fixed point characterization is really the right one. But, at least if we follow Bekka, de la Harpe and Valette (let's call it BHV), I think we need to do a few things before being able to prove their theorem G.3.1:

  • define type aliases to equip a group with left or right uniformity. This is not strictly a requirement, but I expect it will be nicer to work with right-uniformly-continuous function if we can spell them with type aliases (and I have fun versions of some proofs that require playing with these). Note that "left-uniformly-continuous" in BHV means uniformly continuous for the right uniformity for Bourbaki.
  • define convolution in multiplicative non-abelian groups, and prove the basic properties (notably that :L1×LL\ast:L^1\times L^\infty \to L^\infty actually takes values in right-uniformly-continuous function) without sigma-finiteness. This might require showing uniqueness of regular haar measures (note docs#MeasureTheory.Measure.haarMeasure_unique assumes sigma-finiteness).
  • we also need some facts about the (L1,(L1))(L^1, (L^1)^*) duality, namely that positive integrable functions of norm 1 map to a dense subset of means on (L1)(L^1)^* or LlL^\infty_l. This is left as an exercise in BHV if I remember correctly, but it's not entirely trivial because you need to be careful about positivity
  • we need to prove the complex version on a few results on real locally convex spaces (Hahn-Banach separation and some of its consequences mostly).

Anatole Dedecker (Sep 30 2023 at 15:03):

Antoine Chambert-Loir said:

Anatole Dedecker said:

Antoine Chambert-Loir This is precisely what you claim, right? That inner regularity for all borel sets is more useful than docs#MeasureTheory.Measure.Regular

I just claim that exterior regularity is a good thing when you have it, but not something to expect in general (beyond the world of Polish spaces).

And is it because you trade it for stronger inner regularity? Or just that the measures you care about are not meant to represent linear functionals on Cc(X)C_c(X) at all?

Antoine Chambert-Loir (Sep 30 2023 at 15:47):

Fremlin has a good discussion of Haar measures and their “uniqueness” (spoiler: as a function on sets, there is no uniqueness in general).

Antoine Chambert-Loir (Sep 30 2023 at 15:48):

Also, recently, model theory made new concepts emerge, such as Roelcke compactness, which has some interest for large spaces, such as function spaces.

Sebastien Gouezel (Oct 01 2023 at 06:30):

Anatole Dedecker said:

not only is the map L(μ)Ll(μ)L^\infty(\mu) \to L^\infty_l(\mu) not injective (i.e "we can assume the mean is zero on locally null sets", which is easy to state), it's also not surjective (i.e "we can assume the mean extends to this whole space", which is rather annoying to state without making reference to that bigger state).

I don't understand why it is not surjective. Let me try to prove instead it is surjective. Take an element of Ll(μ)L^\infty_l(\mu), and then a measurable representative f. It is bounded by some constant M on a set which is locally almost everything. Let F be the truncation mapping points larger than M to M, and points smaller than -M to -M, and the identity inbetween. Then F o f coincides locally almost everywhere with f, and it is bounded and measurable. It defines an element of L(μ)L^\infty(\mu), which maps to f in Ll(μ)L^\infty_l(\mu). Did I overlook something?

Anatole Dedecker (Oct 01 2023 at 11:45):

/me should think twice before making "obvious" claims...

More seriously, I'm confused. Your argument looks right, but one of the reasons I made that claim is that I remember that one of the issue that arises when you try to show L(L1)L^\infty \simeq (L^1)' is that to build an element of LL^\infty from a linear form on L1L^1 you need to "glue" elements of L(B)L^\infty(B) where BB has finite measure, which may prevent surjectivity. And indeed, both https://math.stackexchange.com/a/405587/828303 and Fremlin 243G claim that, even in the semi-finite case, you need something more to get that L(L1)L^\infty \to (L^1)' is surjective...

Sebastien Gouezel (Oct 01 2023 at 11:52):

Note that the fact that LlL^\infty_l is the dual of L1L^1 is not true in general...

Anatole Dedecker (Oct 01 2023 at 12:21):

Oh. That explains it indeed...

Anatole Dedecker (Oct 01 2023 at 12:25):

I've found an even better result: theorem 9.4.8 of Measure Theory by Cohn states that, although we do not have L(L1)L^\infty \simeq (L^1)' for general regular measures on locally compact spaces, we do have an isomorphism as long as we are on a locally compact group.

Sebastien Gouezel (Oct 01 2023 at 12:56):

Yes, that's what is behind Fremlin's argument also.

Sebastien Gouezel (Oct 01 2023 at 12:57):

But this is only true for inner regular measures. I think I'll refactor our Haar measure to use the inner regular one instead of the outer regular one, as it is definitely better behaved from a functional analysis point of view.

Anatole Dedecker (Oct 01 2023 at 13:06):

I think Cohn's definition of regularity is exactly docs#MeasureTheory.Measure.regular though.

Anatole Dedecker (Oct 01 2023 at 13:07):

Ultimately there is a bijection between outer regular and inner regular measures right? Maybe the safest thing to do is to add this translation explicitly so that we're not blocked in the future (we still have to choose which one we base the theory onto, but even if we choose the "wrong" one it wouldn't cause that much trouble).

Sebastien Gouezel (Oct 01 2023 at 13:08):

Then his statement is not correct: for the regular Haar measure on R×R\mathbb{R} \times \mathbb{R} where the first copy is discrete, the set R×{0}\mathbb{R} \times \{0\} only contains zero and infinite measure subsets, so its characteristic function is nonzero in LL^\infty but still it is orthogonal to all L1L^1 functions.

Anatole Dedecker (Oct 01 2023 at 13:09):

Ah yes that's the same example of course... Sorry for getting confused

Sebastien Gouezel (Oct 01 2023 at 13:10):

My plan is to have a notion of preHaarMeasure where one would just require invariance, finiteness on compacts and positivity on opens (what is now called HaarMeasure). And then prove as many things as possible just assuming this. Additionally, have HaarMeasure require inner regularity. And prove existence and uniqueness of a preHaarMeasure which is regular, and also existence and uniqueness of a preHaarMeasure which is inner regular (i.e., of a HaarMeasure).

Anatole Dedecker (Oct 01 2023 at 13:15):

That sounds good!

Cameron Zwarich (Oct 04 2023 at 06:25):

Anatole Dedecker said:

I've found an even better result: theorem 9.4.8 of Measure Theory by Cohn states that, although we do not have L(L1)L^\infty \simeq (L^1)' for general regular measures on locally compact spaces, we do have an isomorphism as long as we are on a locally compact group.

Cohn proves earlier (in 7.5.4 in the 2nd edition) that this duality holds for the completion of regular Borel measures (for the same definition currently used by Lean) on LCH spaces. However, for Haar measures he proves in 9.4.8 that this holds even for the measure space given by the restriction of Haar measure to Borel sets. His definition of LL^\infty is what was previously called LlL_l^\infty in this thread.

While inner-regular measures seem like a more sensible choice for more general topological measure theory, for harmonic analysis on LCGs the definition in terms of mixed outer/inner regularity has been standard, and I think you will find some subtle reliance on this. One example is the Vitali-Carathéodory theorem that L1L^1 functions can be approximated by lower/upper-semicontinuous functions from above/below.

Sebastien Gouezel (Oct 04 2023 at 06:39):

Recent textbooks I've looked at (Bogachev, Fremlin) all emphasize that the inner regular version is better, especially for Haar measure on locally compact groups. For L^1 functions, both measures will gives the same result (they only disagree in non sigma-finite situations, and the set of nonzero points of an L^1 function is sigma-finite), so Vitali-Caratheodory will hold whatever the choice of the Haar measure.

Sebastien Gouezel (Oct 05 2023 at 05:34):

Sebastien Gouezel said:

Vitali-Caratheodory will hold whatever the choice of the Haar measure.

Scratch that, it's just wrong. The two Haar measures agree on what the L^1 space is (i.e., there is a canonical isometry between the two of them), but only as a space of equivalence classes of functions (and the equivalence relation is not the same on the left and on the right, although the quotients are canonically isomorphic). They disagree on what an integrable function is, and indeed for the inner regular measure some integrable functions will not satisfy Vitali-Caratheodory (the characteristic function of R×{0}\mathbb{R} \times \{0\} is an example: it is almost everywhere zero for the inner Haar measure, so integrable, but still it can not be approximated from above by an integrable lower semicontinuous function).

Antoine Chambert-Loir (Oct 05 2023 at 09:00):

what do you mean by : “the equivalence relation is not the same although the quotients are canonically isomorphic”?

Sebastien Gouezel (Oct 05 2023 at 09:03):

When you build equivalence classes of functions, you identify two functions if they coincide almost everywhere. As you have two measures, you have two notions of "coinciding almost everywhere", which are genuinely different. But since the spaces of integrable functions you start from are also different, the quotients you get happen to be the same (well, canonically isomorphic to be precise).

Kevin Buzzard (Oct 05 2023 at 09:04):

Any sentence containing the word canonical is by definition not precise, the word is used precisely to remove precision

Ruben Van de Velde (Oct 05 2023 at 09:10):

It is used canonically to remove precision?

Sebastien Gouezel (Oct 05 2023 at 09:11):

ok, let me be precise :-)
Let μ\mu be the inner regular Haar measure, and ν\nu the outer regular one. Let L1(μ)\mathcal{L}^1(\mu) be the space of integrable functions for μ\mu (genuine functions, not equivalence classes), and L1(μ)L^1(\mu) the space of equivalence classes of integrable functions for μ\mu. There are more zero measure sets for μ\mu than for ν\nu, and more integrable functions for μ\mu than for ν\nu (the characteristic function of R×{0}\mathbb{R} \times \{0\} is integrable for μ\mu but not for ν\nu). The composition of the inclusion L1(ν)L1(μ)\mathcal{L}^1(\nu) \to \mathcal{L}^1(\mu) and the quotient map L1(μ)L1(μ)\mathcal{L}^1(\mu) \to L^1(\mu) gives a natural map L1(ν)L1(μ)\mathcal{L}^1(\nu) \to L^1(\mu). It descends to the quotient, giving a map L1(ν)L1(μ)L^1(\nu) \to L^1(\mu), which happens to be a bijective isometry.

Kevin Buzzard (Oct 05 2023 at 09:12):

This is an extraordinary subtlety in the theory

Antoine Chambert-Loir (Oct 05 2023 at 09:13):

OK, thanks! In the above discussion, I had not been able to note the inclusion L1(ν)L1(μ) \mathcal L^1(\nu) \to \mathcal L^1(\mu) .

Antoine Chambert-Loir (Oct 05 2023 at 09:14):

Kevin Buzzard said:

This is an extraordinary subtlety in the theory

That's amazing, and also frightening, to realize how much detail is overlooked or forgotten in our standard (and nevertheless quite good) early math education.

Sebastien Gouezel (Oct 05 2023 at 09:14):

Most authors don't need to care, because they choose once and for all the inner regular Haar measure, or the outer regular Haar measure. Note that this identification is true for all LpL^p spaces but for LL^\infty, where the space for the inner one is nicer than the space for the outer one (it is smaller, and coincides with the dual of L1L^1).

Sebastien Gouezel (Oct 05 2023 at 09:15):

(And in reality all this doesn't matter, because all locally compact groups of interest happen to also be sigma-compact, and then the two Haar measures coincide).

Anatole Dedecker (Oct 05 2023 at 09:25):

I think the most surprising part is not that there are two standards, it’s that modern measure theorists seem to have a definite answer to "which one is more useful" yet (in my experience) most people teach the other one

Kevin Buzzard (Oct 05 2023 at 09:29):

What I was surprised by was that I am using Haar measure everywhere when I'm doing representation theory of p-adic groups but never encountered this subtlety -- but now I understand it's because it's not there in the cases which come up in my work (they're all sigma compact)

Sebastien Gouezel (Oct 05 2023 at 09:36):

I have to say I was completely unaware of this 10 days ago. And I'm glad I read enough measure theory since then to fill the gaps. That's one of the reasons I like so much formalizing -- you have to really understand what is going on, even the gory details noone ever mentions.

Antoine Chambert-Loir (Oct 05 2023 at 13:13):

Also : when you view measures as linear forms on continuous functions with compact support, this subtleties are totally absent (in that framework, the Haar measure is unique).

Antoine Chambert-Loir (Oct 05 2023 at 13:16):

If you allow a bit of provocation (those, who know, know) : while people claim the σ-algebra point of view is the only one that is valid to develop integration, it's only true for probability theory, and a lot of analysis (PDEs in particular) is perfectly happy with the point of view of Radon measures, to the point that distribution theory is a kind of generalization of it.


Last updated: Dec 20 2023 at 11:08 UTC