Documentation

Mathlib.Analysis.InnerProductSpace.Affine

Normed affine spaces over an inner product space #

theorem inner_vsub_left_eq_zero_symm {š•œ : Type u_1} {V : Type u_2} {P : Type u_3} [RCLike š•œ] [NormedAddCommGroup V] [InnerProductSpace š•œ V] [MetricSpace P] [NormedAddTorsor V P] {a b : P} {v : V} :
inner š•œ (a -ᵄ b) v = 0 ↔ inner š•œ (b -ᵄ a) v = 0
theorem inner_vsub_right_eq_zero_symm {š•œ : Type u_1} {V : Type u_2} {P : Type u_3} [RCLike š•œ] [NormedAddCommGroup V] [InnerProductSpace š•œ V] [MetricSpace P] [NormedAddTorsor V P] {v : V} {a b : P} :
inner š•œ v (a -ᵄ b) = 0 ↔ inner š•œ v (b -ᵄ a) = 0

In this section, the first left/right indicates where the common argument to vsub is, and the section refers to the argument of inner that ends up in the dist.

The lemma shapes are such that the relevant argument of inner remains unchanged, and that the other vsub preserves the position of the unchanging argument.

theorem dist_sq_lineMap_lineMap_of_inner_eq_zero {V : Type u_2} {P : Type u_3} [NormedAddCommGroup V] [InnerProductSpace ā„ V] [MetricSpace P] [NormedAddTorsor V P] {a b c : P} (t₁ tā‚‚ : ā„) (h_inner : inner ā„ (b -ᵄ a) (c -ᵄ a) = 0) :
dist ((AffineMap.lineMap a b) t₁) ((AffineMap.lineMap a c) tā‚‚) ^ 2 = t₁ ^ 2 * dist a b ^ 2 + tā‚‚ ^ 2 * dist a c ^ 2

Squared distance between two points on lines from a common origin, given orthogonality of the direction vectors.

theorem dist_sq_lineMap_of_inner_eq_zero {V : Type u_2} {P : Type u_3} [NormedAddCommGroup V] [InnerProductSpace ā„ V] [MetricSpace P] [NormedAddTorsor V P] {a b p : P} (t : ā„) (h_inner : inner ā„ (p -ᵄ a) (b -ᵄ a) = 0) :
dist p ((AffineMap.lineMap a b) t) ^ 2 = dist p a ^ 2 + t ^ 2 * dist a b ^ 2

Squared distance from p to a point on the line from a to b, given that p -ᵄ a is orthogonal to b -ᵄ a.

theorem dist_sq_of_inner_eq_zero {V : Type u_2} {P : Type u_3} [NormedAddCommGroup V] [InnerProductSpace ā„ V] [MetricSpace P] [NormedAddTorsor V P] {a b p : P} (h_inner : inner ā„ (p -ᵄ a) (b -ᵄ a) = 0) :
dist p b ^ 2 = dist p a ^ 2 + dist a b ^ 2

Pythagorean theorem: if p -ᵄ a is orthogonal to b -ᵄ a, then dist p b ^ 2 = dist p a ^ 2 + dist a b ^ 2.