Zulip Chat Archive
Stream: Is there code for X?
Topic: exponential function to a natural power
Mark Andrew Gerads (Sep 23 2022 at 03:46):
This should definitely be in mathlib (I need it), but library_search!
is not finding it.
lemma expPowEqExpMul (z:ℂ) (n : ℕ) : exp (z) ^ n = exp (z * n) :=
begin
induction n with n ih,
simp only [pow_zero, nat.cast_zero, mul_zero, complex.exp_zero],
rw [pow_succ],
rw (show (n.succ:ℂ) = n + 1, by {simp} ),
rw (show (z * (n + 1)) = z + z * n, by {ring} ),
rw complex.exp_add z _,
congr,
exact ih,
end
Moritz Doll (Sep 23 2022 at 03:51):
Moritz Doll (Sep 23 2022 at 03:52):
modulo symmetry and commuting factors
Eric Wieser (Sep 23 2022 at 07:00):
Last updated: Dec 20 2023 at 11:08 UTC