Skip to content

Commit 67b4128

Browse files
committed
chore: split MeasureTheory.Integral.Lebesgue.Basic (#23860)
* `.Add` contains some versions of the monotone convergence theorem, Fatou's lemma and addition and constant multiplication of integrals. * `.Sub` contains subtraction of integrals and more versions of monotone convergence (in particular those versions operating on _antitone_ sequences of functions). * `.Markov` contains Markov's inequality and lemmas that depend on it. * `.DominatedConvergence` contains the dominated convergence theorem. * Results on maps of measures have been moved to `.MeasurePreserving`, which already deals with measure-preserving _maps_. Since the scope has broadened, the file has been renamed to `.Map`.
1 parent 7daf90f commit 67b4128

File tree

17 files changed

+1170
-1037
lines changed

17 files changed

+1170
-1037
lines changed

Mathlib.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4175,10 +4175,15 @@ import Mathlib.MeasureTheory.Integral.IntervalIntegral.IntegrationByParts
41754175
import Mathlib.MeasureTheory.Integral.IntervalIntegral.Periodic
41764176
import Mathlib.MeasureTheory.Integral.Layercake
41774177
import Mathlib.MeasureTheory.Integral.Lebesgue
4178+
import Mathlib.MeasureTheory.Integral.Lebesgue.Add
41784179
import Mathlib.MeasureTheory.Integral.Lebesgue.Basic
41794180
import Mathlib.MeasureTheory.Integral.Lebesgue.Countable
4181+
import Mathlib.MeasureTheory.Integral.Lebesgue.DominatedConvergence
4182+
import Mathlib.MeasureTheory.Integral.Lebesgue.Map
4183+
import Mathlib.MeasureTheory.Integral.Lebesgue.Markov
41804184
import Mathlib.MeasureTheory.Integral.Lebesgue.MeasurePreserving
41814185
import Mathlib.MeasureTheory.Integral.Lebesgue.Norm
4186+
import Mathlib.MeasureTheory.Integral.Lebesgue.Sub
41824187
import Mathlib.MeasureTheory.Integral.LebesgueNormedSpace
41834188
import Mathlib.MeasureTheory.Integral.Marginal
41844189
import Mathlib.MeasureTheory.Integral.MeanInequalities

Mathlib/MeasureTheory/Function/AEEqFun.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Johannes Hölzl, Zhouhang Zhou
55
-/
66
import Mathlib.Dynamics.Ergodic.MeasurePreserving
77
import Mathlib.MeasureTheory.Function.StronglyMeasurable.AEStronglyMeasurable
8-
import Mathlib.MeasureTheory.Integral.Lebesgue.Basic
8+
import Mathlib.MeasureTheory.Integral.Lebesgue.Add
99
import Mathlib.Order.Filter.Germ.Basic
1010
import Mathlib.Topology.ContinuousMap.Algebra
1111

Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Zhouhang Zhou
55
-/
66
import Mathlib.MeasureTheory.Function.StronglyMeasurable.AEStronglyMeasurable
7+
import Mathlib.MeasureTheory.Integral.Lebesgue.DominatedConvergence
78
import Mathlib.MeasureTheory.Integral.Lebesgue.Norm
89
import Mathlib.MeasureTheory.Measure.WithDensity
910

Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -9,6 +9,7 @@ import Mathlib.MeasureTheory.Function.AEEqFun
99
import Mathlib.MeasureTheory.Function.LpSeminorm.Defs
1010
import Mathlib.MeasureTheory.Function.SpecialFunctions.Basic
1111
import Mathlib.MeasureTheory.Integral.Lebesgue.Countable
12+
import Mathlib.MeasureTheory.Integral.Lebesgue.Sub
1213

1314
/-!
1415
# Basic theorems about ℒp space

Mathlib/MeasureTheory/Function/StronglyMeasurable/ENNReal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Rémy Degenne
55
-/
66

77
import Mathlib.MeasureTheory.Function.StronglyMeasurable.AEStronglyMeasurable
8-
import Mathlib.MeasureTheory.Integral.Lebesgue.Basic
8+
import Mathlib.MeasureTheory.Integral.Lebesgue.Add
99

1010
/-!
1111
# Finitely strongly measurable functions with value in ENNReal

Mathlib/MeasureTheory/Group/FundamentalDomain.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Yury Kudryashov, Alex Kontorovich, Heather Macbeth
55
-/
66
import Mathlib.MeasureTheory.Group.Action
77
import Mathlib.MeasureTheory.Group.Pointwise
8-
import Mathlib.MeasureTheory.Integral.Lebesgue.MeasurePreserving
8+
import Mathlib.MeasureTheory.Integral.Lebesgue.Map
99
import Mathlib.MeasureTheory.Integral.SetIntegral
1010

1111
/-!

Mathlib/MeasureTheory/Integral/Indicator.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Kalle Kytölä
55
-/
66
import Mathlib.MeasureTheory.Constructions.BorelSpace.Metrizable
7-
import Mathlib.MeasureTheory.Integral.Lebesgue.Basic
7+
import Mathlib.MeasureTheory.Integral.Lebesgue.DominatedConvergence
88

99
/-!
1010
# Results about indicator functions, their integrals, and measures

Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean

Lines changed: 450 additions & 0 deletions
Large diffs are not rendered by default.

Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean

Lines changed: 0 additions & 993 deletions
Large diffs are not rendered by default.

Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,8 @@ Copyright (c) 2018 Mario Carneiro. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Mario Carneiro, Johannes Hölzl
55
-/
6-
import Mathlib.MeasureTheory.Integral.Lebesgue.Basic
6+
import Mathlib.MeasureTheory.Integral.Lebesgue.Map
7+
import Mathlib.MeasureTheory.Integral.Lebesgue.Markov
78
import Mathlib.MeasureTheory.Measure.Count
89

910
/-!

0 commit comments

Comments
 (0)