Zulip Chat Archive
Stream: Is there code for X?
Topic: Measurable space over probability measures
Markus de Medeiros (Feb 18 2025 at 00:30):
I'm working on cleaning up a lemma related to the Giry monad over probability spaces. Is there a MeasurableSpace
instance for ProbabilityMeasure
somewhere that I'm somehow not triggering or is this missing?
mwe:
import Mathlib.MeasureTheory.Measure.GiryMonad
import Mathlib.MeasureTheory.Measure.ProbabilityMeasure
noncomputable section
open ENNReal MeasureTheory MeasureTheory.Measure
variable {α : Type*} [MeasurableSpace α]
#synth MeasurableSpace (Measure α) -- OK
#synth MeasurableSpace { μ : Measure α // IsProbabilityMeasure μ } -- OK
-- #synth MeasurableSpace (ProbabilityMeasure α) -- Fails
Last updated: May 02 2025 at 03:31 UTC