Stieltjes measures on the real line #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
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 #
stieltjes_functionis a structure containing a function fromℝ → ℝ, together with the assertions that it is monotone and right-continuous. Tof : stieltjes_function, one associates a Borel measuref.measure.f.measure_Iocasserts thatf.measure (Ioc a b) = of_real (f b - f a)f.measure_Iooasserts thatf.measure (Ioo a b) = of_real (left_lim f b - f a).f.measure_Iccandf.measure_Icoare analogous.
Basic properties of Stieltjes functions #
- to_fun : ℝ → ℝ
- mono' : monotone self.to_fun
- right_continuous' : ∀ (x : ℝ), continuous_within_at self.to_fun (set.Ici x) x
Bundled monotone right-continuous real functions, used to construct Stieltjes measures.
Instances for stieltjes_function
- stieltjes_function.has_sizeof_inst
- stieltjes_function.has_coe_to_fun
- stieltjes_function.inhabited
Equations
The identity of ℝ as a Stieltjes function, used to construct Lebesgue measure.
Equations
- stieltjes_function.id = {to_fun := id ℝ, mono' := stieltjes_function.id._proof_1, right_continuous' := stieltjes_function.id._proof_2}
Equations
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
- hf.stieltjes_function = {to_fun := function.right_lim f, mono' := _, right_continuous' := _}
The outer measure associated to a Stieltjes function #
The Stieltjes outer measure associated to a Stieltjes function.
Equations
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.
The measure associated to a Stieltjes function #
The measure associated to a Stieltjes function, giving mass f b - f a to the
interval (a, b].