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

Commit

Permalink
chore(measure_theory/{constructions/prod,measure/lebesgue}): split (#…
Browse files Browse the repository at this point in the history
…19039)

Reorganize some files in measure theory, with the goal of removing the dependence of Lebesgue measure on the Bochner integral.

`measure_theory/constructions/prod` is split into `prod/basic` and `prod/integral`; the former imports the Lebesgue integral but not the Bochner integral.

`measure_theory/measure/haar` is renamed `measure_theory/measure/haar/basic`.
`measure_theory/measure/haar_of_inner` is renamed `measure_theory/measure/haar/inner_product_space`.
`measure_theory/measure/haar_of_basis` is renamed `measure_theory/measure/haar/of_basis`.

`measure_theory/measure/lebesgue` is split into `measure_theory/measure/lebesgue/basic` and `measure_theory/measure/lebesgue/integral`, with the former not importing the Bochner integral.

`measure_theory/measure/complex_lebesgue` is renamed `measure_theory/measure/lebesgue/complex`.

`measure_theory/measure/haar_lebesgue` is split into `measure_theory/measure/lebesgue/eq_haar` and `measure_theory/measure/haar/normed_space`, with the former not importing the Bochner integral.

A few lemmas about Haar measure in normed spaces or fields are also moved from `measure_theory/group/measure` to the newly-created `measure_theory/measure/haar/normed_space`, since the former no longer imports `normed_space`.
  • Loading branch information
hrmacbeth committed May 18, 2023
1 parent aa66698 commit fd5edc4
Show file tree
Hide file tree
Showing 41 changed files with 738 additions and 600 deletions.
3 changes: 2 additions & 1 deletion archive/100-theorems-list/9_area_of_a_circle.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,10 @@ Copyright (c) 2021 James Arthur, Benjamin Davidson, Andrew Souther. All rights r
Released under Apache 2.0 license as described in the file LICENSE.
Authors: James Arthur, Benjamin Davidson, Andrew Souther
-/
import measure_theory.integral.fund_thm_calculus
import analysis.special_functions.sqrt
import analysis.special_functions.trigonometric.inverse_deriv
import measure_theory.integral.fund_thm_calculus
import measure_theory.measure.lebesgue.integral

/-!
# Freek № 9: The Area of a Circle
Expand Down
4 changes: 3 additions & 1 deletion counterexamples/phillips.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel
-/
import analysis.normed_space.hahn_banach.extension
import measure_theory.measure.lebesgue
import measure_theory.integral.set_integral
import measure_theory.measure.lebesgue.basic
import topology.continuous_function.bounded

/-!
# A counterexample on Pettis integrability
Expand Down
1 change: 1 addition & 0 deletions src/analysis/box_integral/integrability.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import analysis.box_integral.basic
import measure_theory.integral.set_integral
import measure_theory.measure.regular

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/box_integral/partition/measure.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import analysis.box_integral.partition.additive
import measure_theory.measure.lebesgue
import measure_theory.measure.lebesgue.basic

/-!
# Box-additive functions defined by measures
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/calculus/bump_function_findim.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Sébastien Gouëzel
import analysis.calculus.series
import analysis.convolution
import analysis.inner_product_space.euclidean_dist
import measure_theory.measure.haar_lebesgue
import measure_theory.measure.haar.normed_space
import data.set.pointwise.support

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/complex/cauchy_integral.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import measure_theory.measure.complex_lebesgue
import measure_theory.measure.lebesgue.complex
import measure_theory.integral.divergence_theorem
import measure_theory.integral.circle_integral
import analysis.calculus.dslope
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/convex/measure.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Yury Kudryashov
-/
import analysis.convex.topology
import analysis.normed_space.add_torsor_bases
import measure_theory.measure.haar_lebesgue
import measure_theory.measure.lebesgue.eq_haar

/-!
# Convex sets are null-measurable
Expand Down
7 changes: 4 additions & 3 deletions src/analysis/convolution.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,12 +3,13 @@ Copyright (c) 2022 Floris van Doorn. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn
-/
import analysis.calculus.bump_function_inner
import analysis.calculus.parametric_integral
import measure_theory.constructions.prod.integral
import measure_theory.function.locally_integrable
import measure_theory.group.integration
import measure_theory.group.prod
import measure_theory.function.locally_integrable
import analysis.calculus.bump_function_inner
import measure_theory.integral.interval_integral
import analysis.calculus.parametric_integral

/-!
# Convolution of functions
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/fourier/fourier_transform.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: David Loeffler

import analysis.complex.circle
import measure_theory.group.integration
import measure_theory.measure.haar_of_basis
import measure_theory.measure.haar.of_basis

/-!
# The Fourier transform
Expand Down
1 change: 1 addition & 0 deletions src/analysis/fourier/poisson_summation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,6 +7,7 @@ import analysis.fourier.add_circle
import analysis.fourier.fourier_transform
import analysis.p_series
import analysis.schwartz_space
import measure_theory.measure.lebesgue.integral

/-!
# Poisson's summation formula
Expand Down
8 changes: 5 additions & 3 deletions src/analysis/fourier/riemann_lebesgue_lemma.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,12 +4,14 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: David Loeffler
-/

import measure_theory.function.continuous_map_dense
import measure_theory.group.integration
import analysis.fourier.fourier_transform
import analysis.inner_product_space.dual
import topology.metric_space.emetric_paracompact
import analysis.inner_product_space.euclidean_dist
import measure_theory.function.continuous_map_dense
import measure_theory.group.integration
import measure_theory.integral.set_integral
import measure_theory.measure.haar.normed_space
import topology.metric_space.emetric_paracompact

/-!
# The Riemann-Lebesgue Lemma
Expand Down
5 changes: 3 additions & 2 deletions src/analysis/special_functions/improper_integrals.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,10 +3,11 @@ Copyright (c) 2023 David Loeffler. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: David Loeffler
-/
import measure_theory.integral.integral_eq_improper
import analysis.special_functions.integrals
import measure_theory.group.integration
import measure_theory.integral.exp_decay
import analysis.special_functions.integrals
import measure_theory.integral.integral_eq_improper
import measure_theory.measure.lebesgue.integral

/-!
# Evaluation of specific improper integrals
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/special_functions/japanese_bracket.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Moritz Doll. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Moritz Doll
-/
import measure_theory.measure.haar_lebesgue
import measure_theory.measure.lebesgue.eq_haar
import measure_theory.integral.layercake

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/measure_theory/constructions/pi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Floris van Doorn. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn
-/
import measure_theory.constructions.prod
import measure_theory.constructions.prod.basic
import measure_theory.group.measure
import topology.constructions

Expand Down
Loading

0 comments on commit fd5edc4

Please sign in to comment.