Zulip Chat Archive

Stream: new members

Topic: Non-necessarily unconditionally convergent series


Gihan Marasingha (Dec 26 2020 at 12:48):

Really basic question, but where are the 'algebra of limits' theorems in mathlib for series in, say, a normed vector space? For instance, where is the theorem that the series of the sum of two convergent series is convergent?

Johan Commelin (Dec 26 2020 at 13:38):

@Gihan Marasingha

src/topology/algebra/monoid.lean
68:lemma tendsto_mul {a b : M} : tendsto (λp:M×M, p.fst * p.snd) (𝓝 (a, b)) (𝓝 (a * b)) :=

Patrick Massot (Dec 26 2020 at 14:02):

We have nothing specific for series.

Patrick Massot (Dec 26 2020 at 14:03):

Of course this doesn't prevent you from getting that the sum of two convergent series is convergent, but this will explicitly be a lemma about their partial sums.

Patrick Massot (Dec 26 2020 at 14:03):

The main issue is we never decided whether series should be indexed by natural numbers of something more general.

Frédéric Dupuis (Dec 26 2020 at 14:48):

If you're OK with unconditional convergence only, summable.add and friends in topology/algebra/infinite_sum might suit your purpose.

Frédéric Dupuis (Dec 26 2020 at 14:49):

Oh, I should have read the title of that post before replying, shouldn't I?


Last updated: Dec 20 2023 at 11:08 UTC