Skip to content

Commit

Permalink
fix(geometry/euclidean/angle/unoriented/right_angle): lemma naming co…
Browse files Browse the repository at this point in the history
…nsistency (#17273)

Adjust the name of one lemma for `tan` to be consistent with the names of corresponding `sin` and `cos` lemmas.
  • Loading branch information
jsm28 committed Nov 5, 2022
1 parent ef5d936 commit c59f261
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/geometry/euclidean/angle/unoriented/right_angle.lean
Expand Up @@ -486,7 +486,7 @@ begin
end

/-- The tangent of an angle in a right-angled triangle as a ratio of sides. -/
lemma tan_angle_eq_of_angle_eq_pi_div_two {p₁ p₂ p₃ : P} (h : ∠ p₁ p₂ p₃ = π / 2) :
lemma tan_angle_of_angle_eq_pi_div_two {p₁ p₂ p₃ : P} (h : ∠ p₁ p₂ p₃ = π / 2) :
real.tan (∠ p₂ p₃ p₁) = dist p₁ p₂ / dist p₃ p₂ :=
begin
rw [angle, ←inner_eq_zero_iff_angle_eq_pi_div_two, real_inner_comm, ←neg_eq_zero,
Expand Down

0 comments on commit c59f261

Please sign in to comment.