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

Commit 286e6ba

Browse files
committed
feat(geometry/euclidean/angle/oriented/basic): rotation and negation lemmas (#17277)
Add more lemmas about the interaction of rotation and negation.
1 parent 79f700b commit 286e6ba

File tree

1 file changed

+17
-0
lines changed

1 file changed

+17
-0
lines changed

src/geometry/euclidean/angle/oriented/basic.lean

Lines changed: 17 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -631,6 +631,10 @@ begin
631631
simp [rotation]
632632
end
633633

634+
/-- Rotation by π is negation. -/
635+
lemma rotation_pi_apply (x : V) : o.rotation π x = -x :=
636+
by simp
637+
634638
/-- Rotation by π / 2 is the "right-angle-rotation" map `J`. -/
635639
lemma rotation_pi_div_two : o.rotation (π / 2 : ℝ) = J :=
636640
begin
@@ -664,6 +668,19 @@ begin
664668
ring,
665669
end
666670

671+
/-- Negating a rotation is equivalent to rotation by π plus the angle. -/
672+
lemma neg_rotation (θ : real.angle) (x : V) : -o.rotation θ x = o.rotation (π + θ) x :=
673+
by rw [←o.rotation_pi_apply, rotation_rotation]
674+
675+
/-- Negating a rotation by -π / 2 is equivalent to rotation by π / 2. -/
676+
@[simp] lemma neg_rotation_neg_pi_div_two (x : V) :
677+
-o.rotation (-π / 2 : ℝ) x = o.rotation (π / 2 : ℝ) x :=
678+
by rw [neg_rotation, ←real.angle.coe_add, neg_div, ←sub_eq_add_neg, sub_half]
679+
680+
/-- Negating a rotation by π / 2 is equivalent to rotation by -π / 2. -/
681+
lemma neg_rotation_pi_div_two (x : V) : -o.rotation (π / 2 : ℝ) x = o.rotation (-π / 2 : ℝ) x :=
682+
neg_eq_iff_neg_eq.1 $ o.neg_rotation_neg_pi_div_two _
683+
667684
/-- Rotating the first of two vectors by `θ` scales their Kahler form by `cos (-θ) + sin (-θ) * I`.
668685
-/
669686
lemma kahler_rotation_left' (x y : V) (θ : real.angle) :

0 commit comments

Comments
 (0)