Skip to content

Commit

Permalink
feat(analysis/special_functions/trigonometric/basic): `tan_pi_div_two…
Browse files Browse the repository at this point in the history
…_sub` (#17024)

We have lemmas `sin_pi_div_two_sub` and `cos_pi_div_two_sub`.  Add corresponding `tan_pi_div_two_sub` lemmas (real and complex).
  • Loading branch information
jsm28 committed Oct 21, 2022
1 parent 86b9ee4 commit d94370d
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/analysis/special_functions/trigonometric/basic.lean
Expand Up @@ -761,6 +761,9 @@ tan_periodic.sub_eq x
lemma tan_pi_sub (x : ℝ) : tan (π - x) = -tan x :=
tan_neg x ▸ tan_periodic.sub_eq'

lemma tan_pi_div_two_sub (x : ℝ) : tan (π / 2 - x) = (tan x)⁻¹ :=
by rw [tan_eq_sin_div_cos, tan_eq_sin_div_cos, inv_div, sin_pi_div_two_sub, cos_pi_div_two_sub]

lemma tan_nat_mul_pi (n : ℕ) : tan (n * π) = 0 :=
tan_zero ▸ tan_periodic.nat_mul_eq n

Expand Down Expand Up @@ -990,6 +993,9 @@ tan_periodic.sub_eq x
lemma tan_pi_sub (x : ℂ) : tan (π - x) = -tan x :=
tan_neg x ▸ tan_periodic.sub_eq'

lemma tan_pi_div_two_sub (x : ℂ) : tan (π / 2 - x) = (tan x)⁻¹ :=
by rw [tan_eq_sin_div_cos, tan_eq_sin_div_cos, inv_div, sin_pi_div_two_sub, cos_pi_div_two_sub]

lemma tan_nat_mul_pi (n : ℕ) : tan (n * π) = 0 :=
tan_zero ▸ tan_periodic.nat_mul_eq n

Expand Down

0 comments on commit d94370d

Please sign in to comment.