mathlib3 documentation

analysis.convex.intrinsic

Intrinsic frontier and interior #

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

This file defines the intrinsic frontier, interior and closure of a set in a normed additive torsor. These are also known as relative frontier, interior, closure.

The intrinsic frontier/interior/closure of a set s is the frontier/interior/closure of s considered as a set in its affine span.

The intrinsic interior is in general greater than the topological interior, the intrinsic frontier in general less than the topological frontier, and the intrinsic closure in cases of interest the same as the topological closure.

Definitions #

Results #

The main results are:

References #

TODO #

def intrinsic_interior (𝕜 : Type u_1) {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
set P

The intrinsic interior of a set is its interior considered as a set in its affine span.

Equations
def intrinsic_frontier (𝕜 : Type u_1) {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
set P

The intrinsic frontier of a set is its frontier considered as a set in its affine span.

Equations
def intrinsic_closure (𝕜 : Type u_1) {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
set P

The intrinsic closure of a set is its closure considered as a set in its affine span.

Equations
@[simp]
theorem mem_intrinsic_interior {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} {x : P} :
@[simp]
theorem mem_intrinsic_frontier {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} {x : P} :
@[simp]
theorem mem_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} {x : P} :
theorem intrinsic_interior_subset {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
theorem intrinsic_frontier_subset {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} (hs : is_closed s) :
theorem intrinsic_frontier_subset_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
theorem subset_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
@[simp]
theorem intrinsic_interior_empty {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] :
@[simp]
theorem intrinsic_frontier_empty {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] :
@[simp]
theorem intrinsic_closure_empty {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] :
@[simp]
theorem intrinsic_closure_nonempty {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
@[protected]
theorem set.nonempty.intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :

Alias of the reverse direction of intrinsic_closure_nonempty.

theorem set.nonempty.of_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :

Alias of the forward direction of intrinsic_closure_nonempty.

@[simp]
theorem intrinsic_interior_singleton {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (x : P) :
intrinsic_interior 𝕜 {x} = {x}
@[simp]
theorem intrinsic_frontier_singleton {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (x : P) :
@[simp]
theorem intrinsic_closure_singleton {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (x : P) :
intrinsic_closure 𝕜 {x} = {x}

Note that neither intrinsic_interior nor intrinsic_frontier is monotone.

theorem intrinsic_closure_mono {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s t : set P} (h : s t) :
theorem interior_subset_intrinsic_interior {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
theorem intrinsic_closure_subset_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
theorem intrinsic_frontier_subset_frontier {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
theorem intrinsic_closure_subset_affine_span {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} :
@[simp]
theorem intrinsic_closure_diff_intrinsic_frontier {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
@[simp]
theorem intrinsic_closure_diff_intrinsic_interior {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
@[simp]
theorem intrinsic_interior_union_intrinsic_frontier {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
@[simp]
theorem intrinsic_frontier_union_intrinsic_interior {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
theorem is_closed_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} (hs : is_closed (affine_span 𝕜 s)) :
theorem is_closed_intrinsic_frontier {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} (hs : is_closed (affine_span 𝕜 s)) :
@[simp]
theorem affine_span_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
@[protected]
theorem is_closed.intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] {s : set P} (hs : is_closed (coe ⁻¹' s)) :
@[simp]
theorem intrinsic_closure_idem {𝕜 : Type u_1} {V : Type u_2} {P : Type u_5} [ring 𝕜] [add_comm_group V] [module 𝕜 V] [topological_space P] [add_torsor V P] (s : set P) :
@[simp]
theorem affine_isometry.image_intrinsic_interior {𝕜 : Type u_1} {V : Type u_2} {W : Type u_3} {Q : Type u_4} {P : Type u_5} [normed_field 𝕜] [seminormed_add_comm_group V] [seminormed_add_comm_group W] [normed_space 𝕜 V] [normed_space 𝕜 W] [metric_space P] [pseudo_metric_space Q] [normed_add_torsor V P] [normed_add_torsor W Q] (φ : P →ᵃⁱ[𝕜] Q) (s : set P) :
@[simp]
theorem affine_isometry.image_intrinsic_frontier {𝕜 : Type u_1} {V : Type u_2} {W : Type u_3} {Q : Type u_4} {P : Type u_5} [normed_field 𝕜] [seminormed_add_comm_group V] [seminormed_add_comm_group W] [normed_space 𝕜 V] [normed_space 𝕜 W] [metric_space P] [pseudo_metric_space Q] [normed_add_torsor V P] [normed_add_torsor W Q] (φ : P →ᵃⁱ[𝕜] Q) (s : set P) :
@[simp]
theorem affine_isometry.image_intrinsic_closure {𝕜 : Type u_1} {V : Type u_2} {W : Type u_3} {Q : Type u_4} {P : Type u_5} [normed_field 𝕜] [seminormed_add_comm_group V] [seminormed_add_comm_group W] [normed_space 𝕜 V] [normed_space 𝕜 W] [metric_space P] [pseudo_metric_space Q] [normed_add_torsor V P] [normed_add_torsor W Q] (φ : P →ᵃⁱ[𝕜] Q) (s : set P) :
@[simp]
@[protected]

The intrinsic interior of a nonempty convex set is nonempty.