The category of measurable spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Measurable spaces and measurable functions form a (concrete) category Meas
.
Main definitions #
-
Measure : Meas ⥤ Meas
: the functor which sends a measurable spaceX
to the space of measures onX
; it is a monad (the "Giry monad"). -
Borel : Top ⥤ Meas
: sends a topological spaceX
toX
equipped with theσ
-algebra of Borel sets (theσ
-algebra generated by the open subsets ofX
).
Tags #
measurable space, giry monad, borel
The category of measurable spaces and measurable functions.
Equations
Equations
- X.measurable_space = X.str
Equations
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.)
The Giry monad, i.e. the monadic structure associated with Measure
.
Equations
- Meas.Giry = {to_functor := Meas.Measure, η' := {app := λ (X : Meas), ⟨measure_theory.measure.dirac X.str, _⟩, naturality' := Meas.Giry._proof_2}, μ' := {app := λ (X : Meas), ⟨measure_theory.measure.join X.str, _⟩, naturality' := Meas.Giry._proof_4}, assoc' := Meas.Giry._proof_5, left_unit' := Meas.Giry._proof_6, right_unit' := Meas.Giry._proof_7}
An example for an algebra on Measure
: the nonnegative Lebesgue integral is a hom, behaving
nicely under the monad operations.
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