Zulip Chat Archive

Stream: Is there code for X?

Topic: Splitting a complex summable tsum into real and imaginary


Mark Gerads (Jul 12 2022 at 21:01):

Is imagPartsOfSumEqSumOfImagParts in the library somewhere? I would like proof so I can get closer to proving ruesRealToReal. If you have insight into the other 2 sorries, that would also be nice.

import all

open classical complex real topological_space

open_locale topological_space big_operators


-- rues is the Root of Unity Exponential Sum function
-- inspired by the relationship between exp and cosh
noncomputable
def rues (n:) (z:) :  :=
  tsum (λ (k:), z ^ (n*k) / (n*k).factorial)

lemma ruesSummable (n:) (z:) : summable (λ (k:), z ^ (n*k) / (n*k).factorial):=
begin
  rw [summable],
  sorry,
end

lemma imagPartsOfSumEqSumOfImagParts (f:) (hf:summable f):
      im (∑' (k : ), f k) = (∑' (k : ), im (f k)):=
begin
  sorry,
end

lemma ruesRealToReal (n:) (h:n>0) (x:) : (rues n x).im = 0 :=
begin
  rw [rues, imagPartsOfSumEqSumOfImagParts],
  {
    suffices h : ∑' (k : ), im (x ^ (n * k) / (n * k)!) = ∑' (k : ), 0,
    simp only [tsum_zero, h],
    congr' 1,
    ext1,
    sorry,
  },
  exact ruesSummable n x,
end

Ruben Van de Velde (Jul 12 2022 at 21:43):

Is it true? What if the real part diverges and the imaginary part converges to something nonzero?

Eric Wieser (Jul 12 2022 at 21:52):

docs#continuous_linear_map.map_tsum?

Eric Wieser (Jul 12 2022 at 21:53):

Combined with docs#complex.im_clm

Mark Gerads (Jul 12 2022 at 22:16):

@Ruben Van de Velde If that were the case, then the sum does not converge in ℂ. I have (f:ℕ→ℂ) (hf:summable f).

Eric Wieser (Jul 12 2022 at 22:18):

Then the above should work

Mark Gerads (Jul 12 2022 at 22:19):

I'm trying.

Mark Gerads (Jul 12 2022 at 22:26):

I got it.

lemma imagPartsOfSumEqSumOfImagParts (f:) (hf:summable f):
      im (∑' (k : ), f k) = (∑' (k : ), im (f k)):=
begin
  let h:= continuous_linear_map.map_tsum complex.im_clm hf,
  continuity,
end

Eric Wieser (Jul 12 2022 at 22:38):

I suspect you can remove everything from the begin to the := (inclusive), and everything after the first cons

Eric Wieser (Jul 12 2022 at 22:39):

You might want to look at #naming too; while it wouldn't have helped you here, following the rules for naming can often lead to finding an existing lemma.

Eric Wieser (Jul 12 2022 at 22:40):

That would be called complex.im_tsum I think


Last updated: Dec 20 2023 at 11:08 UTC