Stieltjes measures on the real line #
Consider a function f : ℝ → ℝ which is monotone and right-continuous. Then one can define a
corresponding measure, giving mass f b - f a to the interval (a, b]. We implement more
generally this notion for f : R → ℝ where R is a conditionally complete dense linear order.
Main definitions #
StieltjesFunction Ris a structure containing a function fromR → ℝ, together with the assertions that it is monotone and right-continuous. Tof : StieltjesFunction R, one associates a Borel measuref.measure.f.measure_Iocasserts thatf.measure (Ioc a b) = ofReal (f b - f a)f.measure_Iooasserts thatf.measure (Ioo a b) = ofReal (leftLim f b - f a).f.measure_Iccandf.measure_Icoare analogous.Monotone.stieltjesFunction: to a monotone functionf, associate the Stieltjes function equal to the right limit off. This makes it possible to associate a Stieltjes measure to any monotone function.
Implementation #
We define Stieltjes functions over any conditionally complete dense linear order, to be able
to cover the cases of ℝ≥0 and [0, T] in addition to the classical case of ℝ. This creates
a few issues, mostly with the management of bottom and top elements. To handle these, we need
two technical definitions:
Iotop a bis the intervalIoo a bifbis not top, andIoc a bifbis top.botSetis the empty set if there is no bot element, and{x}ifxis bot.
These definitions are just handy tools for some proofs of this file, so they are only included there, and not exported.
Note that the theory of Stieltjes measures is not completely satisfactory when there is a bot
element x: any Stieljes measure gives zero mass to {x} in this case, so the Dirac mass at x
is not representable as a Stieljes measure.
Basic properties of Stieltjes functions #
Bundled monotone right-continuous real functions, used to construct Stieltjes measures.
- toFun : R → ℝ
The underlying function
ℝ → ℝ.Do NOT use directly. Use the coercion instead.
- mono' : Monotone ↑self
- right_continuous' (x : R) : ContinuousWithinAt (↑self) (Set.Ici x) x
Instances For
Equations
The identity of ℝ as a Stieltjes function, used to construct Lebesgue measure.
Equations
- StieltjesFunction.id = { toFun := id, mono' := StieltjesFunction.id._proof_1, right_continuous' := StieltjesFunction.id._proof_2 }
Instances For
Constant functions are Stieltjes function.
Equations
- StieltjesFunction.const R c = { toFun := fun (x : R) => c, mono' := ⋯, right_continuous' := ⋯ }
Instances For
Equations
- StieltjesFunction.instInhabited = { default := StieltjesFunction.const R 0 }
The sum of two Stieltjes functions is a Stieltjes function.
Instances For
Equations
- StieltjesFunction.instAddZeroClass = { zero := StieltjesFunction.const R 0, add := StieltjesFunction.add, zero_add := ⋯, add_zero := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
If a function f : R → ℝ 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.stieltjesFunction = { toFun := Function.rightLim f, mono' := ⋯, right_continuous' := ⋯ }
Instances For
The outer measure associated to a Stieltjes function #
Length of an interval. This is the largest monotone function which correctly measures all intervals.
Equations
Instances For
The Stieltjes outer measure associated to a Stieltjes function.
Equations
Instances For
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.
To be able to handle also the top element if there is one, we use Iotop instead of Ioo in the
statement. As these intervals are all open, this does not change the proof.
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]. If there is a bot element, it gives zero mass to it.