mathlib documentation

measure_theory.measure.stieltjes

Stieltjes measures on the real line #

Consider a function f : ℝ → ℝ which is monotone and right-continuous. Then one can define a corrresponding measure, giving mass f b - f a to the interval (a, b].

Main definitions #

Basic properties of Stieltjes functions #

structure stieltjes_function  :

Bundled monotone right-continuous real functions, used to construct Stieltjes measures.

Instances for stieltjes_function
@[protected]

The identity of as a Stieltjes function, used to construct Lebesgue measure.

Equations
noncomputable def monotone.stieltjes_function {f : } (hf : monotone f) :

If a function f : ℝ → ℝ is monotone, then the function mapping x to the right limit of f at x is a Stieltjes function, i.e., it is monotone and right-continuous.

Equations

The outer measure associated to a Stieltjes function #

noncomputable def stieltjes_function.length (f : stieltjes_function) (s : set ) :

Length of an interval. This is the largest monotone function which correctly measures all intervals.

Equations
theorem stieltjes_function.length_mono (f : stieltjes_function) {s₁ s₂ : set } (h : s₁ s₂) :
f.length s₁ f.length s₂
@[protected]

The Stieltjes outer measure associated to a Stieltjes function.

Equations
theorem stieltjes_function.length_subadditive_Icc_Ioo (f : stieltjes_function) {a b : } {c d : } (ss : set.Icc a b (i : ), set.Ioo (c i) (d i)) :
ennreal.of_real (f b - f a) ∑' (i : ), ennreal.of_real (f (d i) - f (c i))

If a compact interval [a, b] is covered by a union of open interval (c i, d i), then f b - f a ≤ ∑ f (d i) - f (c i). This is an auxiliary technical statement to prove the same statement for half-open intervals, the point of the current statement being that one can use compactness to reduce it to a finite sum, and argue by induction on the size of the covering set.

@[simp]

The measure associated to a Stieltjes function #

@[protected, irreducible]

The measure associated to a Stieltjes function, giving mass f b - f a to the interval (a, b].

Equations
Instances for stieltjes_function.measure