Skip to content

Commit

Permalink
feat(l1_space): add measurability to integrable (#4170)
Browse files Browse the repository at this point in the history
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).
  • Loading branch information
fpvandoorn committed Sep 22, 2020
1 parent 2ae199f commit b4641ef
Show file tree
Hide file tree
Showing 6 changed files with 684 additions and 611 deletions.
234 changes: 107 additions & 127 deletions src/measure_theory/bochner_integration.lean

Large diffs are not rendered by default.

2 changes: 1 addition & 1 deletion src/measure_theory/borel_space.lean
Expand Up @@ -741,7 +741,7 @@ namespace continuous_linear_map

variables [measurable_space α]
variables {𝕜 : Type*} [normed_field 𝕜]
variables {E : Type*} [normed_group E] [normed_space 𝕜 E] [measurable_space E] [borel_space E]
variables {E : Type*} [normed_group E] [normed_space 𝕜 E] [measurable_space E] [opens_measurable_space E]
variables {F : Type*} [normed_group F] [normed_space 𝕜 F] [measurable_space F] [borel_space F]

protected lemma measurable (L : E →L[𝕜] F) : measurable L :=
Expand Down
286 changes: 127 additions & 159 deletions src/measure_theory/interval_integral.lean

Large diffs are not rendered by default.

0 comments on commit b4641ef

Please sign in to comment.