Documentation

Mathlib.MeasureTheory.Measure.LevyProkhorovMetric

The Lévy-Prokhorov distance on spaces of finite measures and probability measures #

Main definitions #

Main results #

Todo #

Tags #

finite measure, probability measure, weak convergence, convergence in distribution, metrizability

Lévy-Prokhorov metric #

The Lévy-Prokhorov edistance between measures: d(μ,ν) = inf {r ≥ 0 | ∀ B, μ B ≤ ν Bᵣ + r ∧ ν B ≤ μ Bᵣ + r}.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem MeasureTheory.meas_le_of_le_of_forall_le_meas_thickening_add {Ω : Type u_2} [MeasurableSpace Ω] [MetricSpace Ω] {ε₁ : ENNReal} {ε₂ : ENNReal} (μ : MeasureTheory.Measure Ω) (ν : MeasureTheory.Measure Ω) (h_le : ε₁ ε₂) {B : Set Ω} (hε₁ : μ B ν (Metric.thickening ε₁.toReal B) + ε₁) :
    μ B ν (Metric.thickening ε₂.toReal B) + ε₂
    theorem MeasureTheory.left_measure_le_of_levyProkhorovEDist_lt {Ω : Type u_2} [MeasurableSpace Ω] [MetricSpace Ω] {μ : MeasureTheory.Measure Ω} {ν : MeasureTheory.Measure Ω} {c : ENNReal} (h : MeasureTheory.levyProkhorovEDist μ ν < c) {B : Set Ω} (B_mble : MeasurableSet B) :
    μ B ν (Metric.thickening c.toReal B) + c
    theorem MeasureTheory.right_measure_le_of_levyProkhorovEDist_lt {Ω : Type u_2} [MeasurableSpace Ω] [MetricSpace Ω] {μ : MeasureTheory.Measure Ω} {ν : MeasureTheory.Measure Ω} {c : ENNReal} (h : MeasureTheory.levyProkhorovEDist μ ν < c) {B : Set Ω} (B_mble : MeasurableSet B) :
    ν B μ (Metric.thickening c.toReal B) + c
    theorem MeasureTheory.levyProkhorovEDist_le_of_forall_add_pos_le {Ω : Type u_2} [MeasurableSpace Ω] [MetricSpace Ω] (μ : MeasureTheory.Measure Ω) (ν : MeasureTheory.Measure Ω) (δ : ENNReal) (h : ∀ (ε : ENNReal) (B : Set Ω), 0 < εε < MeasurableSet Bμ B ν (Metric.thickening (δ + ε).toReal B) + δ + ε ν B μ (Metric.thickening (δ + ε).toReal B) + δ + ε) :
    theorem MeasureTheory.levyProkhorovEDist_le_of_forall {Ω : Type u_2} [MeasurableSpace Ω] [MetricSpace Ω] (μ : MeasureTheory.Measure Ω) (ν : MeasureTheory.Measure Ω) (δ : ENNReal) (h : ∀ (ε : ENNReal) (B : Set Ω), δ < εε < MeasurableSet Bμ B ν (Metric.thickening ε.toReal B) + ε ν B μ (Metric.thickening ε.toReal B) + ε) :

    The Lévy-Prokhorov distance between finite measures: d(μ,ν) = inf {r ≥ 0 | ∀ B, μ B ≤ ν Bᵣ + r ∧ ν B ≤ μ Bᵣ + r}.

    Equations
    Instances For

      A type synonym, to be used for Measure α, FiniteMeasure α, or ProbabilityMeasure α, when they are to be equipped with the Lévy-Prokhorov distance.

      Equations
      Instances For

        The Lévy-Prokhorov distance levyProkhorovEDist makes Measure Ω a pseudoemetric space. The instance is recorded on the type synonym LevyProkhorov (Measure Ω) := Measure Ω.

        Equations

        The Lévy-Prokhorov distance levyProkhorovDist makes FiniteMeasure Ω a pseudometric space. The instance is recorded on the type synonym LevyProkhorov (FiniteMeasure Ω) := FiniteMeasure Ω.

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

        The Lévy-Prokhorov distance levyProkhorovDist makes ProbabilityMeasure Ω a pseudoemetric space. The instance is recorded on the type synonym LevyProkhorov (ProbabilityMeasure Ω) := ProbabilityMeasure Ω.

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