@[instance]
Equations
- X.measurable_space = X.str
@[instance]
Equations
@[instance]
Equations
Measure X
is the measurable space of measures over the measurable space X
. It is the
weakest measurable space, s.t. λμ, μ s is measurable for all measurable sets s
in X
. An
important purpose is to assign a monadic structure on it, the Giry monad. In the Giry monad,
the pure values are the Dirac measure, and the bind operation maps to the integral:
(μ >>= ν) s = ∫ x. (ν x) s dμ
.
In probability theory, the Meas
-morphisms X → Prob X
are (sub-)Markov kernels (here Prob
is
the restriction of Measure
to (sub-)probability space.)
@[instance]
The Giry monad, i.e. the monadic structure associated with Measure
.
Equations
- Meas.category_theory.monad = {η := {app := λ (X : Meas), ⟨measure_theory.measure.dirac X.str, _⟩, naturality' := Meas.category_theory.monad._proof_2}, μ := {app := λ (X : Meas), ⟨measure_theory.measure.join X.str, _⟩, naturality' := Meas.category_theory.monad._proof_4}, assoc' := Meas.category_theory.monad._proof_5, left_unit' := Meas.category_theory.monad._proof_6, right_unit' := Meas.category_theory.monad._proof_7}
An example for an algebra on Measure
: the nonnegative Lebesgue integral is a hom, behaving
nicely under the monad operations.
@[instance]
Equations
- Top.has_forget_to_Meas = category_theory.bundled_hom.mk_has_forget₂ borel (λ (X Y : category_theory.bundled topological_space) (f : X ⟶ Y), ⟨f.to_fun, _⟩) Top.has_forget_to_Meas._proof_2