Documentation

Mathlib.MeasureTheory.Decomposition.Jordan

Jordan decomposition #

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 #

Main results #

Tags #

Jordan decomposition theorem

A Jordan decomposition of a measurable space is a pair of mutually singular, finite measures.

Instances For
    theorem MeasureTheory.JordanDecomposition.ext {α : Type u_2} {inst✝ : MeasurableSpace α} {x y : JordanDecomposition α} (posPart : x.posPart = y.posPart) (negPart : x.negPart = y.negPart) :
    x = y
    Equations
    • One or more equations did not get rendered due to their size.
    @[simp]

    The signed measure associated with a Jordan decomposition.

    Equations
    Instances For

      Given a signed measure s, s.toJordanDecomposition is the Jordan decomposition j, such that s = j.toSignedMeasure. This property is known as the Jordan decomposition theorem, and is shown by MeasureTheory.SignedMeasure.toSignedMeasure_toJordanDecomposition.

      Equations
      Instances For
        @[simp]

        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.toJordanDecomposition.posPart and s.toJordanDecomposition.negPart respectively.

        Note that we use MeasureTheory.JordanDecomposition.toSignedMeasure to represent the signed measure corresponding to s.toJordanDecomposition.posPart - s.toJordanDecomposition.negPart.

        theorem MeasureTheory.SignedMeasure.subset_positive_null_set {α : Type u_1} [MeasurableSpace α] {s : SignedMeasure α} {u v w : Set α} (hu : MeasurableSet u) (hv : MeasurableSet v) (hw : MeasurableSet w) (hsu : VectorMeasure.restrict 0 u VectorMeasure.restrict s u) (hw₁ : s w = 0) (hw₂ : w u) (hwt : v w) :
        s v = 0

        A subset v of a null-set w has zero measure if w is a subset of a positive set u.

        theorem MeasureTheory.SignedMeasure.subset_negative_null_set {α : Type u_1} [MeasurableSpace α] {s : SignedMeasure α} {u v w : Set α} (hu : MeasurableSet u) (hv : MeasurableSet v) (hw : MeasurableSet w) (hsu : VectorMeasure.restrict s u VectorMeasure.restrict 0 u) (hw₁ : s w = 0) (hw₂ : w u) (hwt : v w) :
        s v = 0

        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.

        The total variation of a signed measure.

        Equations
        Instances For