Documentation

BrownianMotion.Continuity.KolmogorovChentsov

Kolmogorov-Chentsov theorem #

theorem measurable_limUnder {ι : Type u_1} {X : Type u_2} {E : Type u_3} [MeasurableSpace X] [TopologicalSpace E] [PolishSpace E] [MeasurableSpace E] [BorelSpace E] [Countable ι] {l : Filter ι} [l.IsCountablyGenerated] {f : ιXE} [hE : Nonempty E] (hf : ∀ (i : ι), Measurable (f i)) :
Measurable fun (x : X) => limUnder l fun (x_1 : ι) => f x_1 x
theorem MeasureTheory.Measure.measure_inter_eq_of_measure_eq_measure_univ {α : Type u_1} {x✝ : MeasurableSpace α} {μ : Measure α} {s t : Set α} (hs : MeasurableSet s) (h : μ t = μ Set.univ) (ht_ne_top : μ t ) :
μ (t s) = μ s
theorem MeasureTheory.Measure.measure_inter_eq_of_ae {α : Type u_1} {x✝ : MeasurableSpace α} {μ : Measure α} [IsFiniteMeasure μ] {s t : Set α} (hs : MeasurableSet s) (ht : NullMeasurableSet t μ) (h : ∀ᵐ (a : α) μ, a t) (ht_ne_top : μ t ) :
μ (t s) = μ s
theorem Asymptotics.IsEquivalent.add_const_of_norm_tendsto_atTop {α : Type u_1} {β : Type u_2} [NormedField β] [LinearOrder β] [IsStrictOrderedRing β] {u v : αβ} {l : Filter α} {c : β} (huv : IsEquivalent l u v) (hv : Filter.Tendsto (norm v) l Filter.atTop) :
IsEquivalent l (fun (x : α) => u x + c) v
theorem Asymptotics.IsEquivalent.const_add_of_norm_tendsto_atTop {α : Type u_1} {β : Type u_2} [NormedField β] [LinearOrder β] [IsStrictOrderedRing β] {u v : αβ} {l : Filter α} {c : β} (huv : IsEquivalent l u v) (hv : Filter.Tendsto (norm v) l Filter.atTop) :
IsEquivalent l (fun (x : α) => c + u x) v
theorem Asymptotics.IsEquivalent.add_add_of_nonneg {α : Type u_1} {t u v w : α} (hu : 0 u) (hw : 0 w) {l : Filter α} (htu : IsEquivalent l t u) (hvw : IsEquivalent l v w) :
IsEquivalent l (t + v) (u + w)
theorem Asymptotics.IsEquivalent.rpow_of_nonneg {α : Type u_1} {t u : α} (hu : 0 u) {l : Filter α} (h : IsEquivalent l t u) {r : } :
IsEquivalent l (t ^ r) (u ^ r)
theorem Set.iUnion_le_nat :
⋃ (n : ), {i : | i n} = univ
structure FiniteExhaustion {α : Type u_1} (s : Set α) :
Type u_1
Instances For
    instance FiniteExhaustion.instFiniteElemCoeNatSet {α : Type u_1} {s : Set α} {K : FiniteExhaustion s} {n : } :
    Finite (K n)
    @[simp]
    theorem FiniteExhaustion.toFun_eq_coe {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) :
    K.toFun = K
    theorem FiniteExhaustion.Finite {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) (n : ) :
    (K n).Finite
    theorem FiniteExhaustion.subset_succ {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) (n : ) :
    K n K (n + 1)
    theorem FiniteExhaustion.subset {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) {m n : } (h : m n) :
    K m K n
    theorem FiniteExhaustion.iUnion_eq {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) :
    ⋃ (n : ), K n = s
    noncomputable def FiniteExhaustion.choice {α : Type u_2} (s : Set α) [Countable s] :
    Equations
    Instances For
      def FiniteExhaustion.prod {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) {β : Type u_2} {t : Set β} (K' : FiniteExhaustion t) :
      Equations
      • K.prod K' = { toFun := fun (n : ) => K n ×ˢ K' n, Finite' := , subset_succ' := , iUnion_eq' := }
      Instances For
        theorem FiniteExhaustion.prod_apply {α : Type u_1} {s : Set α} (K : FiniteExhaustion s) {β : Type u_2} {t : Set β} (K' : FiniteExhaustion t) (n : ) :
        (K.prod K') n = K n ×ˢ K' n
        theorem measure_add_ge_le_add_measure_ge {Ω : Type u_1} {x✝ : MeasurableSpace Ω} {P : MeasureTheory.Measure Ω} {f g : ΩENNReal} {x u : ENNReal} (hu : u x) :
        P {ω : Ω | x f ω + g ω} P {ω : Ω | u f ω} + P {ω : Ω | x - u g ω}
        theorem measure_add_ge_le_add_measure_ge_half {Ω : Type u_1} {x✝ : MeasurableSpace Ω} {P : MeasureTheory.Measure Ω} {f g : ΩENNReal} {x : ENNReal} :
        P {ω : Ω | x f ω + g ω} P {ω : Ω | x / 2 f ω} + P {ω : Ω | x / 2 g ω}
        theorem ProbabilityTheory.lintegral_div_edist_le_sum_integral_edist_le {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoEMetricSpace T] [PseudoEMetricSpace E] [MeasurableSpace E] [BorelSpace E] (hT : EMetric.diam Set.univ < ) (hX : IsAEKolmogorovProcess X P p q M) ( : 0 < β) {J : Set T} [Countable J] :
        ∫⁻ (ω : Ω), ⨆ (s : J), ⨆ (t : J), edist (X (↑s) ω) (X (↑t) ω) ^ p / edist s t ^ (β * p) P ∑' (k : ), 2 ^ (k * β * p) * ∫⁻ (ω : Ω), ⨆ (s : J), ⨆ (t : { t : J // edist s t 2 * 2⁻¹ ^ k * (EMetric.diam Set.univ + 1) }), edist (X (↑s) ω) (X (↑t) ω) ^ p P
        noncomputable def ProbabilityTheory.constL (T : Type u_4) [PseudoEMetricSpace T] (c : ENNReal) (d p q β : ) :
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          theorem ProbabilityTheory.constL_lt_top {T : Type u_1} {c : ENNReal} {d p q : } {β : NNReal} [PseudoEMetricSpace T] (hT : EMetric.diam Set.univ < ) (hc : c ) (hd_pos : 0 < d) (hp_pos : 0 < p) (hdq_lt : d < q) (hβ_lt : β < (q - d) / p) :
          constL T c d p q β <
          theorem ProbabilityTheory.finite_kolmogorov_chentsov {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {c : ENNReal} {d p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoEMetricSpace T] [PseudoEMetricSpace E] [MeasurableSpace E] [BorelSpace E] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hX : IsAEKolmogorovProcess X P p q M) (hd_pos : 0 < d) (hdq_lt : d < q) (hβ_pos : 0 < β) (T' : Set T) [hT' : Finite T'] :
          ∫⁻ (ω : Ω), ⨆ (s : T'), ⨆ (t : T'), edist (X (↑s) ω) (X (↑t) ω) ^ p / edist s t ^ (β * p) P M * constL T c d p q β
          theorem ProbabilityTheory.countable_kolmogorov_chentsov {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {c : ENNReal} {d p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoEMetricSpace T] [PseudoEMetricSpace E] [MeasurableSpace E] [BorelSpace E] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hX : IsAEKolmogorovProcess X P p q M) (hd_pos : 0 < d) (hdq_lt : d < q) (hβ_pos : 0 < β) (T' : Set T) [Countable T'] :
          ∫⁻ (ω : Ω), ⨆ (s : T'), ⨆ (t : T'), edist (X (↑s) ω) (X (↑t) ω) ^ p / edist s t ^ (β * p) P M * constL T c d p q β
          theorem ProbabilityTheory.IsKolmogorovProcess.ae_iSup_rpow_edist_div_lt_top {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {c : ENNReal} {d p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] [MeasurableSpace E] [BorelSpace E] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hX : IsKolmogorovProcess X P p q M) (hc : c ) (hd_pos : 0 < d) (hdq_lt : d < q) (hβ_pos : 0 < β) (hβ_lt : β < (q - d) / p) {T' : Set T} (hT' : T'.Countable) :
          ∀ᵐ (ω : Ω) P, ⨆ (s : T'), ⨆ (t : T'), edist (X (↑s) ω) (X (↑t) ω) ^ p / edist s t ^ (β * p) <
          def ProbabilityTheory.holderSet {T : Type u_1} {Ω : Type u_2} {E : Type u_3} [PseudoMetricSpace T] [EMetricSpace E] (X : TΩE) (T' : Set T) (p β : ) :
          Set Ω
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem ProbabilityTheory.IsKolmogorovProcess.measurableSet_holderSet {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] (hX : IsKolmogorovProcess X P p q M) {T' : Set T} (hT' : T'.Countable) :
            MeasurableSet (holderSet X T' p β)
            theorem ProbabilityTheory.holderWith_of_mem_holderSet {T : Type u_1} {Ω : Type u_2} {E : Type u_3} {X : TΩE} {c : ENNReal} {d p : } {β : NNReal} [PseudoMetricSpace T] [EMetricSpace E] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hd_pos : 0 < d) (hp_pos : 0 < p) (hβ_pos : 0 < β) {T' : Set T} {ω : Ω} ( : ω holderSet X T' p β) :
            HolderWith ((fun (ω : Ω) => ⨆ (s : T'), ⨆ (t : T'), edist (X (↑s) ω) (X (↑t) ω) ^ p / edist s t ^ (β * p)) ω ^ p⁻¹).toNNReal β fun (t : T') => X (↑t) ω
            theorem ProbabilityTheory.uniformContinuous_of_mem_holderSet {T : Type u_1} {Ω : Type u_2} {E : Type u_3} {X : TΩE} {c : ENNReal} {d p : } {β : NNReal} [PseudoMetricSpace T] [EMetricSpace E] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hd_pos : 0 < d) (hp_pos : 0 < p) (hβ_pos : 0 < β) {T' : Set T} {ω : Ω} ( : ω holderSet X T' p β) :
            UniformContinuous fun (t : T') => X (↑t) ω
            theorem ProbabilityTheory.continuous_of_mem_holderSet {T : Type u_1} {Ω : Type u_2} {E : Type u_3} {X : TΩE} {c : ENNReal} {d p : } {β : NNReal} [PseudoMetricSpace T] [EMetricSpace E] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hd_pos : 0 < d) (hp_pos : 0 < p) (hβ_pos : 0 < β) {T' : Set T} {ω : Ω} ( : ω holderSet X T' p β) :
            Continuous fun (t : T') => X (↑t) ω
            theorem ProbabilityTheory.IsKolmogorovProcess.tendstoInMeasure_of_mem_holderSet {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {p q : } {M : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] (hX : IsKolmogorovProcess X P p q M) (hq_pos : 0 < q) {T' : Set T} {u : T'} {t : T} (hu : Filter.Tendsto (fun (n : ) => (u n)) Filter.atTop (nhds t)) :
            MeasureTheory.TendstoInMeasure P (fun (n : ) => X (u n)) Filter.atTop (X t)
            theorem ProbabilityTheory.exists_modification_holder_aux' {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {c : ENNReal} {d p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] [MeasurableSpace E] [BorelSpace E] [Nonempty E] [SecondCountableTopology T] [CompleteSpace E] [SecondCountableTopology E] [MeasureTheory.IsFiniteMeasure P] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hX : IsKolmogorovProcess X P p q M) (hc : c ) (hd_pos : 0 < d) (hdq_lt : d < q) (hβ_pos : 0 < β) (hβ_lt : β < (q - d) / p) :
            ∃ (Y : TΩE), (∀ (t : T), Measurable (Y t)) (∀ (t : T), Y t =ᵐ[P] X t) ∀ (ω : Ω), ∃ (C : NNReal), HolderWith C β fun (x : T) => Y x ω
            theorem ProbabilityTheory.exists_modification_holder_aux {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {c : ENNReal} {d p q : } {M β : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] [MeasurableSpace E] [BorelSpace E] [Nonempty E] [SecondCountableTopology T] [CompleteSpace E] [SecondCountableTopology E] [MeasureTheory.IsFiniteMeasure P] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hX : IsAEKolmogorovProcess X P p q M) (hc : c ) (hd_pos : 0 < d) (hdq_lt : d < q) (hβ_pos : 0 < β) (hβ_lt : β < (q - d) / p) :
            ∃ (Y : TΩE), (∀ (t : T), Measurable (Y t)) (∀ (t : T), Y t =ᵐ[P] X t) ∀ (ω : Ω), MemHolder β fun (x : T) => Y x ω
            theorem ProbabilityTheory.StronglyMeasurable.measurableSet_eq_of_continuous {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} [PseudoMetricSpace T] [EMetricSpace E] [SecondCountableTopology T] {f g : TΩE} (hf : ∀ (ω : Ω), Continuous fun (x : T) => f x ω) (hg : ∀ (ω : Ω), Continuous fun (x : T) => g x ω) (hf_meas : ∀ (t : T), MeasureTheory.StronglyMeasurable (f t)) (hg_meas : ∀ (t : T), MeasureTheory.StronglyMeasurable (g t)) :
            MeasurableSet {ω : Ω | ∀ (t : T), f t ω = g t ω}
            theorem ProbabilityTheory.exists_modification_holder {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {c : ENNReal} {d p q : } {M : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] [MeasurableSpace E] [BorelSpace E] [Nonempty E] [SecondCountableTopology T] [CompleteSpace E] [SecondCountableTopology E] [MeasureTheory.IsFiniteMeasure P] (hT : HasBoundedInternalCoveringNumber Set.univ c d) (hX : IsAEKolmogorovProcess X P p q M) (hc : c ) (hd_pos : 0 < d) (hdq_lt : d < q) :
            ∃ (Y : TΩE), (∀ (t : T), Measurable (Y t)) (∀ (t : T), Y t =ᵐ[P] X t) ∀ (β : NNReal), 0 < ββ < (q - d) / p∀ (ω : Ω), MemHolder β fun (x : T) => Y x ω
            theorem ProbabilityTheory.exists_modification_holder' {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {d p q : } {M : NNReal} {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] [MeasurableSpace E] [BorelSpace E] [Nonempty E] [SecondCountableTopology T] [CompleteSpace E] [SecondCountableTopology E] [MeasureTheory.IsFiniteMeasure P] {C : Set T} {c : ENNReal} (hC : IsCoverWithBoundedCoveringNumber C Set.univ c fun (x : ) => d) (hX : IsAEKolmogorovProcess X P p q M) (hc : ∀ (n : ), c n ) (hd_pos : 0 < d) (hdq_lt : d < q) :
            ∃ (Y : TΩE), (∀ (t : T), Measurable (Y t)) (∀ (t : T), Y t =ᵐ[P] X t) ∀ (ω : Ω) (t : T), Unhds t, ∀ (β : NNReal), 0 < ββ < (q - d) / p∃ (C : NNReal), HolderOnWith C β (fun (x : T) => Y x ω) U
            theorem ProbabilityTheory.exists_modification_holder_iSup {T : Type u_1} {Ω : Type u_2} {E : Type u_3} { : MeasurableSpace Ω} {X : TΩE} {d : } {P : MeasureTheory.Measure Ω} [PseudoMetricSpace T] [EMetricSpace E] [MeasurableSpace E] [BorelSpace E] [Nonempty E] [SecondCountableTopology T] [CompleteSpace E] [SecondCountableTopology E] [MeasureTheory.IsFiniteMeasure P] {C : Set T} {c : ENNReal} {p q : } {M : NNReal} (hC : IsCoverWithBoundedCoveringNumber C Set.univ c fun (x : ) => d) (hX : ∀ (n : ), IsAEKolmogorovProcess X P (p n) (q n) (M n)) (hc : ∀ (n : ), c n ) (hd_pos : 0 < d) (hdq_lt : ∀ (n : ), d < q n) :
            ∃ (Y : TΩE), (∀ (t : T), Measurable (Y t)) (∀ (t : T), Y t =ᵐ[P] X t) ∀ (ω : Ω) (t : T) (β : NNReal), 0 < ββ < ⨆ (n : ), (q n - d) / p nUnhds t, ∃ (C : NNReal), HolderOnWith C β (fun (x : T) => Y x ω) U