Documentation

Mathlib.MeasureTheory.Function.AbsolutelyContinuous

Absolutely Continuous Functions #

This file defines absolutely continuous functions on a closed interval uIcc a b and proves some basic properties about absolutely continuous functions.

A function f is absolutely continuous on uIcc a b if for any ε > 0, there is δ > 0 such that for any finite disjoint collection of intervals uIoc (a i) (b i) for i < n where a i, b i are all in uIcc a b for i < n, if ∑ i ∈ range n, dist (a i) (b i) < δ, then ∑ i ∈ range n, dist (f (a i)) (f (b i)) < ε.

We give a filter version of the definition of absolutely continuous functions in AbsolutelyContinuousOnInterval based on AbsolutelyContinuousOnInterval.totalLengthFilter and AbsolutelyContinuousOnInterval.disjWithin and prove its equivalence with the ε-δ definition in absolutelyContinuousOnInterval_iff.

We use the filter version to prove that absolutely continuous functions are closed under

We use the the ε-δ definition to prove that

Tags #

absolutely continuous

The filter on the collection of all the finite sequences of uIoc intervals induced by the function that maps the finite sequence of the intervals to the total length of the intervals. Details:

  1. Technically the filter is on ℕ × (ℕ → X × X). A finite sequence uIoc (a i) (b i), i < n is represented by any E : ℕ × (ℕ → X × X) which satisfies E.1 = n and E.2 i = (a i, b i) for i < n. Its total length is ∑ i ∈ Finset.range n, dist (a i) (b i).
  2. For a sequence G : ℕ → ℕ × (ℕ → X × X), G convergence along totalLengthFilter means that the total length of G j, i.e., ∑ i ∈ Finset.range (G j).1, dist ((G j).2 i).1 ((G j).2 i).2), tends to 0 as j tends to infinity.
Equations
Instances For
    theorem AbsolutelyContinuousOnInterval.hasBasis_totalLengthFilter {X : Type u_1} [PseudoMetricSpace X] :
    totalLengthFilter.HasBasis (fun (ε : ) => 0 < ε) fun (ε : ) => {E : × (X × X) | iFinset.range E.1, dist (E.2 i).1 (E.2 i).2 < ε}

    The subcollection of all the finite sequences of uIoc intervals consisting of uIoc (a i) (b i), i < n where a i, b i are all in uIcc a b for i < n and uIoc (a i) (b i) are mutually disjoint for i < n. Technically the finite sequence uIoc (a i) (b i), i < n is represented by any E : ℕ × (ℕ → ℝ × ℝ) which satisfies E.1 = n and E.2 i = (a i, b i) for i < n.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      def AbsolutelyContinuousOnInterval {X : Type u_1} [PseudoMetricSpace X] (f : X) (a b : ) :

      AbsolutelyContinuousOnInterval f a b: A function f is absolutely continuous on uIcc a b if the function which (intuitively) maps uIoc (a i) (b i), i < n to ∑ i ∈ Finset.range n, dist (f (a i)) (f (b i)) tendsto 𝓝 0 wrt totalLengthFilter restricted to disjWithin a b. This is equivalent to the traditional ε-δ definition: for any ε > 0, there is δ > 0 such that for any finite disjoint collection of intervals uIoc (a i) (b i) for i < n where a i, b i are all in uIcc a b for i < n, if ∑ i ∈ range n, dist (a i) (b i) < δ, then ∑ i ∈ range n, dist (f (a i)) (f (b i)) < ε.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem absolutelyContinuousOnInterval_iff {X : Type u_1} [PseudoMetricSpace X] (f : X) (a b : ) :
        AbsolutelyContinuousOnInterval f a b ε > 0, δ > 0, EAbsolutelyContinuousOnInterval.disjWithin a b, iFinset.range E.1, dist (E.2 i).1 (E.2 i).2 < δiFinset.range E.1, dist (f (E.2 i).1) (f (E.2 i).2) < ε

        The traditional ε-δ definition of absolutely continuous: A function f is absolutely continuous on uIcc a b if for any ε > 0, there is δ > 0 such that for any finite disjoint collection of intervals uIoc (a i) (b i) for i < n where a i, b i are all in uIcc a b for i < n, if ∑ i ∈ range n, dist (a i) (b i) < δ, then ∑ i ∈ range n, dist (f (a i)) (f (b i)) < ε.

        theorem AbsolutelyContinuousOnInterval.const_smul {F : Type u_2} [SeminormedAddCommGroup F] {a b : } {f : F} {M : Type u_3} [SeminormedRing M] [Module M F] [NormSMulClass M F] (α : M) (hf : AbsolutelyContinuousOnInterval f a b) :
        AbsolutelyContinuousOnInterval (fun (x : ) => α f x) a b

        If f is absolutely continuous on uIcc a b, then f is uniformly continuous on uIcc a b.

        If f is absolutely continuous on uIcc a b, then f is continuous on uIcc a b.

        theorem AbsolutelyContinuousOnInterval.exists_bound {F : Type u_2} [SeminormedAddCommGroup F] {a b : } {f : F} (hf : AbsolutelyContinuousOnInterval f a b) :
        ∃ (C : ), xSet.uIcc a b, f x C

        If f is absolutely continuous on uIcc a b, then f is bounded on uIcc a b.

        theorem AbsolutelyContinuousOnInterval.fun_smul {F : Type u_2} [SeminormedAddCommGroup F] {a b : } {M : Type u_3} [SeminormedRing M] [Module M F] [NormSMulClass M F] {f : M} {g : F} (hf : AbsolutelyContinuousOnInterval f a b) (hg : AbsolutelyContinuousOnInterval g a b) :
        AbsolutelyContinuousOnInterval (fun (x : ) => f x g x) a b

        If f and g are absolutely continuous on uIcc a b, then f • g is absolutely continuous on uIcc a b.

        If f and g are absolutely continuous on uIcc a b, then f • g is absolutely continuous on uIcc a b.

        If f and g are absolutely continuous on uIcc a b, then f * g is absolutely continuous on uIcc a b.

        If f and g are absolutely continuous on uIcc a b, then f * g is absolutely continuous on uIcc a b.

        If f is Lipschitz on uIcc a b, then f is absolutely continuous on uIcc a b.

        If f is absolutely continuous on uIcc a b, then f has bounded variation on uIcc a b.