Zulip Chat Archive

Stream: new members

Topic: simple power lemma


Matthew Honnor (May 16 2022 at 20:11):

Dear all, I was expecting simp to close the following simple lemma but it will not. I have then tried using cardinal.power_add and library search but these didn't work as well. Any help would be great.

import analysis.complex.basic

lemma equality_of_powers { u :  }{ z :  }{k :  }{ b :  }
  ( h : ¬(b < k) ) :
  (z - u) ^ (b - k) * (z - u) ^ k = (z - u) ^ b :=
  begin
    rw  cardinal.power_add,
  end

Thanks in advance.

Yaël Dillies (May 16 2022 at 21:05):

docs#pow_sub will lead you there

Yaël Dillies (May 16 2022 at 21:12):

Oof. I wrote this message 50min ago


Last updated: Dec 20 2023 at 11:08 UTC