Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2023-02-15 17:45 32253a1a

View on Github →

split(topology/algebra/infinite_sum): Split into four files (#18414) 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.

Estimated changes

deleted theorem commute.tsum_left
deleted theorem commute.tsum_right
deleted theorem finite_of_summable_const
modified theorem has_sum.const_smul
deleted theorem has_sum.div_const
deleted theorem has_sum.mul
deleted theorem has_sum.mul_eq
deleted theorem has_sum.mul_left
deleted theorem has_sum.mul_right
deleted theorem has_sum.nonneg
deleted theorem has_sum.nonpos
deleted theorem has_sum.smul_const
deleted theorem has_sum_div_const_iff
deleted theorem has_sum_le
deleted theorem has_sum_le_inj
deleted theorem has_sum_le_of_sum_le
deleted theorem has_sum_lt
deleted theorem has_sum_mono
deleted theorem has_sum_mul_left_iff
deleted theorem has_sum_mul_right_iff
deleted theorem has_sum_of_is_lub
deleted theorem has_sum_strict_mono
deleted theorem has_sum_zero_iff
deleted theorem is_lub_has_sum'
deleted theorem is_lub_has_sum
deleted theorem le_has_sum'
deleted theorem le_has_sum
deleted theorem le_has_sum_of_le_sum
deleted theorem le_tsum'
deleted theorem le_tsum
deleted theorem sum_le_has_sum
deleted theorem sum_le_tsum
modified theorem summable.const_smul
deleted theorem summable.div_const
deleted theorem summable.mul_left
deleted theorem summable.mul_right
deleted theorem summable.smul_const
deleted theorem summable.tsum_mul_left
deleted theorem summable.tsum_mul_right
deleted theorem summable_abs_iff
deleted theorem summable_div_const_iff
deleted theorem summable_mul_left_iff
deleted theorem summable_mul_right_iff
modified theorem summable_op
modified theorem summable_star_iff'
modified theorem tsum_const_smul
deleted theorem tsum_div_const
deleted theorem tsum_eq_zero_iff
deleted theorem tsum_le_of_sum_le'
deleted theorem tsum_le_of_sum_le
deleted theorem tsum_le_of_sum_range_le
deleted theorem tsum_le_tsum
deleted theorem tsum_le_tsum_of_inj
deleted theorem tsum_lt_tsum
deleted theorem tsum_mono
deleted theorem tsum_mul_left
deleted theorem tsum_mul_right
deleted theorem tsum_mul_tsum
deleted theorem tsum_ne_zero_iff
deleted theorem tsum_nonneg
deleted theorem tsum_nonpos
deleted theorem tsum_pos
deleted theorem tsum_smul_const
deleted theorem tsum_strict_mono
added theorem has_sum.nonneg
added theorem has_sum.nonpos
added theorem has_sum_le
added theorem has_sum_le_inj
added theorem has_sum_le_of_sum_le
added theorem has_sum_lt
added theorem has_sum_mono
added theorem has_sum_of_is_lub
added theorem has_sum_strict_mono
added theorem has_sum_zero_iff
added theorem is_lub_has_sum'
added theorem is_lub_has_sum
added theorem le_has_sum'
added theorem le_has_sum
added theorem le_has_sum_of_le_sum
added theorem le_tsum'
added theorem le_tsum
added theorem sum_le_has_sum
added theorem sum_le_tsum
added theorem summable_abs_iff
added theorem tsum_eq_zero_iff
added theorem tsum_le_of_sum_le'
added theorem tsum_le_of_sum_le
added theorem tsum_le_tsum
added theorem tsum_le_tsum_of_inj
added theorem tsum_lt_tsum
added theorem tsum_mono
added theorem tsum_ne_zero_iff
added theorem tsum_nonneg
added theorem tsum_nonpos
added theorem tsum_pos
added theorem tsum_strict_mono