Skip to content

Commit

Permalink
feat(analysis/special_functions/trigonometric): Added lemma cos_ne_ze…
Browse files Browse the repository at this point in the history
…ro_iff (#3743)

I added the theorem `cos_ne_zero_iff`, a corollary to the preexisting theorem `cos_eq_zero_iff`
<!-- put comments you want to keep out of the PR commit here -->
  • Loading branch information
benjamindavidson committed Aug 13, 2020
1 parent ced7469 commit b1e56a2
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/analysis/special_functions/trigonometric.lean
Expand Up @@ -714,6 +714,9 @@ begin
sub_add_eq_sub_sub_swap, sub_self, zero_sub, neg_mul_eq_neg_mul, int.cast_neg] }
end

theorem cos_ne_zero_iff {θ : ℝ} : cos θ ≠ 0 ↔ ∀ k : ℤ, θ ≠ (2 * k + 1) * pi / 2 :=
by rw [← not_exists, not_iff_not, cos_eq_zero_iff]

lemma cos_eq_one_iff_of_lt_of_lt {x : ℝ} (hx₁ : -(2 * π) < x) (hx₂ : x < 2 * π) : cos x = 1 ↔ x = 0 :=
⟨λ h, let ⟨n, hn⟩ := (cos_eq_one_iff x).1 h in
begin
Expand Down

0 comments on commit b1e56a2

Please sign in to comment.