Gamma distributions over ℝ #
Define the gamma measure over the reals.
Main definitions #
gammaPDFReal
: the functiona r x ↦ r ^ a / (Gamma a) * x ^ (a-1) * exp (-(r * x))
for0 ≤ x
or0
else, which is the probability density function of a gamma distribution with shapea
and rater
(whenha : 0 < a
andhr : 0 < r
).gammaPDF
:ℝ≥0∞
-valued pdf,gammaPDF a r = ENNReal.ofReal (gammaPDFReal a r)
.gammaMeasure
: a gamma measure onℝ
, parametrized by its shapea
and rater
.gammaCDFReal
: the CDF given by the definition of CDF inProbabilityTheory.CDF
applied to the gamma measure.
The pdf of the gamma distribution, as a function valued in ℝ≥0∞
Equations
Instances For
The gamma pdf is measurable.
The gamma pdf is strongly measurable
theorem
ProbabilityTheory.gammaPDFReal_pos
{x a r : ℝ}
(ha : 0 < a)
(hr : 0 < r)
(hx : 0 < x)
:
0 < gammaPDFReal a r x
The gamma pdf is positive for all positive reals
theorem
ProbabilityTheory.gammaPDFReal_nonneg
{a r : ℝ}
(ha : 0 < a)
(hr : 0 < r)
(x : ℝ)
:
0 ≤ gammaPDFReal a r x
The gamma pdf is nonnegative
Measure defined by the gamma distribution
Equations
- ProbabilityTheory.gammaMeasure a r = MeasureTheory.volume.withDensity (ProbabilityTheory.gammaPDF a r)
Instances For
CDF of the gamma distribution
Equations
Instances For
theorem
ProbabilityTheory.gammaCDFReal_eq_integral
{a r : ℝ}
(ha : 0 < a)
(hr : 0 < r)
(x : ℝ)
:
↑(gammaCDFReal a r) x = ∫ (x : ℝ) in Set.Iic x, gammaPDFReal a r x