Poisson distributions over ℕ #
Define the Poisson measure over the natural numbers
Main definitions #
- poissonPMFReal: the function- fun n ↦ exp (- λ) * λ ^ n / n!for- n ∈ ℕ, which is the probability density function of a Poisson distribution with rate- λ > 0.
- poissonPMF:- ℝ≥0∞-valued pdf,- poissonPMF λ = ENNReal.ofReal (poissonPMFReal λ).
- poissonMeasure: a Poisson measure on- ℕ, parametrized by its rate- λ.
theorem
ProbabilityTheory.poissonPMFRealSum
(r : NNReal)
 :
HasSum (fun (n : ℕ) => poissonPMFReal r n) 1
The Poisson pmf is positive for all natural numbers
The pmf of the Poisson distribution depending on its rate, as a PMF.
Equations
- ProbabilityTheory.poissonPMF r = ⟨fun (n : ℕ) => ENNReal.ofReal (ProbabilityTheory.poissonPMFReal r n), ⋯⟩
Instances For
The Poisson pmf is measurable.
Measure defined by the Poisson distribution