Documentation

Mathlib.MeasureTheory.Function.SpecialFunctions.Sinc

Measurability and integrability of the sinc function #

Main statements #

theorem Measurable.sinc {α : Type u_1} {x✝ : MeasurableSpace α} {f : α} (hf : Measurable f) :
Measurable fun (x : α) => Real.sinc (f x)
theorem AEMeasurable.sinc {α : Type u_1} {x✝ : MeasurableSpace α} {f : α} {μ : MeasureTheory.Measure α} (hf : AEMeasurable f μ) :
AEMeasurable (fun (x : α) => Real.sinc (f x)) μ
theorem MeasureTheory.StronglyMeasurable.sinc {α : Type u_1} {x✝ : MeasurableSpace α} {f : α} (hf : StronglyMeasurable f) :
StronglyMeasurable fun (x : α) => Real.sinc (f x)
theorem MeasureTheory.AEStronglyMeasurable.sinc {α : Type u_1} {x✝ : MeasurableSpace α} {f : α} {μ : Measure α} (hf : AEStronglyMeasurable f μ) :
AEStronglyMeasurable (fun (x : α) => Real.sinc (f x)) μ