Zulip Chat Archive

Stream: new members

Topic: Working with tsum


Matthew Honnor (May 12 2022 at 19:09):

Dear all, I am struggling to work with infinite sums. I have included the code of my specific problem below but I am also interested in how to show that two tsums are equal.

I don't know how to make progress on the proof of the simple lemma below.

import analysis.complex.basic

def analytic_sum_term ( a :    ) ( z :  ) ( u :  ) :    :=
  λ k , a k *( z - u )^k

noncomputable def analytic_sum ( u :  ) ( a :    ) :    :=
  λ z, ∑' k : , analytic_sum_term a z u k

lemma analytic_sum_leading_term { u :  }{ a :    }
  ( h : analytic_sum u a u = 0 ) :
  a 0 = 0 :=
  begin
    rw analytic_sum at h,
    norm_num at h,
    rw analytic_sum_term at h,
    simp at h,

  end

Thanks in advance for any help.


Last updated: Dec 20 2023 at 11:08 UTC