Zulip Chat Archive

Stream: mathlib4

Topic: Measure on an infinite product


Yury G. Kudryashov (Oct 11 2023 at 01:08):

I have an idea how we can merge two definitions of an indexed product of measures (finite product of σ-finite measures and an infinite product of probability measures) into one. We define the typeclass

-- todo: better name
class MeasureFamily {ι : Type*} {π : ι  Type*} [ i, MeasurableSpace (π i)] (μ :  i, Measure (π i)) : Prop where
  sigmaFinite :  i, SigmaFinite (μ i)
  isProbabilityMeasure : ∀ᶠ i in cofinite, IsProbabilityMeasure (μ i)

with an instance assuming [Finite ι] and an instance assuming [∀ i, IsProbabilityMeasure (μ i)].
Then we define one instance assuming [MeasureFamily μ] (we use the current construction for the non-probability finite product part and another construction for the probability part) and prove lemmas about it.

Yury G. Kudryashov (Oct 11 2023 at 01:08):

What do you think? I do understand that this is a nontrivial refactor.

Yury G. Kudryashov (Oct 11 2023 at 01:08):

If I try it, then how should I call the new typeclass?

Kevin Buzzard (Oct 11 2023 at 03:41):

Restricted infinite products are a generalisation of this. Here you have infinitely many spaces of infinite measure but each is equipped with a preferred subspace of measure 1. Each element in the restricted product must be outside the preferred subspace only finitely often but the finite bad set can depend on the element. So it's a direct limit of the construction you explain above.

Yury G. Kudryashov (Oct 11 2023 at 04:18):

What is the σ-algebra of measurable sets in this case?
We can have this definition but it can be added later because it leads to a measure on a different type, not the pi type.

Yaël Dillies (Oct 11 2023 at 06:59):

Yury G. Kudryashov said:

If I try it, then how should I call the new typeclass?

IsCofinitelyProbabilityMeasure? Not great...

Sebastien Gouezel (Oct 11 2023 at 07:16):

That's a good idea. But do we already have the product of infinitely many probability measures?

Yury G. Kudryashov (Oct 11 2023 at 12:44):

Not yet.

Yaël Dillies (Jul 18 2024 at 08:51):

@Yury G. Kudryashov, has anything moved on that front? @Kin Yau James Wong and I need the infinite product of probability measures to construct a (trivial) Gibbs measure

Yury G. Kudryashov (Jul 18 2024 at 13:34):

Not yet.

Yury G. Kudryashov (Jul 18 2024 at 13:35):

If you're going to work on this, I suggest that we talk about it first.

Yaël Dillies (Jul 18 2024 at 13:51):

Yeah, this is one of the first things we need for our project, so we need to work on this/convince you to do it for us

Sébastien Gouëzel (Jul 18 2024 at 14:24):

It has been done by Etienne Marion in his M1 internship with me, but it's not PRed to mathlib yet.

Yaël Dillies (Jul 18 2024 at 14:52):

Do you have any pointers for me?

Peter Pfaffelhuber (Jul 18 2024 at 18:21):

Yaël Dillies schrieb:

Yury G. Kudryashov, has anything moved on that front? Kin Yau James Wong and I need the infinite product of probability measures to construct a (trivial) Gibbs measure

Isn't this a simple example of the Kolmogorv Extension Theorem? @Rémy Degenne and I have worked this out, but still need to PR this to Mathlib. https://github.com/RemyDegenne/kolmogorov_extension4

Yaël Dillies (Jul 18 2024 at 19:17):

Yes it is

Yaël Dillies (Jul 19 2024 at 13:27):

@Peter Pfaffelhuber, I see MeasureTheory.independentFamily in your repo. However:

  • Do we really need all those topological assumptions? I would the infinite product of probability doesn't require anything like that (but maybe I'm just ignorant).
  • There's no API for it :sad:

Rémy Degenne (Jul 19 2024 at 13:30):

If you don't want topological assumptions, you need to restrict the index type. If you index over N, you don't need any assumption and can use the Ionescu-Tulcea theorem. This is what Etienne has done with Sébastien.

Yaël Dillies (Jul 19 2024 at 13:34):

I see. In our case, we care about ℤⁿ, so we would rather assume countability of the index type than topological stuff on the codomain

Yaël Dillies (Jul 19 2024 at 13:34):

Do you know where I can find Etienne's project?

Yury G. Kudryashov (Jul 19 2024 at 14:11):

About making different cases co-exist in Mathlib. I think that we should define the pi measure in some highly non-constructive way (e.g., the infimum of all measures such that for all s : ι → Set α with Set.Finite {i | μ i (s i) > 1}, the measure of Set.pi Set.univ s is ≥ tprod fun i ↦ μ i (s i) (not sure about > 1 vs ≠ 1; not sure if we need to require Countable ι, Set.Countable {i | s i ≠ univ}, or none). Then we can have a Prop-valued typeclass saying that a given family of measures admits a measure such that we have = tprod .... This way we can have instances with different assumptions and theorems assuming this TC.

Sébastien Gouëzel (Jul 19 2024 at 16:22):

You don't need topological assumptions for the product mesure, whatever the index set. Etienne has proved that. I'm currently getting the code in a reasonable state, should be ready today.

Peter Pfaffelhuber (Jul 19 2024 at 16:30):

This sounds like Corollary 8.25 in Kallenberg (Foundations of Modern Probability, 3rd edition). (If you have any dependency between coordinates, however, you will need some topological structure of the underlying spaces, as far as I know.)

Rémy Degenne (Jul 19 2024 at 16:38):

Sorry, I misread the thread and wrote nonsense. I meant that the extension theorem we used actually required assumptions in general.
The special case of the product measure is different.

Sébastien Gouëzel (Jul 19 2024 at 19:29):

You can find the definition of the general product measure in https://github.com/sgouezel/kolmogorov_extension4/blob/master/KolmogorovExtension4/MesureProduit2.lean. See productMeasure in this file, with some basic API after the definition.

Yaël Dillies (Jul 24 2024 at 16:03):

(now https://github.com/sgouezel/kolmogorov_extension4/blob/master/KolmogorovExtension4/ProductMeasure.lean)

Etienne Marion (Mar 25 2025 at 11:31):

#22555 just got merged, so infinite products of probability measures are now in Mathlib :tada:


Last updated: May 02 2025 at 03:31 UTC