Pareto distributions over ℝ #
Define the Pareto measure over the reals.
Main definitions #
paretoPDFReal
: the functiont r x ↦ r * t ^ r * x ^ -(r + 1)
fort ≤ x
or0
else, which is the probability density function of a Pareto distribution with scalet
and shaper
(whenht : 0 < t
andhr : 0 < r
).paretoPDF
:ℝ≥0∞
-valued pdf,paretoPDF t r = ENNReal.ofReal (paretoPDFReal t r)
.paretoMeasure
: a Pareto measure onℝ
, parametrized by its scalet
and shaper
.paretoCDFReal
: the CDF given by the definition of CDF inProbabilityTheory.CDF
applied to the Pareto measure.
The pdf of the Pareto distribution, as a function valued in ℝ≥0∞
.
Equations
Instances For
The Pareto pdf is measurable.
The Pareto pdf is strongly measurable.
theorem
ProbabilityTheory.paretoPDFReal_pos
{t r x : ℝ}
(ht : 0 < t)
(hr : 0 < r)
(hx : t ≤ x)
:
0 < paretoPDFReal t r x
The Pareto pdf is positive for all reals >= t
.
theorem
ProbabilityTheory.paretoPDFReal_nonneg
{t r : ℝ}
(ht : 0 ≤ t)
(hr : 0 ≤ r)
(x : ℝ)
:
0 ≤ paretoPDFReal t r x
The Pareto pdf is nonnegative.
Measure defined by the Pareto distribution.
Equations
- ProbabilityTheory.paretoMeasure t r = MeasureTheory.volume.withDensity (ProbabilityTheory.paretoPDF t r)
Instances For
theorem
ProbabilityTheory.paretoCDFReal_eq_integral
{t r : ℝ}
(ht : 0 < t)
(hr : 0 < r)
(x : ℝ)
:
↑(cdf (paretoMeasure t r)) x = ∫ (x : ℝ) in Set.Iic x, paretoPDFReal t r x
CDF of the Pareto distribution equals the integral of the PDF.