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

Commit b0b5cd4

Browse files
committed
feat(geometry/euclidean): circumradius simp lemmas (#3834)
Mark `dist_circumcenter_eq_circumradius` as a `simp` lemma. Also add a variant of that lemma where the distance is the other way round so `simp` can work with both forms.
1 parent 43337f7 commit b0b5cd4

File tree

1 file changed

+11
-1
lines changed

1 file changed

+11
-1
lines changed

src/geometry/euclidean.lean

Lines changed: 11 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1185,10 +1185,20 @@ s.circumcenter_circumradius_unique_dist_eq.1.1
11851185

11861186
/-- All points have distance from the circumcenter equal to the
11871187
circumradius. -/
1188-
lemma dist_circumcenter_eq_circumradius {n : ℕ} (s : simplex ℝ P n) :
1188+
@[simp] lemma dist_circumcenter_eq_circumradius {n : ℕ} (s : simplex ℝ P n) :
11891189
∀ i, dist (s.points i) s.circumcenter = s.circumradius :=
11901190
s.circumcenter_circumradius_unique_dist_eq.1.2
11911191

1192+
/-- All points have distance to the circumcenter equal to the
1193+
circumradius. -/
1194+
@[simp] lemma dist_circumcenter_eq_circumradius' {n : ℕ} (s : simplex ℝ P n) :
1195+
∀ i, dist s.circumcenter (s.points i) = s.circumradius :=
1196+
begin
1197+
intro i,
1198+
rw dist_comm,
1199+
exact dist_circumcenter_eq_circumradius _ _
1200+
end
1201+
11921202
/-- Given a point in the affine span from which all the points are
11931203
equidistant, that point is the circumcenter. -/
11941204
lemma eq_circumcenter_of_dist_eq {n : ℕ} (s : simplex ℝ P n) {p : P}

0 commit comments

Comments
 (0)