mathlib3 documentation

geometry.euclidean.triangle

Triangles #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

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 linear_algebra.affine_space.

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 (possible degenerate) triangles in Euclidean affine spaces.

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

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

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

theorem euclidean_geometry.oangle_add_oangle_add_oangle_eq_pi {V : Type u_1} {P : Type u_2} [normed_add_comm_group V] [inner_product_space V] [metric_space P] [normed_add_torsor V P] [module.oriented V (fin 2)] [fact (fdim V = 2)] {p1 p2 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.