Skip to content

Commit 8372ba7

Browse files
committed
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces (#27378)
This PR continues the work from #25578. Original PR: #25578 - [x] depends on: #31395
1 parent 63a90fe commit 8372ba7

File tree

2 files changed

+185
-254
lines changed

2 files changed

+185
-254
lines changed

Mathlib/Geometry/Euclidean/Circumcenter.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -84,7 +84,7 @@ theorem existsUnique_dist_eq_of_insert {s : AffineSubspace ℝ P}
8484
· rw [hp₁, hpo,
8585
dist_sq_smul_orthogonal_vadd_smul_orthogonal_vadd (orthogonalProjection_mem p) hcc _ _
8686
(vsub_orthogonalProjection_mem_direction_orthogonal s p),
87-
← dist_eq_norm_vsub V p, dist_comm _ cc]
87+
Real.norm_eq_abs, abs_mul_abs_self, ← dist_eq_norm_vsub V p, dist_comm _ cc]
8888
simp only [ycc₂]
8989
field
9090
· rw [dist_sq_eq_dist_orthogonalProjection_sq_add_dist_orthogonalProjection_sq _ (hps hp₁),
@@ -122,7 +122,7 @@ theorem existsUnique_dist_eq_of_insert {s : AffineSubspace ℝ P}
122122
rw [hpo, hcc₃'', hcr₃val, ← mul_self_inj_of_nonneg dist_nonneg (Real.sqrt_nonneg _),
123123
dist_sq_smul_orthogonal_vadd_smul_orthogonal_vadd (orthogonalProjection_mem p) hcc₃' _ _
124124
(vsub_orthogonalProjection_mem_direction_orthogonal s p),
125-
dist_comm, ← dist_eq_norm_vsub V p,
125+
Real.norm_eq_abs, abs_mul_abs_self, dist_comm, ← dist_eq_norm_vsub V p,
126126
Real.mul_self_sqrt (add_nonneg (mul_self_nonneg _) (mul_self_nonneg _))] at hcr₃
127127
change x * x + _ * (y * y) = _ at hcr₃
128128
rw [show
@@ -605,7 +605,7 @@ theorem reflection_circumcenter_eq_affineCombination_of_pointsWithCircumcenter {
605605
↑((s.face hc).orthogonalProjectionSpan s.circumcenter) := by
606606
apply eq_orthogonalProjection_of_eq_subspace
607607
simp [W]
608-
rw [EuclideanGeometry.reflection_apply, h_faces, s.orthogonalProjection_circumcenter hc,
608+
rw [reflection_apply', h_faces, s.orthogonalProjection_circumcenter hc,
609609
circumcenter_eq_centroid, s.face_centroid_eq_centroid hc,
610610
centroid_eq_affineCombination_of_pointsWithCircumcenter,
611611
circumcenter_eq_affineCombination_of_pointsWithCircumcenter, ← @vsub_eq_zero_iff_eq V,

0 commit comments

Comments
 (0)