Documentation

Mathlib.Geometry.Euclidean.Triangle

Triangles #

This file proves basic geometrical results about distances and angles in (possibly degenerate) triangles in real inner product spaces and Euclidean affine spaces. More specialized results, and results developed for simplices in general rather than just for triangles, are in separate files. Definitions and results that make sense in more general affine spaces rather than just in the Euclidean case go under LinearAlgebra.AffineSpace.

Implementation notes #

Results in this file are generally given in a form with only those non-degeneracy conditions needed for the particular result, rather than requiring affine independence of the points of a triangle unnecessarily.

References #

Geometrical results on triangles in real inner product spaces #

This section develops some results on (possibly degenerate) triangles in real inner product spaces, where those definitions and results can most conveniently be developed in terms of vectors and then used to deduce corresponding results for Euclidean affine spaces.

The cosine of the sum of two angles in a possibly degenerate triangle (where two given sides are nonzero), vector angle form.

The sine of the sum of two angles in a possibly degenerate triangle (where two given sides are nonzero), vector angle form.

The cosine of the sum of the angles of a possibly degenerate triangle (where two given sides are nonzero), vector angle form.

The sine of the sum of the angles of a possibly degenerate triangle (where two given sides are nonzero), vector angle form.

The sum of the angles of a possibly degenerate triangle (where the two given sides are nonzero), vector angle form.

Geometrical results on triangles in Euclidean affine spaces #

This section develops some geometrical definitions and results on (possibly degenerate) triangles in Euclidean affine spaces.

theorem EuclideanGeometry.dist_sq_eq_dist_sq_add_dist_sq_sub_two_mul_dist_mul_dist_mul_cos_angle {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (p1 : P) (p2 : P) (p3 : P) :
dist p1 p3 * dist p1 p3 = dist p1 p2 * dist p1 p2 + dist p3 p2 * dist p3 p2 - 2 * dist p1 p2 * dist p3 p2 * Real.cos (EuclideanGeometry.angle p1 p2 p3)

Law of cosines (cosine rule), angle-at-point form.

theorem EuclideanGeometry.law_cos {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (p1 : P) (p2 : P) (p3 : P) :
dist p1 p3 * dist p1 p3 = dist p1 p2 * dist p1 p2 + dist p3 p2 * dist p3 p2 - 2 * dist p1 p2 * dist p3 p2 * Real.cos (EuclideanGeometry.angle p1 p2 p3)

Alias of EuclideanGeometry.dist_sq_eq_dist_sq_add_dist_sq_sub_two_mul_dist_mul_dist_mul_cos_angle.


Law of cosines (cosine rule), angle-at-point form.

theorem EuclideanGeometry.angle_eq_angle_of_dist_eq {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {p1 : P} {p2 : P} {p3 : P} (h : dist p1 p2 = dist p1 p3) :

Isosceles Triangle Theorem: Pons asinorum, angle-at-point form.

Converse of pons asinorum, angle-at-point form.

theorem EuclideanGeometry.angle_add_angle_add_angle_eq_pi {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] {p1 : P} {p2 : P} {p3 : P} (h2 : p2 p1) (h3 : p3 p1) :

The sum of the angles of a triangle (possibly degenerate, where the given vertex is distinct from the others), angle-at-point.

theorem EuclideanGeometry.oangle_add_oangle_add_oangle_eq_pi {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] [Module.Oriented V (Fin 2)] [Fact (FiniteDimensional.finrank V = 2)] {p1 : P} {p2 : P} {p3 : P} (h21 : p2 p1) (h32 : p3 p2) (h13 : p1 p3) :

The sum of the angles of a triangle (possibly degenerate, where the triangle is a line), oriented angles at point.

theorem EuclideanGeometry.dist_sq_mul_dist_add_dist_sq_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) (p : P) (h : EuclideanGeometry.angle b p c = Real.pi) :
dist a b ^ 2 * dist c p + dist a c ^ 2 * dist b p = dist b c * (dist a p ^ 2 + dist b p * dist c p)

Stewart's Theorem.

theorem EuclideanGeometry.dist_sq_add_dist_sq_eq_two_mul_dist_midpoint_sq_add_half_dist_sq {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (a : P) (b : P) (c : P) :
dist a b ^ 2 + dist a c ^ 2 = 2 * (dist a (midpoint b c) ^ 2 + (dist b c / 2) ^ 2)

Apollonius's Theorem.

theorem EuclideanGeometry.dist_mul_of_eq_angle_of_dist_mul {V : Type u_1} {P : Type u_2} [NormedAddCommGroup V] [InnerProductSpace V] [MetricSpace P] [NormedAddTorsor V P] (a : P) (b : P) (c : P) (a' : P) (b' : P) (c' : P) (r : ) (h : EuclideanGeometry.angle a' b' c' = EuclideanGeometry.angle a b c) (hab : dist a' b' = r * dist a b) (hcb : dist c' b' = r * dist c b) :
dist a' c' = r * dist a c