Skip to content

Commit

Permalink
feat(analysis/special_functions/trigonometric/angle): more 2π = 0 lem…
Browse files Browse the repository at this point in the history
…mas (#11482)

Add some more lemmas useful for manipulation of `real.angle` expressions.
  • Loading branch information
jsm28 committed Jan 16, 2022
1 parent ed57bdd commit f4b93c8
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/analysis/special_functions/trigonometric/angle.lean
Expand Up @@ -63,6 +63,15 @@ begin
simp [two_mul, sub_eq_add_neg]
end

lemma sub_coe_pi_eq_add_coe_pi (θ : angle) : θ - π = θ + π :=
by rw [sub_eq_add_neg, neg_coe_pi]

@[simp] lemma two_nsmul_coe_pi : (2 : ℕ) • (π : angle) = 0 :=
by simp [←coe_nat_mul_eq_nsmul]

@[simp] lemma two_zsmul_coe_pi : (2 : ℤ) • (π : angle) = 0 :=
by simp [←coe_int_mul_eq_zsmul]

theorem cos_eq_iff_eq_or_eq_neg {θ ψ : ℝ} : cos θ = cos ψ ↔ (θ : angle) = ψ ∨ (θ : angle) = -ψ :=
begin
split,
Expand Down

0 comments on commit f4b93c8

Please sign in to comment.