Skip to content

Commit

Permalink
feat: show that the Riemann integral is equal to the Bochner integral…
Browse files Browse the repository at this point in the history
… for continuous functions (#10144)
  • Loading branch information
xroblot committed Feb 11, 2024
1 parent 7d2b303 commit 877599c
Showing 1 changed file with 14 additions and 1 deletion.
15 changes: 14 additions & 1 deletion Mathlib/Analysis/BoxIntegral/Integrability.lean
Expand Up @@ -5,7 +5,6 @@ Authors: Yury Kudryashov
-/
import Mathlib.Analysis.BoxIntegral.Basic
import Mathlib.MeasureTheory.Integral.SetIntegral
import Mathlib.MeasureTheory.Measure.Regular

#align_import analysis.box_integral.integrability from "leanprover-community/mathlib"@"fd5edc43dc4f10b85abfe544b88f82cf13c5f844"

Expand All @@ -16,6 +15,8 @@ In this file we prove that any Bochner integrable function is McShane integrable
Henstock and `GP` integrable) with the same integral. The proof is based on
[Russel A. Gordon, *The integrals of Lebesgue, Denjoy, Perron, and Henstock*][Gordon55].
We deduce that the same is true for the Riemann integral for continuous functions.
## Tags
integral, McShane integral, Bochner integral
Expand Down Expand Up @@ -302,4 +303,16 @@ theorem IntegrableOn.hasBoxIntegral [CompleteSpace E] {f : (ι → ℝ) → E} {
exact hfg_mono x (hNx (π.tag J))
#align measure_theory.integrable_on.has_box_integral MeasureTheory.IntegrableOn.hasBoxIntegral

/-- If `f : ℝⁿ → E` is continuous on a rectangular box `I`, then it is Box integrable on `I`
w.r.t. a locally finite measure `μ` with the same integral. -/
theorem ContinuousOn.hasBoxIntegral [CompleteSpace E] {f : (ι → ℝ) → E} (μ : Measure (ι → ℝ))
[IsLocallyFiniteMeasure μ] {I : Box ι} (hc : ContinuousOn f (Box.Icc I))
(l : IntegrationParams) :
HasIntegral.{u, v, v} I l f μ.toBoxAdditive.toSMul (∫ x in I, f x ∂μ) := by
obtain ⟨y, hy⟩ := BoxIntegral.integrable_of_continuousOn l hc μ
convert hy
have : IntegrableOn f I μ :=
IntegrableOn.mono_set (hc.integrableOn_compact I.isCompact_Icc) Box.coe_subset_Icc
exact HasIntegral.unique (IntegrableOn.hasBoxIntegral this ⊥ rfl) (HasIntegral.mono hy bot_le)

end MeasureTheory

0 comments on commit 877599c

Please sign in to comment.