Zulip Chat Archive
Stream: Is there code for X?
Topic: Convergence of a complex series bounded by a geometric sum
Mark Gerads (Oct 04 2021 at 11:07):
image.png
I [need something like this] and[ want to know if someone already did this].
Ruben Van de Velde (Oct 04 2021 at 11:12):
I'd start looking at https://leanprover-community.github.io/mathlib_docs/analysis/specific_limits.html
Mark Gerads (Oct 04 2021 at 11:57):
The entire file (_target/deps/mathlib/src/analysis/specific_limits.lean) does not have a single 'ℂ' in it.
Yaël Dillies (Oct 04 2021 at 11:58):
That's because it might not be the correct level of generality.
Yaël Dillies (Oct 04 2021 at 11:59):
What about docs#summable_geometric_of_norm_lt_1? That sounds close.
Yury G. Kudryashov (Oct 04 2021 at 12:08):
This plus something like docs#summable_of_norm_bounded
Mark Gerads (Oct 04 2021 at 12:37):
Yaël Dillies said:
What about docs#summable_geometric_of_norm_lt_1? That sounds close.
If I were to generalize, I need something along the lines of :
lemma summable_bounded_by_geometric_of_norm_lt_1
{f : ℕ → K} (h0 : ∥ξ∥ < 1) (h1 : ∀ (k : ℕ), ∥ξ ^ k∥ ≥ ∥f k∥)
: summable f :=
Yury G. Kudryashov said:
This plus something like docs#summable_of_norm_bounded
summable_of_norm_bounded is indeed the missing piece I needed.
Last updated: Dec 20 2023 at 11:08 UTC