Documentation

Mathlib.Probability.Variance

Variance of random variables #

We define the variance of a real-valued random variable as Var[X] = 𝔼[(X - 𝔼[X])^2] (in the ProbabilityTheory locale).

Main definitions #

Main results #

def ProbabilityTheory.evariance {Ω : Type u_1} {x✝ : MeasurableSpace Ω} (X : Ω) (μ : MeasureTheory.Measure Ω) :

The ℝ≥0∞-valued variance of a real-valued random variable defined as the Lebesgue integral of (X - 𝔼[X])^2.

Equations
Instances For
    def ProbabilityTheory.variance {Ω : Type u_1} {x✝ : MeasurableSpace Ω} (X : Ω) (μ : MeasureTheory.Measure Ω) :

    The -valued variance of a real-valued random variable defined by applying ENNReal.toReal to evariance.

    Equations
    Instances For

      The ℝ≥0∞-valued variance of the real-valued random variable X according to the measure μ.

      This is defined as the Lebesgue integral of (X - 𝔼[X])^2.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        The ℝ≥0∞-valued variance of the real-valued random variable X according to the volume measure.

        This is defined as the Lebesgue integral of (X - 𝔼[X])^2.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For

          The -valued variance of the real-valued random variable X according to the measure μ.

          It is set to 0 if X has infinite variance.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For

            The -valued variance of the real-valued random variable X according to the volume measure.

            It is set to 0 if X has infinite variance.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              theorem MeasureTheory.Memℒp.evariance_lt_top {Ω : Type u_1} {m : MeasurableSpace Ω} {X : Ω} {μ : Measure Ω} [IsFiniteMeasure μ] (hX : Memℒp X 2 μ) :
              theorem ProbabilityTheory.evariance_eq_lintegral_ofReal {Ω : Type u_1} {m : MeasurableSpace Ω} (X : Ω) (μ : MeasureTheory.Measure Ω) :
              evariance X μ = ∫⁻ (ω : Ω), ENNReal.ofReal ((X ω - (x : Ω), X x μ) ^ 2) μ
              theorem MeasureTheory.Memℒp.variance_eq_of_integral_eq_zero {Ω : Type u_1} {m : MeasurableSpace Ω} {X : Ω} {μ : Measure Ω} (hX : Memℒp X 2 μ) (hXint : (x : Ω), X x μ = 0) :
              ProbabilityTheory.variance X μ = (x : Ω), (X ^ 2) x μ
              theorem MeasureTheory.Memℒp.variance_eq {Ω : Type u_1} {m : MeasurableSpace Ω} {X : Ω} {μ : Measure Ω} [IsFiniteMeasure μ] (hX : Memℒp X 2 μ) :
              ProbabilityTheory.variance X μ = (x : Ω), ((X - fun (x : Ω) => (x : Ω), X x μ) ^ 2) x μ
              @[simp]
              theorem ProbabilityTheory.evariance_eq_zero_iff {Ω : Type u_1} {m : MeasurableSpace Ω} {X : Ω} {μ : MeasureTheory.Measure Ω} (hX : AEMeasurable X μ) :
              evariance X μ = 0 X =ᵐ[μ] fun (x : Ω) => (x : Ω), X x μ
              theorem ProbabilityTheory.evariance_mul {Ω : Type u_1} {m : MeasurableSpace Ω} (c : ) (X : Ω) (μ : MeasureTheory.Measure Ω) :
              evariance (fun (ω : Ω) => c * X ω) μ = ENNReal.ofReal (c ^ 2) * evariance X μ
              @[simp]
              theorem ProbabilityTheory.variance_nonneg {Ω : Type u_1} {m : MeasurableSpace Ω} (X : Ω) (μ : MeasureTheory.Measure Ω) :
              0 variance X μ
              theorem ProbabilityTheory.variance_mul {Ω : Type u_1} {m : MeasurableSpace Ω} (c : ) (X : Ω) (μ : MeasureTheory.Measure Ω) :
              variance (fun (ω : Ω) => c * X ω) μ = c ^ 2 * variance X μ
              theorem ProbabilityTheory.variance_smul {Ω : Type u_1} {m : MeasurableSpace Ω} (c : ) (X : Ω) (μ : MeasureTheory.Measure Ω) :
              variance (c X) μ = c ^ 2 * variance X μ
              theorem ProbabilityTheory.variance_smul' {Ω : Type u_1} {m : MeasurableSpace Ω} {A : Type u_2} [CommSemiring A] [Algebra A ] (c : A) (X : Ω) (μ : MeasureTheory.Measure Ω) :
              variance (c X) μ = c ^ 2 variance X μ
              theorem ProbabilityTheory.variance_def' {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure μ] {X : Ω} (hX : MeasureTheory.Memℒp X 2 μ) :
              variance X μ = (x : Ω), (X ^ 2) x μ - ( (x : Ω), X x μ) ^ 2
              theorem ProbabilityTheory.evariance_def' {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure μ] {X : Ω} (hX : MeasureTheory.AEStronglyMeasurable X μ) :
              evariance X μ = ∫⁻ (ω : Ω), (X ω‖₊ ^ 2) μ - ENNReal.ofReal (( (x : Ω), X x μ) ^ 2)
              theorem ProbabilityTheory.meas_ge_le_evariance_div_sq {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} {X : Ω} (hX : MeasureTheory.AEStronglyMeasurable X μ) {c : NNReal} (hc : c 0) :
              μ {ω : Ω | c |X ω - (x : Ω), X x μ|} evariance X μ / c ^ 2

              Chebyshev's inequality for ℝ≥0∞-valued variance.

              theorem ProbabilityTheory.meas_ge_le_variance_div_sq {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsFiniteMeasure μ] {X : Ω} (hX : MeasureTheory.Memℒp X 2 μ) {c : } (hc : 0 < c) :
              μ {ω : Ω | c |X ω - (x : Ω), X x μ|} ENNReal.ofReal (variance X μ / c ^ 2)

              Chebyshev's inequality: one can control the deviation probability of a real random variable from its expectation in terms of the variance.

              theorem ProbabilityTheory.IndepFun.variance_add {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure μ] {X Y : Ω} (hX : MeasureTheory.Memℒp X 2 μ) (hY : MeasureTheory.Memℒp Y 2 μ) (h : IndepFun X Y μ) :
              variance (X + Y) μ = variance X μ + variance Y μ

              The variance of the sum of two independent random variables is the sum of the variances.

              theorem ProbabilityTheory.IndepFun.variance_sum {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure μ] {ι : Type u_2} {X : ιΩ} {s : Finset ι} (hs : is, MeasureTheory.Memℒp (X i) 2 μ) (h : (↑s).Pairwise fun (i j : ι) => IndepFun (X i) (X j) μ) :
              variance (∑ is, X i) μ = is, variance (X i) μ

              The variance of a finite sum of pairwise independent random variables is the sum of the variances.

              theorem ProbabilityTheory.variance_le_sub_mul_sub {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure μ] {a b : } {X : Ω} (h : ∀ᵐ (ω : Ω) μ, X ω Set.Icc a b) (hX : AEMeasurable X μ) :
              variance X μ (b - (x : Ω), X x μ) * ( (x : Ω), X x μ - a)

              The Bhatia-Davis inequality on variance

              The variance of a random variable X satisfying a ≤ X ≤ b almost everywhere is at most (b - 𝔼 X) * (𝔼 X - a).

              theorem ProbabilityTheory.variance_le_sq_of_bounded {Ω : Type u_1} {m : MeasurableSpace Ω} {μ : MeasureTheory.Measure Ω} [MeasureTheory.IsProbabilityMeasure μ] {a b : } {X : Ω} (h : ∀ᵐ (ω : Ω) μ, X ω Set.Icc a b) (hX : AEMeasurable X μ) :
              variance X μ ((b - a) / 2) ^ 2

              Popoviciu's inequality on variance

              The variance of a random variable X satisfying a ≤ X ≤ b almost everywhere is at most ((b - a) / 2) ^ 2.