Jordan decomposition #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file proves the existence and uniqueness of the Jordan decomposition for signed measures.
The Jordan decomposition theorem states that, given a signed measure s
, there exists a
unique pair of mutually singular measures μ
and ν
, such that s = μ - ν
.
The Jordan decomposition theorem for measures is a corollary of the Hahn decomposition theorem and is useful for the Lebesgue decomposition theorem.
Main definitions #
measure_theory.jordan_decomposition
: a Jordan decomposition of a measurable space is a pair of mutually singular finite measures. We sayj
is a Jordan decomposition of a signed measures
ifs = j.pos_part - j.neg_part
.measure_theory.signed_measure.to_jordan_decomposition
: the Jordan decomposition of a signed measure.measure_theory.signed_measure.to_jordan_decomposition_equiv
: is theequiv
betweenmeasure_theory.signed_measure
andmeasure_theory.jordan_decomposition
formed bymeasure_theory.signed_measure.to_jordan_decomposition
.
Main results #
measure_theory.signed_measure.to_signed_measure_to_jordan_decomposition
: the Jordan decomposition theorem.measure_theory.jordan_decomposition.to_signed_measure_injective
: the Jordan decomposition of a signed measure is unique.
Tags #
Jordan decomposition theorem
- pos_part : measure_theory.measure α
- neg_part : measure_theory.measure α
- pos_part_finite : measure_theory.is_finite_measure self.pos_part
- neg_part_finite : measure_theory.is_finite_measure self.neg_part
- mutually_singular : self.pos_part.mutually_singular self.neg_part
A Jordan decomposition of a measurable space is a pair of mutually singular, finite measures.
Instances for measure_theory.jordan_decomposition
Equations
- measure_theory.jordan_decomposition.has_zero = {zero := {pos_part := 0, neg_part := 0, pos_part_finite := _, neg_part_finite := _, mutually_singular := _}}
Equations
Equations
- measure_theory.jordan_decomposition.has_involutive_neg = {neg := λ (j : measure_theory.jordan_decomposition α), {pos_part := j.neg_part, neg_part := j.pos_part, pos_part_finite := _, neg_part_finite := _, mutually_singular := _}, neg_neg := _}
Equations
- measure_theory.jordan_decomposition.has_smul = {smul := λ (r : nnreal) (j : measure_theory.jordan_decomposition α), {pos_part := r • j.pos_part, neg_part := r • j.neg_part, pos_part_finite := _, neg_part_finite := _, mutually_singular := _}}
The signed measure associated with a Jordan decomposition.
Equations
A Jordan decomposition provides a Hahn decomposition.
Given a signed measure s
, s.to_jordan_decomposition
is the Jordan decomposition j
,
such that s = j.to_signed_measure
. This property is known as the Jordan decomposition
theorem, and is shown by
measure_theory.signed_measure.to_signed_measure_to_jordan_decomposition
.
Equations
- s.to_jordan_decomposition = let i : set α := classical.some _, hi : measurable_set (classical.some _) ∧ 0.restrict (classical.some _) ≤ measure_theory.vector_measure.restrict s (classical.some _) ∧ measure_theory.vector_measure.restrict s (classical.some _)ᶜ ≤ 0.restrict (classical.some _)ᶜ := _ in {pos_part := s.to_measure_of_zero_le i _ _, neg_part := s.to_measure_of_le_zero iᶜ _ _, pos_part_finite := _, neg_part_finite := _, mutually_singular := _}
The Jordan decomposition theorem: Given a signed measure s
, there exists a pair of
mutually singular measures μ
and ν
such that s = μ - ν
. In this case, the measures μ
and ν
are given by s.to_jordan_decomposition.pos_part
and
s.to_jordan_decomposition.neg_part
respectively.
Note that we use measure_theory.jordan_decomposition.to_signed_measure
to represent the
signed measure corresponding to
s.to_jordan_decomposition.pos_part - s.to_jordan_decomposition.neg_part
.
A subset v
of a null-set w
has zero measure if w
is a subset of a positive set u
.
A subset v
of a null-set w
has zero measure if w
is a subset of a negative set u
.
If the symmetric difference of two positive sets is a null-set, then so are the differences between the two sets.
If the symmetric difference of two negative sets is a null-set, then so are the differences between the two sets.
The Jordan decomposition of a signed measure is unique.
measure_theory.signed_measure.to_jordan_decomposition
and
measure_theory.jordan_decomposition.to_signed_measure
form a equiv
.
Equations
The total variation of a signed measure.