Zulip Chat Archive
Stream: Is there code for X?
Topic: Product of infinitely-many probability measures
Oliver Nash (Sep 20 2024 at 10:49):
I'd like to be able to take the product of infinitely-many probability measures. Am I right in thinking we do not yet have this construction?
Oliver Nash (Sep 20 2024 at 10:50):
For example, the following works:
import Mathlib
open MeasureTheory
variable {ι : Type*} {α : ι → Type*}
[∀ i, MeasurableSpace (α i)]
(μ : (i : ι) → Measure (α i))
[∀ i, IsProbabilityMeasure (μ i)]
variable [Fintype ι] -- This is what I would like to drop
noncomputable example : Measure ((i : ι) → α i) := Measure.pi μ
#synth IsProbabilityMeasure (Measure.pi μ)
but not if I drop the [Fintype ι]
.
Rémy Degenne (Sep 20 2024 at 10:51):
Not in Mathlib yet. It's in https://github.com/sgouezel/kolmogorov_extension4 (work of @Etienne Marion ), which depends on https://github.com/RemyDegenne/kolmogorov_extension4/ , and both need to make their way to Mathlib.
Oliver Nash (Sep 20 2024 at 10:51):
Oh excellent, great to know they're en route: thanks!
Last updated: May 02 2025 at 03:31 UTC