Zulip Chat Archive

Stream: Is there code for X?

Topic: Uncountable sum diverges


Praneeth Kolichala (Feb 17 2022 at 04:23):

For example, the uncountable sum of real numbers diverges. I have a proof, but it is long and might duplicate lemmas that already exist, since I'm still getting familiar with this part of mathlib:

Code

Some of these lemmas seem like they should be in the library already, but I couldn't find them using library_search.

Also, my feeling is that some of the typeclass constraints are unnecessary. I tried to essentially port my proof from the one in real numbers, but this might not be the most efficient way to do it in general.

Yury G. Kudryashov (Feb 17 2022 at 06:33):

Here is an idea of a simpler proof. The main lemma is

open set filter
lemma filter.tendsto.countable_set_of_ne {α X : Type*} [topological_space X] [t1_space X]
  {f : α  X} {b : X} (hf : tendsto f cofinite (𝓝 b)) [is_countably_generated (𝓝 b)] :
  countable {a | f a  b}

Yury G. Kudryashov (Feb 17 2022 at 06:34):

Your statement follows from this lemma and docs#summable.tendsto_cofinite_zero

Yury G. Kudryashov (Feb 17 2022 at 06:41):

To prove this lemma, choose a specific countable basis of nhds of b (e.g., using docs#filter.exists_antitone_basis). The preimage of each neighborhood is cofinite, hence the complement of the preimage of their intersection is countable. Due to docs#bInter_basis_nhds, this intersection is {b} and you get the desired statement.


Last updated: Dec 20 2023 at 11:08 UTC