Documentation

Mathlib.Analysis.Calculus.LineDeriv.Measurable

Measurability of the line derivative #

We prove in measurable_lineDeriv that the line derivative of a function (with respect to a locally compact scalar field) is measurable, provided the function is continuous.

In measurable_lineDeriv_uncurry, assuming additionally that the source space is second countable, we show that (x, v) ↦ lineDeriv 𝕜 f x v is also measurable.

An assumption such as continuity is necessary, as otherwise one could alternate in a non-measurable way between differentiable and non-differentiable functions along the various lines directed by v.

Measurability of the line derivative lineDeriv 𝕜 f x v with respect to a fixed direction v.

theorem measurable_lineDeriv {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] [LocallyCompactSpace 𝕜] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace 𝕜 E] [MeasurableSpace E] [OpensMeasurableSpace E] {F : Type u_3} [NormedAddCommGroup F] [NormedSpace 𝕜 F] [CompleteSpace F] {f : EF} {v : E} [MeasurableSpace F] [BorelSpace F] (hf : Continuous f) :
Measurable fun (x : E) => lineDeriv 𝕜 f x v
theorem aemeasurable_lineDeriv {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] [LocallyCompactSpace 𝕜] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace 𝕜 E] [MeasurableSpace E] [OpensMeasurableSpace E] {F : Type u_3} [NormedAddCommGroup F] [NormedSpace 𝕜 F] [CompleteSpace F] {f : EF} {v : E} [MeasurableSpace F] [BorelSpace F] (hf : Continuous f) (μ : MeasureTheory.Measure E) :
AEMeasurable (fun (x : E) => lineDeriv 𝕜 f x v) μ

Measurability of the line derivative lineDeriv 𝕜 f x v when varying both x and v. For this, we need an additional second countability assumption on E to make sure that open sets are measurable in E × E.

theorem aemeasurable_lineDeriv_uncurry {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] [LocallyCompactSpace 𝕜] {E : Type u_2} [NormedAddCommGroup E] [NormedSpace 𝕜 E] [MeasurableSpace E] [OpensMeasurableSpace E] {F : Type u_3} [NormedAddCommGroup F] [NormedSpace 𝕜 F] [CompleteSpace F] {f : EF} [SecondCountableTopology E] [MeasurableSpace F] [BorelSpace F] (hf : Continuous f) (μ : MeasureTheory.Measure (E × E)) :
AEMeasurable (fun (p : E × E) => lineDeriv 𝕜 f p.1 p.2) μ