Documentation

Mathlib.Geometry.Euclidean.Inversion.Basic

Inversion in an affine space #

In this file we define inversion in a sphere in an affine space. This map sends each point x to the point y such that y -ᵥ c = (R / dist x c) ^ 2 • (x -ᵥ c), where c and R are the center and the radius the sphere.

In many applications, it is convenient to assume that the inversions swaps the center and the point at infinity. In order to stay in the original affine space, we define the map so that it sends center to itself.

Currently, we prove only a few basic lemmas needed to prove Ptolemy's inequality, see EuclideanGeometry.mul_dist_le_mul_dist_add_mul_dist.

def EuclideanGeometry.inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (c : P) (R : ) (x : P) :
P

Inversion in a sphere in an affine space. This map sends each point x to the point y such that y -ᵥ c = (R / dist x c) ^ 2 • (x -ᵥ c), where c and R are the center and the radius the sphere.

Equations
Instances For
    theorem EuclideanGeometry.inversion_def {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] :
    EuclideanGeometry.inversion = fun (c : P) (R : ) (x : P) => (R / dist x c) ^ 2 (x -ᵥ c) +ᵥ c

    Basic properties #

    In this section we prove that EuclideanGeometry.inversion c R is involutive and preserves the sphere Metric.sphere c R. We also prove that the distance to the center of the image of x under this inversion is given by R ^ 2 / dist x c.

    Distance from the image of a point under inversion to the center. This formula accidentally works for x = c.

    Distance from the center of an inversion to the image of a point under the inversion. This formula accidentally works for x = c.

    theorem EuclideanGeometry.inversion_eq_center {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {c : P} {x : P} {R : } (hR : R 0) :
    @[simp]
    theorem EuclideanGeometry.center_eq_inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {c : P} {x : P} {R : } (hR : R 0) :
    @[simp]

    Similarity of triangles #

    If inversion with center O sends A to A' and B to B', then the triangle OB'A' is similar to the triangle OAB with coefficient R ^ 2 / (|OA|*|OB|) and the triangle OA'B is similar to the triangle OAB' with coefficient |OB|/|OA|. We formulate these statements in terms of ratios of the lengths of their sides.

    theorem EuclideanGeometry.dist_inversion_inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {c : P} {x : P} {y : P} (hx : x c) (hy : y c) (R : ) :

    Distance between the images of two points under an inversion.

    theorem EuclideanGeometry.dist_inversion_mul_dist_center_eq {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {c : P} {x : P} {y : P} {R : } (hx : x c) (hy : y c) :

    Ptolemy's inequality #

    theorem EuclideanGeometry.mul_dist_le_mul_dist_add_mul_dist {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (a : P) (b : P) (c : P) (d : P) :
    dist a c * dist b d dist a b * dist c d + dist b c * dist a d

    Ptolemy's inequality: in a quadrangle ABCD, |AC| * |BD| ≤ |AB| * |CD| + |BC| * |AD|. If ABCD is a convex cyclic polygon, then this inequality becomes an equality, see EuclideanGeometry.mul_dist_add_mul_dist_eq_mul_dist_of_cospherical.

    Continuity of inversion #

    theorem Filter.Tendsto.inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {α : Type u_3} {x : P} {c : P} {R : } {l : Filter α} {fc : αP} {fx : αP} {fR : α} (hc : Filter.Tendsto fc l (nhds c)) (hR : Filter.Tendsto fR l (nhds R)) (hx : Filter.Tendsto fx l (nhds x)) (hne : x c) :
    Filter.Tendsto (fun (a : α) => EuclideanGeometry.inversion (fc a) (fR a) (fx a)) l (nhds (EuclideanGeometry.inversion c R x))
    theorem ContinuousWithinAt.inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {X : Type u_3} [TopologicalSpace X] {c : XP} {x : XP} {R : X} {a₀ : X} {s : Set X} (hc : ContinuousWithinAt c s a₀) (hR : ContinuousWithinAt R s a₀) (hx : ContinuousWithinAt x s a₀) (hne : x a₀ c a₀) :
    ContinuousWithinAt (fun (a : X) => EuclideanGeometry.inversion (c a) (R a) (x a)) s a₀
    theorem ContinuousAt.inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {X : Type u_3} [TopologicalSpace X] {c : XP} {x : XP} {R : X} {a₀ : X} (hc : ContinuousAt c a₀) (hR : ContinuousAt R a₀) (hx : ContinuousAt x a₀) (hne : x a₀ c a₀) :
    ContinuousAt (fun (a : X) => EuclideanGeometry.inversion (c a) (R a) (x a)) a₀
    theorem ContinuousOn.inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {X : Type u_3} [TopologicalSpace X] {c : XP} {x : XP} {R : X} {s : Set X} (hc : ContinuousOn c s) (hR : ContinuousOn R s) (hx : ContinuousOn x s) (hne : as, x a c a) :
    ContinuousOn (fun (a : X) => EuclideanGeometry.inversion (c a) (R a) (x a)) s
    theorem Continuous.inversion {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {X : Type u_3} [TopologicalSpace X] {c : XP} {x : XP} {R : X} (hc : Continuous c) (hR : Continuous R) (hx : Continuous x) (hne : ∀ (a : X), x a c a) :
    Continuous fun (a : X) => EuclideanGeometry.inversion (c a) (R a) (x a)