Spheres #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines and proves basic results about spheres and cospherical sets of points in Euclidean affine spaces.
Main definitions #
-
euclidean_geometry.sphere
bundles acenter
and aradius
. -
euclidean_geometry.cospherical
is the property of a set of points being equidistant from some point. -
euclidean_geometry.concyclic
is the property of a set of points being cospherical and coplanar.
- center : P
- radius : ℝ
A sphere P
bundles a center
and radius
. This definition does not require the radius to
be positive; that should be given as a hypothesis to lemmas that require it.
Instances for euclidean_geometry.sphere
- euclidean_geometry.sphere.has_sizeof_inst
- euclidean_geometry.sphere.nonempty
- euclidean_geometry.set.has_coe
- euclidean_geometry.sphere.has_mem
Equations
- euclidean_geometry.set.has_coe = {coe := λ (s : euclidean_geometry.sphere P), metric.sphere s.center s.radius}
Equations
- euclidean_geometry.sphere.has_mem = {mem := λ (p : P) (s : euclidean_geometry.sphere P), p ∈ ↑s}
A set of points is cospherical if they are equidistant from some point. In two dimensions, this is the same thing as being concyclic.
Equations
- euclidean_geometry.cospherical ps = ∃ (center : P) (radius : ℝ), ∀ (p : P), p ∈ ps → has_dist.dist p center = radius
The definition of cospherical
.
A set of points is cospherical if and only if they lie in some sphere.
The set of points in a sphere is cospherical.
A subset of a cospherical set is cospherical.
The empty set is cospherical.
A single point is cospherical.
Two points are cospherical.
- cospherical : euclidean_geometry.cospherical ps
- coplanar : coplanar ℝ ps
A set of points is concyclic if it is cospherical and coplanar. (Most results are stated
directly in terms of cospherical
instead of using concyclic
.)
A subset of a concyclic set is concyclic.
The empty set is concyclic.
A single point is concyclic.
Two points are concyclic.
Any three points in a cospherical set are affinely independent.
Any three points in a cospherical set are affinely independent.
The three points of a cospherical set are affinely independent.
Suppose that p₁
and p₂
lie in spheres s₁
and s₂
. Then the vector between the centers
of those spheres is orthogonal to that between p₁
and p₂
; this is a version of
inner_vsub_vsub_of_dist_eq_of_dist_eq
for bundled spheres. (In two dimensions, this says that
the diagonals of a kite are orthogonal.)
Two spheres intersect in at most two points in a two-dimensional subspace containing their
centers; this is a version of eq_of_dist_eq_of_dist_eq_of_mem_of_finrank_eq_two
for bundled
spheres.
Two spheres intersect in at most two points in two-dimensional space; this is a version of
eq_of_dist_eq_of_dist_eq_of_finrank_eq_two
for bundled spheres.
Given a point on a sphere and a point not outside it, the inner product between the difference of those points and the radius vector is positive unless the points are equal.
Given a point on a sphere and a point not outside it, the inner product between the difference of those points and the radius vector is nonnegative.
Given a point on a sphere and a point inside it, the inner product between the difference of those points and the radius vector is positive.
Given three collinear points, two on a sphere and one not outside it, the one not outside it is weakly between the other two points.
Given three collinear points, two on a sphere and one inside it, the one inside it is strictly between the other two points.