Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit b4641ef

Browse files
committed
feat(l1_space): add measurability to integrable (#4170)
This PR defines `integrable` such that `integrable` implies `measurable`. The old version is called `has_finite_integral`. This allows us to drop *many* measurability conditions from lemmas that also require integrability. There are some lemmas that have extra measurability conditions, if it has `integrable` as conclusion without corresponding `measurable` hypothesis. There are many results that require an additional `[measurable_space E]` hypothesis, and some that require `[borel_space E]` or `[second_countable_space E]` (usually when using that addition is measurable).
1 parent 2ae199f commit b4641ef

File tree

6 files changed

+684
-611
lines changed

6 files changed

+684
-611
lines changed

src/measure_theory/bochner_integration.lean

Lines changed: 107 additions & 127 deletions
Large diffs are not rendered by default.

src/measure_theory/borel_space.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -741,7 +741,7 @@ namespace continuous_linear_map
741741

742742
variables [measurable_space α]
743743
variables {𝕜 : Type*} [normed_field 𝕜]
744-
variables {E : Type*} [normed_group E] [normed_space 𝕜 E] [measurable_space E] [borel_space E]
744+
variables {E : Type*} [normed_group E] [normed_space 𝕜 E] [measurable_space E] [opens_measurable_space E]
745745
variables {F : Type*} [normed_group F] [normed_space 𝕜 F] [measurable_space F] [borel_space F]
746746

747747
protected lemma measurable (L : E →L[𝕜] F) : measurable L :=

src/measure_theory/interval_integral.lean

Lines changed: 127 additions & 159 deletions
Large diffs are not rendered by default.

0 commit comments

Comments
 (0)