Skip to content

Commit

Permalink
feat(data/complex/exponential): add real.cos_abs (#13177)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Apr 5, 2022
1 parent b011b0e commit cf131e1
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/data/complex/exponential.lean
Expand Up @@ -945,6 +945,9 @@ by rw [← of_real_inj]; simp [sin, sin_add]
@[simp] lemma cos_neg : cos (-x) = cos x :=
by simp [cos, exp_neg]

@[simp] lemma cos_abs : cos (|x|) = cos x :=
by cases le_total x 0; simp only [*, _root_.abs_of_nonneg, abs_of_nonpos, cos_neg]

lemma cos_add : cos (x + y) = cos x * cos y - sin x * sin y :=
by rw ← of_real_inj; simp [cos, cos_add]

Expand Down

0 comments on commit cf131e1

Please sign in to comment.