Beta distributions over ℝ #
Define the beta distribution over the reals.
Main definitions #
betaPDFReal: the functionα β x ↦ (1 / beta α β) * x ^ (α - 1) * (1 - x) ^ (β - 1)for0 < x ∧ x < 1or0else, which is the probability density function of a beta distribution with shape parametersαandβ(when0 < αand0 < β).betaPDF:ℝ≥0∞-valued pdf,betaPDF α β = ENNReal.ofReal (betaPDFReal α β).
The normalizing constant in the beta distribution.
Equations
- ProbabilityTheory.beta α β = Real.Gamma α * Real.Gamma β / Real.Gamma (α + β)
Instances For
Relation between the beta function and the gamma function over the reals.
The probability density function of the beta distribution with shape parameters α and β.
Returns (1 / beta α β) * x ^ (α - 1) * (1 - x) ^ (β - 1)
when 0 < x < 1 and 0 otherwise.
Equations
Instances For
The pdf of the beta distribution, as a function valued in ℝ≥0∞.
Equations
Instances For
The beta pdf is measurable.
The beta pdf is strongly measurable.
Measure defined by the beta distribution.