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

Commit

Permalink
split(topology/algebra/infinite_sum): Split into four files (#18414)
Browse files Browse the repository at this point in the history
Over the past five years, `topology.algebra.infinite_sum` has grown pretty big. This PR splits off a third of it to three new files. Precisely, split `topology.algebra.infinite_sum` into:
* `topology.algebra.infinite_sum.basic`: Definitions and theory in monoids. All this will be multiplicativised in #18405.
* `topology.algebra.infinite_sum.ring`: Interaction of infinite sums and (scalar) multiplication. This mostly cannot be multiplicativised.
* `topology.algebra.infinite_sum.order`: Interaction of infinite sums and order. Most of this will be multiplicativised in #18405.

Incidentally, this brings down some files' imports by quite a lot.

Also move the `star` and `mul_opposite` material to the end of the file to facilitate multiplicativisation in #18405.

Johannes wrote some of all these files, except `topology.algebra.infinite_sum.real` whose first lemma I could trace back as coming from #753, with the others coming from #1739.
  • Loading branch information
YaelDillies committed Feb 15, 2023
1 parent f1e061e commit 32253a1
Show file tree
Hide file tree
Showing 16 changed files with 691 additions and 658 deletions.
2 changes: 1 addition & 1 deletion src/analysis/analytic/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Sébastien Gouëzel, Yury Kudryashov
import analysis.calculus.formal_multilinear_series
import analysis.specific_limits.normed
import logic.equiv.fin
import topology.algebra.module.infinite_sum
import topology.algebra.infinite_sum.module

/-!
# Analytic functions
Expand Down
1 change: 0 additions & 1 deletion src/analysis/analytic/isolated_zeros.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,6 @@ import analysis.analytic.basic
import analysis.calculus.dslope
import analysis.calculus.fderiv_analytic
import analysis.calculus.formal_multilinear_series
import topology.algebra.infinite_sum
import analysis.analytic.uniqueness

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/complex/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Sébastien Gouëzel
import data.complex.module
import data.complex.exponential
import data.is_R_or_C.basic
import topology.algebra.module.infinite_sum
import topology.algebra.infinite_sum.module
import topology.instances.real_vector_space

/-!
Expand Down
2 changes: 1 addition & 1 deletion src/analysis/normed_space/finite_dimension.lean
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@ import analysis.normed_space.operator_norm
import analysis.normed_space.riesz_lemma
import linear_algebra.matrix.to_lin
import topology.algebra.module.finite_dimension
import topology.algebra.module.infinite_sum
import topology.algebra.infinite_sum.module
import topology.instances.matrix

/-!
Expand Down
1 change: 0 additions & 1 deletion src/measure_theory/measure/outer_measure.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,6 @@ import analysis.specific_limits.basic
import measure_theory.pi_system
import data.countable.basic
import data.fin.vec_notation
import topology.algebra.infinite_sum

/-!
# Outer Measures
Expand Down
2 changes: 1 addition & 1 deletion src/number_theory/l_series.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Aaron Anderson
import analysis.normed_space.finite_dimension
import analysis.p_series
import number_theory.arithmetic_function
import topology.algebra.infinite_sum
import topology.algebra.infinite_sum.basic

/-!
# L-series
Expand Down
Loading

0 comments on commit 32253a1

Please sign in to comment.