Zulip Chat Archive
Stream: Is there code for X?
Topic: coe summable
Chris Birkbeck (Jan 25 2023 at 19:06):
Do we have the following:
lemma coe_summable { α : Type*} (f : α → ℝ) : summable ((coe : ℝ → ℂ) ∘ f) ↔ summable f :=
It seems like it must be somewhere but I can't find it.
Eric Wieser (Jan 25 2023 at 19:16):
Does it fall out as a special case of something like docs#summable.mapL?
Eric Wieser (Jan 25 2023 at 19:18):
Aha, docs#summable.map_iff_of_left_inverse, which I added a little while back
Kyle Miller (Jan 25 2023 at 19:29):
That works:
import topology.algebra.infinite_sum
import analysis.complex.basic
lemma coe_summable { α : Type*} (f : α → ℝ) :
summable ((coe : ℝ → ℂ) ∘ f) ↔ summable f :=
begin
apply summable.map_iff_of_left_inverse complex.of_real complex.re_add_group_hom,
exact complex.continuous_of_real,
exact complex.continuous_re,
intro, refl,
end
Chris Birkbeck (Jan 25 2023 at 19:50):
Oh great thanks!
Chris Birkbeck (Jan 25 2023 at 19:52):
I swear I looked at that file for ages, but couldn't see this!
Eric Wieser (Feb 03 2023 at 17:54):
I've PR'd this in #18376 as complex.summable_of_real
Last updated: Dec 20 2023 at 11:08 UTC