Skip to content

Commit

Permalink
feat(geometry/euclidean/basic): `dist_center_eq_dist_center_of_mem_sp…
Browse files Browse the repository at this point in the history
…here'` (#17390)

Add a variant of `dist_center_eq_dist_center_of_mem_sphere`, but with the distances the other way round (analogous to the pair of lemmas `mem_sphere` and `mem_sphere'`).
  • Loading branch information
jsm28 committed Nov 8, 2022
1 parent 936f0a8 commit 2daeda4
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/geometry/euclidean/basic.lean
Expand Up @@ -729,6 +729,10 @@ lemma dist_center_eq_dist_center_of_mem_sphere {p₁ p₂ : P} {s : sphere P} (h
(hp₂ : p₂ ∈ s) : dist p₁ s.center = dist p₂ s.center :=
by rw [mem_sphere.1 hp₁, mem_sphere.1 hp₂]

lemma dist_center_eq_dist_center_of_mem_sphere' {p₁ p₂ : P} {s : sphere P} (hp₁ : p₁ ∈ s)
(hp₂ : p₂ ∈ s) : dist s.center p₁ = dist s.center p₂ :=
by rw [mem_sphere'.1 hp₁, mem_sphere'.1 hp₂]

/-- A set of points is cospherical if they are equidistant from some
point. In two dimensions, this is the same thing as being
concyclic. -/
Expand Down

0 comments on commit 2daeda4

Please sign in to comment.