Zulip Chat Archive

Stream: maths

Topic: Assumptions for continuity in Lp


Yury G. Kudryashov (Aug 12 2023 at 16:28):

I want to prove that docs#DomMulAct action on Lp is a docs#ContinuousSMul action. It suffices to show that indicator (c • s) is continuous in c for all measurable s. What should I assume about the action, topology, and measure for it to be true?

Yury G. Kudryashov (Aug 12 2023 at 16:30):

Formally, I want to have

import Mathlib.MeasureTheory.Function.LpSpace.DomAct.Basic
import Mathlib.MeasureTheory.Function.ContinuousMapDense
import Mathlib.Topology.Algebra.Constructions.DomAct

variable {X M E : Type _}
  [TopologicalSpace X]
  [MeasurableSpace X] [BorelSpace X]
  [Monoid M] [TopologicalSpace M] [MeasurableSpace M] [BorelSpace M]
  [MulAction M X] [ContinuousSMul M X]
  [NormedAddCommGroup E] [NormedSpace  E]
  [SecondCountableTopologyEither X E]
  {μ : Measure X} [SMulInvariantMeasure M X μ] [MoreAssumptions]
  [Fact (1  p)] [hp : Fact (p  )]

instance : ContinuousSMul Mᵈᵐᵃ (Lp E p μ)

Yury G. Kudryashov (Aug 12 2023 at 19:30):

It looks like for a group action, [IsRegular] should be enough.

Antoine Chambert-Loir (Aug 13 2023 at 14:56):

I'd rather test on compactly supported cobtinuous functions, and then it seems that Lebesgue dominated convergence does the job.

Anatole Dedecker (Aug 13 2023 at 15:26):

This only works for Radon measures right? Is this what you meant by IsRegular Yury?(docs#MeasureTheory.Measure.Regular)

Anatole Dedecker (Aug 13 2023 at 15:33):

(this is the only thing that matches so probably yes)

Yury G. Kudryashov (Aug 13 2023 at 16:26):

Yes, I always forget which predicates have Is

Yury G. Kudryashov (Aug 14 2023 at 02:30):

Do we have dominated convergence in Lp?

Sebastien Gouezel (Aug 14 2023 at 07:17):

I don't think so. What version of the theorem are you thinking of?

Yury G. Kudryashov (Aug 14 2023 at 14:41):

I don't think I'll use it now but I was thinking about "if FnLpF_n\in L_p tends to ff a.e. everywhere and all FnF_n are dominated by gLpg\in L_p, then FnF_n tends to ff in LpL_p". Probably, with different versions for fLpf \in L_p as an assumption or as another conclusion.

Rémy Degenne (Aug 14 2023 at 14:58):

You can get the Lp convergence from a uniform integrability assumption with Vitali's convergence theorem, docs#MeasureTheory.tendstoInMeasure_iff_tendsto_Lp and surrounding results.

Rémy Degenne (Aug 14 2023 at 15:01):

docs#MeasureTheory.tendsto_Lp_of_tendsto_ae has docstring "A sequence of uniformly integrable functions which converges μ-a.e. converges in Lp."

Yury G. Kudryashov (Aug 14 2023 at 17:03):

Thank you!


Last updated: Dec 20 2023 at 11:08 UTC