Measurable spaces and measurable functions #
This file provides properties of measurable spaces and the functions and isomorphisms between them.
The definition of a measurable space is in Mathlib/MeasureTheory/MeasurableSpace/Defs.lean
.
A measurable space is a set equipped with a σ-algebra, a collection of subsets closed under complementation and countable union. A function between measurable spaces is measurable if the preimage of each measurable subset is measurable.
σ-algebras on a fixed set α
form a complete lattice. Here we order σ-algebras by writing m₁ ≤ m₂
if every set which is m₁
-measurable is also m₂
-measurable (that is, m₁
is a subset of m₂
).
In particular, any collection of subsets of α
generates a smallest σ-algebra which contains
all of them. A function f : α → β
induces a Galois connection between the lattices of σ-algebras
on α
and β
.
Implementation notes #
Measurability of a function f : α → β
between measurable spaces is defined in terms of the
Galois connection induced by f
.
References #
- https://en.wikipedia.org/wiki/Measurable_space
- https://en.wikipedia.org/wiki/Sigma-algebra
- https://en.wikipedia.org/wiki/Dynkin_system
Tags #
measurable space, σ-algebra, measurable function, dynkin system, π-λ theorem, π-system
The forward image of a measurable space under a function. map f m
contains the sets
s : Set β
whose preimage under f
is measurable.
Equations
- MeasurableSpace.map f m = { MeasurableSet' := fun (s : Set β) => MeasurableSet (f ⁻¹' s), measurableSet_empty := ⋯, measurableSet_compl := ⋯, measurableSet_iUnion := ⋯ }
Instances For
The reverse image of a measurable space under a function. comap f m
contains the sets
s : Set α
such that s
is the f
-preimage of a measurable set in β
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of the reverse direction of measurable_iff_le_map
.
Alias of the forward direction of measurable_iff_le_map
.
Alias of the forward direction of measurable_iff_comap_le
.
Alias of the reverse direction of measurable_iff_comap_le
.
A version of measurable_const
that assumes f x = f y
for all x, y
. This version works
for functions between empty types.
This is slightly different from Measurable.piecewise
. It can be used to show
Measurable (ite (x=0) 0 1)
by
exact Measurable.ite (measurableSet_singleton 0) measurable_const measurable_const
,
but replacing Measurable.ite
by Measurable.piecewise
in that example proof does not work.
The measurability of a set A
is equivalent to the measurability of the indicator function
which takes a constant value b ≠ 0
on a set A
and 0
elsewhere.
If a function coincides with a measurable function outside of a countable set, it is measurable.
We say that a collection of sets is countably spanning if a countable subset spans the
whole type. This is a useful condition in various parts of measure theory. For example, it is
a needed condition to show that the product of two collections generate the product sigma algebra,
see generateFrom_prod_eq
.
Equations
Instances For
Rectangles of countably spanning sets are countably spanning.