Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 9cf494e

Browse files
committed
fix(geometry/euclidean/oriented_angle): correct lemma name (#16821)
`oangle_eq_iff_angle_eq_of_sign_eq` should be called `angle_eq_iff_oangle_eq_of_sign_eq` to match the actual order of the `iff` arguments in the statement.
1 parent a87fad7 commit 9cf494e

File tree

1 file changed

+5
-5
lines changed

1 file changed

+5
-5
lines changed

src/geometry/euclidean/oriented_angle.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -994,7 +994,7 @@ end
994994

995995
/-- If the signs of two oriented angles between nonzero vectors are equal, the oriented angles are
996996
equal if and only if the unoriented angles are equal. -/
997-
lemma oangle_eq_iff_angle_eq_of_sign_eq {w x y z : V} (hw : w ≠ 0) (hx : x ≠ 0) (hy : y ≠ 0)
997+
lemma angle_eq_iff_oangle_eq_of_sign_eq {w x y z : V} (hw : w ≠ 0) (hx : x ≠ 0) (hy : y ≠ 0)
998998
(hz : z ≠ 0) (hs : (b.oangle w x).sign = (b.oangle y z).sign) :
999999
inner_product_geometry.angle w x = inner_product_geometry.angle y z ↔
10001000
b.oangle w x = b.oangle y z :=
@@ -1699,11 +1699,11 @@ lemma oangle_eq_of_angle_eq_of_sign_eq {w x y z : V}
16991699

17001700
/-- If the signs of two oriented angles between nonzero vectors are equal, the oriented angles are
17011701
equal if and only if the unoriented angles are equal. -/
1702-
lemma oangle_eq_iff_angle_eq_of_sign_eq {w x y z : V} (hw : w ≠ 0) (hx : x ≠ 0) (hy : y ≠ 0)
1702+
lemma angle_eq_iff_oangle_eq_of_sign_eq {w x y z : V} (hw : w ≠ 0) (hx : x ≠ 0) (hy : y ≠ 0)
17031703
(hz : z ≠ 0) (hs : (o.oangle w x).sign = (o.oangle y z).sign) :
17041704
inner_product_geometry.angle w x = inner_product_geometry.angle y z ↔
17051705
o.oangle w x = o.oangle y z :=
1706-
(ob).oangle_eq_iff_angle_eq_of_sign_eq hw hx hy hz hs
1706+
(ob).angle_eq_iff_oangle_eq_of_sign_eq hw hx hy hz hs
17071707

17081708
/-- The oriented angle between two nonzero vectors is zero if and only if the unoriented angle
17091709
is zero. -/
@@ -1932,10 +1932,10 @@ lemma oangle_eq_of_angle_eq_of_sign_eq {p₁ p₂ p₃ p₄ p₅ p₆ : P} (h :
19321932

19331933
/-- If the signs of two nondegenerate oriented angles between points are equal, the oriented
19341934
angles are equal if and only if the unoriented angles are equal. -/
1935-
lemma oangle_eq_iff_angle_eq_of_sign_eq {p₁ p₂ p₃ p₄ p₅ p₆ : P} (hp₁ : p₁ ≠ p₂) (hp₃ : p₃ ≠ p₂)
1935+
lemma angle_eq_iff_oangle_eq_of_sign_eq {p₁ p₂ p₃ p₄ p₅ p₆ : P} (hp₁ : p₁ ≠ p₂) (hp₃ : p₃ ≠ p₂)
19361936
(hp₄ : p₄ ≠ p₅) (hp₆ : p₆ ≠ p₅) (hs : (∡ p₁ p₂ p₃).sign = (∡ p₄ p₅ p₆).sign) :
19371937
∠ p₁ p₂ p₃ = ∠ p₄ p₅ p₆ ↔ ∡ p₁ p₂ p₃ = ∡ p₄ p₅ p₆ :=
1938-
(o).oangle_eq_iff_angle_eq_of_sign_eq (vsub_ne_zero.2 hp₁) (vsub_ne_zero.2 hp₃)
1938+
(o).angle_eq_iff_oangle_eq_of_sign_eq (vsub_ne_zero.2 hp₁) (vsub_ne_zero.2 hp₃)
19391939
(vsub_ne_zero.2 hp₄) (vsub_ne_zero.2 hp₆) hs
19401940

19411941
/-- The unoriented angle at `p` between two points not equal to `p` is zero if and only if the

0 commit comments

Comments
 (0)