Pushforward of a measure #
In this file we define the pushforward MeasureTheory.Measure.map f μ
of a measure μ
along an almost everywhere measurable map f
.
If f
is not a.e. measurable, then we define map f μ
to be zero.
Main definitions #
MeasureTheory.Measure.map f μ
: map of the measureμ
along the mapf
.
Main statements #
Lift a linear map between OuterMeasure
spaces such that for each measure μ
every measurable
set is caratheodory-measurable w.r.t. f μ
to a linear map between Measure
spaces.
Equations
- MeasureTheory.Measure.liftLinear f hf = { toFun := fun (μ : MeasureTheory.Measure α) => (f μ.toOuterMeasure).toMeasure ⋯, map_add' := ⋯, map_smul' := ⋯ }
Instances For
The pushforward of a measure as a linear map. It is defined to be 0
if f
is not
a measurable function.
Equations
- MeasureTheory.Measure.mapₗ f = if hf : Measurable f then MeasureTheory.Measure.liftLinear (MeasureTheory.OuterMeasure.map f) ⋯ else 0
Instances For
The pushforward of a measure. It is defined to be 0
if f
is not an almost everywhere
measurable function.
Equations
- MeasureTheory.Measure.map f μ = if hf : AEMeasurable f μ then (MeasureTheory.Measure.mapₗ (AEMeasurable.mk f hf)) μ else 0
Instances For
We can evaluate the pushforward on measurable sets. For non-measurable sets, see
MeasureTheory.Measure.le_map_apply
and MeasurableEquiv.map_apply
.
If map f μ = μ
, then the measure of the preimage of any null measurable set s
is equal to the measure of s
.
Note that this lemma does not assume (a.e.) measurability of f
.
Mapping a measure twice is the same as mapping the measure with the composition. This version is
for measurable functions. See map_map_of_aemeasurable
when they are just ae measurable.
Even if s
is not measurable, we can bound map f μ s
from below.
See also MeasurableEquiv.map_apply
.
Even if s
is not measurable, map f μ s = 0
implies that μ (f ⁻¹' s) = 0
.
Interactions of measurable equivalences and measures
If we map a measure along a measurable equivalence, we can compute the measure on all sets (not just the measurable ones).