Documentation

Mathlib.Geometry.Euclidean.Sphere.SecondInter

Second intersection of a sphere and a line #

This file defines and proves basic results about the second intersection of a sphere with a line through a point on that sphere.

Main definitions #

The second intersection of a sphere with a line through a point on that sphere; that point if it is the only point of intersection of the line with the sphere. The intended use of this definition is when p ∈ s; the definition does not use s.radius, so in general it returns the second intersection with the sphere through p and with center s.center.

Equations
Instances For
    @[simp]

    The distance between secondInter and the center equals the distance between the original point and the center.

    @[simp]

    The point given by secondInter lies on the sphere.

    @[simp]

    If the vector is zero, secondInter gives the original point.

    The point given by secondInter equals the original point if and only if the line is orthogonal to the radius vector.

    A point on a line through a point on a sphere equals that point or secondInter.

    @[simp]

    secondInter is unchanged by multiplying the vector by a nonzero real.

    theorem EuclideanGeometry.Sphere.secondInter_eq_lineMap {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (s : EuclideanGeometry.Sphere P) (p : P) (p' : P) :
    EuclideanGeometry.Sphere.secondInter s p (p' -ᵥ p) = (AffineMap.lineMap p p') (-2 * p' -ᵥ p, p -ᵥ s.center⟫_ / p' -ᵥ p, p' -ᵥ p⟫_)

    If the vector passed to secondInter is given by a subtraction involving the point in secondInter, the result of secondInter may be expressed using lineMap.

    If the vector passed to secondInter is given by a subtraction involving the point in secondInter, the result lies in the span of the two points.

    If the vector passed to secondInter is given by a subtraction involving the point in secondInter, the three points are collinear.

    theorem EuclideanGeometry.Sphere.wbtw_secondInter {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {s : EuclideanGeometry.Sphere P} {p : P} {p' : P} (hp : p s) (hp' : dist p' s.center s.radius) :

    If the vector passed to secondInter is given by a subtraction involving the point in secondInter, and the second point is not outside the sphere, the second point is weakly between the first point and the result of secondInter.

    theorem EuclideanGeometry.Sphere.sbtw_secondInter {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {s : EuclideanGeometry.Sphere P} {p : P} {p' : P} (hp : p s) (hp' : dist p' s.center < s.radius) :

    If the vector passed to secondInter is given by a subtraction involving the point in secondInter, and the second point is inside the sphere, the second point is strictly between the first point and the result of secondInter.