mathlib3 documentation

analysis.normed_space.add_torsor_bases

Bases in normed affine spaces. #

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

This file contains results about bases in normed affine spaces.

Main definitions: #

theorem is_open_map_barycentric_coord {ι : Type u_1} {𝕜 : Type u_2} {E : Type u_3} {P : Type u_4} [nontrivially_normed_field 𝕜] [complete_space 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] [metric_space P] [normed_add_torsor E P] [nontrivial ι] (b : affine_basis ι 𝕜 P) (i : ι) :
@[continuity]
theorem continuous_barycentric_coord {ι : Type u_1} {𝕜 : Type u_2} {E : Type u_3} {P : Type u_4} [nontrivially_normed_field 𝕜] [complete_space 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] [metric_space P] [normed_add_torsor E P] [finite_dimensional 𝕜 E] (b : affine_basis ι 𝕜 P) (i : ι) :
theorem smooth_barycentric_coord {ι : Type u_1} {𝕜 : Type u_2} {E : Type u_3} [nontrivially_normed_field 𝕜] [complete_space 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] [finite_dimensional 𝕜 E] (b : affine_basis ι 𝕜 E) (i : ι) :
theorem affine_basis.interior_convex_hull {ι : Type u_1} {E : Type u_2} [finite ι] [normed_add_comm_group E] [normed_space E] (b : affine_basis ι E) :
interior ((convex_hull ) (set.range b)) = {x : E | (i : ι), 0 < (b.coord i) x}

Given a finite-dimensional normed real vector space, the interior of the convex hull of an affine basis is the set of points whose barycentric coordinates are strictly positive with respect to this basis.

TODO Restate this result for affine spaces (instead of vector spaces) once the definition of convexity is generalised to this setting.

Given a set s of affine-independent points belonging to an open set u, we may extend s to an affine basis, all of whose elements belong to u.

theorem is_open.affine_span_eq_top {V : Type u_1} {P : Type u_2} [normed_add_comm_group V] [normed_space V] [metric_space P] [normed_add_torsor V P] {u : set P} (hu : is_open u) (hne : u.nonempty) :

The affine span of a nonempty open set is .