Skip to content

Commit

Permalink
docs(data/complex/exponential): docstring for de Moivre (#4242)
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Sep 24, 2020
1 parent 02ca5e2 commit 5eedf32
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions src/data/complex/exponential.lean
Original file line number Diff line number Diff line change
Expand Up @@ -741,6 +741,7 @@ by rw [exp_add, exp_mul_I]
lemma exp_eq_exp_re_mul_sin_add_cos : exp x = exp x.re * (cos x.im + sin x.im * I) :=
by rw [← exp_add_mul_I, re_add_im]

/-- De Moivre's formula -/
theorem cos_add_sin_mul_I_pow (n : ℕ) (z : ℂ) : (cos z + sin z * I) ^ n = cos (↑n * z) + sin (↑n * z) * I :=
begin
rw [← exp_mul_I, ← exp_mul_I],
Expand Down

0 comments on commit 5eedf32

Please sign in to comment.