Documentation

Mathlib.MeasureTheory.Measure.WithDensityVectorMeasure

Vector measure defined by an integral #

Given a measure μ and an integrable function f : α → E, we can define a vector measure v such that for all measurable set s, v i = ∫ x in s, f x ∂μ. This definition is useful for the Radon-Nikodym theorem for signed measures.

Main definitions #

Given a measure μ and an integrable function f, μ.withDensityᵥ f is the vector measure which maps the set s to ∫ₛ f ∂μ.

Instances For
    theorem MeasureTheory.withDensityᵥ_apply {α : Type u_1} {m : MeasurableSpace α} {μ : MeasureTheory.Measure α} {E : Type u_3} [NormedAddCommGroup E] [NormedSpace E] {f : αE} (hf : MeasureTheory.Integrable f) {s : Set α} (hs : MeasurableSet s) :
    ↑(MeasureTheory.Measure.withDensityᵥ μ f) s = ∫ (x : α) in s, f xμ

    Having the same density implies the underlying functions are equal almost everywhere.

    theorem MeasureTheory.Integrable.withDensityᵥ_trim_eq_integral {α : Type u_1} {m : MeasurableSpace α} {m0 : MeasurableSpace α} {μ : MeasureTheory.Measure α} (hm : m m0) {f : α} (hf : MeasureTheory.Integrable f) {i : Set α} (hi : MeasurableSet i) :
    ↑(MeasureTheory.VectorMeasure.trim (MeasureTheory.Measure.withDensityᵥ μ f) hm) i = ∫ (x : α) in i, f xμ