Documentation

Mathlib.MeasureTheory.Integral.IntervalIntegral.LebesgueDifferentiationThm

Lebesgue Differentiation Theorem (Interval Version) #

This file proves the interval version of the Lebesgue Differentiation Theorem. There are two versions in this file.

theorem LocallyIntegrable.ae_hasDerivAt_integral {f : } (hf : MeasureTheory.LocallyIntegrable f MeasureTheory.volume) :
∀ᵐ (x : ), ∀ (c : ), HasDerivAt (fun (x : ) => (t : ) in c..x, f t) (f x) x

The (global) interval version of the Lebesgue Differentiation Theorem: if f : ℝ → ℝ is locally integrable, then for almost every x, for any c : ℝ, the derivative of ∫ (t : ℝ) in c..x, f t at x is equal to f x.

theorem IntervalIntegrable.ae_hasDerivAt_integral {f : } {a b : } (hf : IntervalIntegrable f MeasureTheory.volume a b) :
∀ᵐ (x : ), x Set.uIcc a bcSet.uIcc a b, HasDerivAt (fun (x : ) => (t : ) in c..x, f t) (f x) x

The (local) interval version of the Lebesgue Differentiation Theorem: if f : ℝ → ℝ is interval integrable on a..b, then for almost every x ∈ uIcc a b, for any c ∈ uIcc a b, the derivative of ∫ (t : ℝ) in c..x, f t at x is equal to f x.