Zulip Chat Archive
Stream: Is there code for X?
Topic: c ^ n tends to 0 in complexes
Bhavik Mehta (Jan 29 2025 at 19:07):
Do we have this?
import Mathlib.Analysis.Complex.Basic
open Filter Topology
example {c : โ} (hc : โcโ < 1) : Tendsto (c ^ ยท) atTop (๐ 0) := by
sorry
I presume it also works for normed fields or something, but I'd be happy with any reasonable version of the above - loogle and exact? and leansearch are all failing to find it for me
Bhavik Mehta (Jan 29 2025 at 19:11):
Ah, here we go:
example {E : Type*} [NormedDivisionRing E]
{c : E} (hc : โcโ < 1) : Tendsto (c ^ ยท) atTop (๐ 0) := by
rw [tendsto_zero_iff_norm_tendsto_zero]
simpa
I'm still slightly surprised this wasn't in mathlib already, especially since we have docs#tendsto_pow_atTop_nhds_zero_iff
Etienne Marion (Jan 29 2025 at 19:13):
It's docs#tendsto_pow_atTop_nhds_zero_of_norm_lt_one I think?
Etienne Marion (Jan 29 2025 at 19:13):
(deleted)
Etienne Marion (Jan 29 2025 at 19:14):
@loogle โ_โ < 1, Filter.Tendsto
loogle (Jan 29 2025 at 19:14):
:search: tendsto_pow_atTop_nhds_zero_of_norm_lt_one, CStarAlgebra.tendsto_mul_right_of_forall_nonneg_tendsto, and 1 more
Bhavik Mehta (Jan 29 2025 at 19:14):
Ah, so it is. Thank you!
Bhavik Mehta (Jan 29 2025 at 19:15):
I searched nhds, Filter.Tendsto, Filter.atTop, "pow"
and got a ton of unhelpful things
Last updated: May 02 2025 at 03:31 UTC