Lebesgue decomposition #
This file proves the Lebesgue decomposition theorem. The Lebesgue decomposition theorem states that,
given two σ-finite measures μ
and ν
, there exists a σ-finite measure ξ
and a measurable
function f
such that μ = ξ + fν
and ξ
is mutually singular with respect to ν
.
The Lebesgue decomposition provides the Radon-Nikodym theorem readily.
Main definitions #
MeasureTheory.Measure.HaveLebesgueDecomposition
: A pair of measuresμ
andν
is said toHaveLebesgueDecomposition
if there exist a measureξ
and a measurable functionf
, such thatξ
is mutually singular with respect toν
andμ = ξ + ν.withDensity f
MeasureTheory.Measure.singularPart
: If a pair of measuresHaveLebesgueDecomposition
, thensingularPart
chooses the measure fromHaveLebesgueDecomposition
, otherwise it returns the zero measure.MeasureTheory.Measure.rnDeriv
: If a pair of measuresHaveLebesgueDecomposition
, thenrnDeriv
chooses the measurable function fromHaveLebesgueDecomposition
, otherwise it returns the zero function.MeasureTheory.SignedMeasure.HaveLebesgueDecomposition
: A signed measures
and a measureμ
is said toHaveLebesgueDecomposition
if both the positive part and negative part ofs
HaveLebesgueDecomposition
with respect toμ
.MeasureTheory.SignedMeasure.singularPart
: The singular part between a signed measures
and a measureμ
is simply the singular part of the positive part ofs
with respect toμ
minus the singular part of the negative part ofs
with respect toμ
.MeasureTheory.SignedMeasure.rnDeriv
: The Radon-Nikodym derivative of a signed measures
with respect to a measureμ
is the Radon-Nikodym derivative of the positive part ofs
with respect toμ
minus the Radon-Nikodym derivative of the negative part ofs
with respect toμ
.
Main results #
MeasureTheory.Measure.haveLebesgueDecomposition_of_sigmaFinite
: the Lebesgue decomposition theorem.MeasureTheory.Measure.eq_singularPart
: Given measuresμ
andν
, ifs
is a measure mutually singular toν
andf
is a measurable function such thatμ = s + fν
, thens = μ.singularPart ν
.MeasureTheory.Measure.eq_rnDeriv
: Given measuresμ
andν
, ifs
is a measure mutually singular toν
andf
is a measurable function such thatμ = s + fν
, thenf = μ.rnDeriv ν
.MeasureTheory.SignedMeasure.singularPart_add_withDensity_rnDeriv_eq
: the Lebesgue decomposition theorem between a signed measure and a σ-finite positive measure.
Tags #
Lebesgue decomposition theorem
- lebesgue_decomposition : ∃ p, Measurable p.snd ∧ MeasureTheory.Measure.MutuallySingular p.fst ν ∧ μ = p.fst + MeasureTheory.Measure.withDensity ν p.snd
A pair of measures μ
and ν
is said to HaveLebesgueDecomposition
if there exists a
measure ξ
and a measurable function f
, such that ξ
is mutually singular with respect to
ν
and μ = ξ + ν.withDensity f
.
Instances
If a pair of measures HaveLebesgueDecomposition
, then singularPart
chooses the
measure from HaveLebesgueDecomposition
, otherwise it returns the zero measure. For sigma-finite
measures, μ = μ.singularPart ν + ν.withDensity (μ.rnDeriv ν)
.
Instances For
If a pair of measures HaveLebesgueDecomposition
, then rnDeriv
chooses the
measurable function from HaveLebesgueDecomposition
, otherwise it returns the zero function.
For sigma-finite measures, μ = μ.singularPart ν + ν.withDensity (μ.rnDeriv ν)
.
Instances For
The Radon-Nikodym derivative of a sigma-finite measure μ
with respect to another
measure ν
is ν
-almost everywhere finite.
Given measures μ
and ν
, if s
is a measure mutually singular to ν
and f
is a
measurable function such that μ = s + fν
, then s = μ.singularPart μ
.
This theorem provides the uniqueness of the singularPart
in the Lebesgue decomposition theorem,
while MeasureTheory.Measure.eq_rnDeriv
provides the uniqueness of the
rnDeriv
.
Given measures μ
and ν
, if s
is a measure mutually singular to ν
and f
is a
measurable function such that μ = s + fν
, then f = μ.rnDeriv ν
.
This theorem provides the uniqueness of the rnDeriv
in the Lebesgue decomposition
theorem, while MeasureTheory.Measure.eq_singularPart
provides the uniqueness of the
singularPart
. Here, the uniqueness is given in terms of the measures, while the uniqueness in
terms of the functions is given in eq_rnDeriv
.
Given measures μ
and ν
, if s
is a measure mutually singular to ν
and f
is a
measurable function such that μ = s + fν
, then f = μ.rnDeriv ν
.
This theorem provides the uniqueness of the rnDeriv
in the Lebesgue decomposition
theorem, while MeasureTheory.Measure.eq_singularPart
provides the uniqueness of the
singularPart
. Here, the uniqueness is given in terms of the functions, while the uniqueness in
terms of the functions is given in eq_withDensity_rnDeriv
.
The Radon-Nikodym derivative of f ν
with respect to ν
is f
.
The Radon-Nikodym derivative of the restriction of a measure to a measurable set is the indicator function of this set.
If two finite measures μ
and ν
are not mutually singular, there exists some ε > 0
and
a measurable set E
, such that ν(E) > 0
and E
is positive with respect to μ - εν
.
This lemma is useful for the Lebesgue decomposition theorem.
Given two measures μ
and ν
, measurableLE μ ν
is the set of measurable
functions f
, such that, for all measurable sets A
, ∫⁻ x in A, f x ∂μ ≤ ν A
.
This is useful for the Lebesgue decomposition theorem.
Instances For
measurableLEEval μ ν
is the set of ∫⁻ x, f x ∂μ
for all f ∈ measurableLE μ ν
.
Instances For
Any pair of finite measures μ
and ν
, HaveLebesgueDecomposition
. That is to say,
there exist a measure ξ
and a measurable function f
, such that ξ
is mutually singular
with respect to ν
and μ = ξ + ν.withDensity f
.
This is not an instance since this is also shown for the more general σ-finite measures with
MeasureTheory.Measure.haveLebesgueDecomposition_of_sigmaFinite
.
The Lebesgue decomposition theorem: Any pair of σ-finite measures μ
and ν
HaveLebesgueDecomposition
. That is to say, there exist a measure ξ
and a measurable function
f
, such that ξ
is mutually singular with respect to ν
and μ = ξ + ν.withDensity f
- posPart : MeasureTheory.Measure.HaveLebesgueDecomposition (MeasureTheory.SignedMeasure.toJordanDecomposition s✝).posPart μ
- negPart : MeasureTheory.Measure.HaveLebesgueDecomposition (MeasureTheory.SignedMeasure.toJordanDecomposition s✝).negPart μ
A signed measure s
is said to HaveLebesgueDecomposition
with respect to a measure μ
if the positive part and the negative part of s
both HaveLebesgueDecomposition
with
respect to μ
.
Instances
Given a signed measure s
and a measure μ
, s.singularPart μ
is the signed measure
such that s.singularPart μ + μ.withDensityᵥ (s.rnDeriv μ) = s
and
s.singularPart μ
is mutually singular with respect to μ
.
Instances For
The Radon-Nikodym derivative between a signed measure and a positive measure.
rnDeriv s μ
satisfies μ.withDensityᵥ (s.rnDeriv μ) = s
if and only if s
is absolutely continuous with respect to μ
and this fact is known as
MeasureTheory.SignedMeasure.absolutelyContinuous_iff_withDensity_rnDeriv_eq
and can be found in MeasureTheory.Decomposition.RadonNikodym
.
Instances For
The Lebesgue Decomposition theorem between a signed measure and a measure:
Given a signed measure s
and a σ-finite measure μ
, there exist a signed measure t
and a
measurable and integrable function f
, such that t
is mutually singular with respect to μ
and s = t + μ.with_densityᵥ f
. In this case t = s.singular_part μ
and
f = s.rn_deriv μ
.
Given a measure μ
, signed measures s
and t
, and a function f
such that t
is
mutually singular with respect to μ
and s = t + μ.withDensityᵥ f
, we have
t = singularPart s μ
, i.e. t
is the singular part of the Lebesgue decomposition between
s
and μ
.
Given a measure μ
, signed measures s
and t
, and a function f
such that t
is
mutually singular with respect to μ
and s = t + μ.withDensityᵥ f
, we have
f = rnDeriv s μ
, i.e. f
is the Radon-Nikodym derivative of s
and μ
.
- rePart : MeasureTheory.SignedMeasure.HaveLebesgueDecomposition (↑MeasureTheory.ComplexMeasure.re c) μ
- imPart : MeasureTheory.SignedMeasure.HaveLebesgueDecomposition (↑MeasureTheory.ComplexMeasure.im c) μ
A complex measure is said to HaveLebesgueDecomposition
with respect to a positive measure
if both its real and imaginary part HaveLebesgueDecomposition
with respect to that measure.
Instances
The singular part between a complex measure c
and a positive measure μ
is the complex
measure satisfying c.singularPart μ + μ.withDensityᵥ (c.rnDeriv μ) = c
. This property is given
by MeasureTheory.ComplexMeasure.singularPart_add_withDensity_rnDeriv_eq
.
Instances For
The Radon-Nikodym derivative between a complex measure and a positive measure.