Documentation

Mathlib.Analysis.Convex.GaugeRescale

"Gauge rescale" homeomorphism between convex sets #

Given two convex von Neumann bounded neighbourhoods of the origin in a real topological vector space, we construct a homeomorphism gaugeRescaleHomeomorph that sends the interior, the closure, and the frontier of one set to the interior, the closure, and the frontier of the other set.

def gaugeRescale {E : Type u_1} [AddCommGroup E] [Module E] (s : Set E) (t : Set E) (x : E) :
E

The gauge rescale map gaugeRescale s t sends each point x to the point y on the same ray that has the same gauge w.r.t. t as x has w.r.t. s.

The characteristic property is satisfied if gauge t x ≠ 0, see gauge_gaugeRescale'. In particular, it is satisfied for all x, provided that t is absorbent and von Neumann bounded.

Equations
Instances For
    theorem gaugeRescale_def {E : Type u_1} [AddCommGroup E] [Module E] (s : Set E) (t : Set E) (x : E) :
    gaugeRescale s t x = (gauge s x / gauge t x) x
    @[simp]
    theorem gaugeRescale_zero {E : Type u_1} [AddCommGroup E] [Module E] (s : Set E) (t : Set E) :
    gaugeRescale s t 0 = 0
    theorem gaugeRescale_smul {E : Type u_1} [AddCommGroup E] [Module E] (s : Set E) (t : Set E) {c : } (hc : 0 c) (x : E) :
    gaugeRescale s t (c x) = c gaugeRescale s t x
    theorem gaugeRescale_self_apply {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] {s : Set E} (hsa : Absorbent s) (hsb : Bornology.IsVonNBounded s) (x : E) :
    gaugeRescale s s x = x
    theorem gauge_gaugeRescale' {E : Type u_1} [AddCommGroup E] [Module E] (s : Set E) {t : Set E} {x : E} (hx : gauge t x 0) :
    gauge t (gaugeRescale s t x) = gauge s x
    theorem gauge_gaugeRescale {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] (s : Set E) {t : Set E} (hta : Absorbent t) (htb : Bornology.IsVonNBounded t) (x : E) :
    gauge t (gaugeRescale s t x) = gauge s x
    theorem gauge_gaugeRescale_le {E : Type u_1} [AddCommGroup E] [Module E] (s : Set E) (t : Set E) (x : E) :
    gauge t (gaugeRescale s t x) gauge s x
    theorem gaugeRescale_gaugeRescale {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] {s : Set E} {t : Set E} {u : Set E} (hta : Absorbent t) (htb : Bornology.IsVonNBounded t) (x : E) :
    def gaugeRescaleEquiv {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] (s : Set E) (t : Set E) (hsa : Absorbent s) (hsb : Bornology.IsVonNBounded s) (hta : Absorbent t) (htb : Bornology.IsVonNBounded t) :
    E E

    gaugeRescale bundled as an Equiv.

    Equations
    Instances For
      theorem mapsTo_gaugeRescale_closure {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [TopologicalAddGroup E] [ContinuousSMul E] {s : Set E} {t : Set E} (hsc : Convex s) (hs₀ : s nhds 0) (htc : Convex t) (ht₀ : 0 t) (hta : Absorbent t) :
      theorem continuous_gaugeRescale {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] [TopologicalAddGroup E] [ContinuousSMul E] {s : Set E} {t : Set E} (hs : Convex s) (hs₀ : s nhds 0) (ht : Convex t) (ht₀ : t nhds 0) (htb : Bornology.IsVonNBounded t) :
      def gaugeRescaleHomeomorph {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] [TopologicalAddGroup E] [ContinuousSMul E] (s : Set E) (t : Set E) (hsc : Convex s) (hs₀ : s nhds 0) (hsb : Bornology.IsVonNBounded s) (htc : Convex t) (ht₀ : t nhds 0) (htb : Bornology.IsVonNBounded t) :
      E ≃ₜ E

      gaugeRescale bundled as a Homeomorph.

      Equations
      Instances For
        theorem image_gaugeRescaleHomeomorph_interior {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] [TopologicalAddGroup E] [ContinuousSMul E] {s : Set E} {t : Set E} (hsc : Convex s) (hs₀ : s nhds 0) (hsb : Bornology.IsVonNBounded s) (htc : Convex t) (ht₀ : t nhds 0) (htb : Bornology.IsVonNBounded t) :
        (gaugeRescaleHomeomorph s t hsc hs₀ hsb htc ht₀ htb) '' interior s = interior t
        theorem image_gaugeRescaleHomeomorph_closure {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] [TopologicalAddGroup E] [ContinuousSMul E] {s : Set E} {t : Set E} (hsc : Convex s) (hs₀ : s nhds 0) (hsb : Bornology.IsVonNBounded s) (htc : Convex t) (ht₀ : t nhds 0) (htb : Bornology.IsVonNBounded t) :
        (gaugeRescaleHomeomorph s t hsc hs₀ hsb htc ht₀ htb) '' closure s = closure t
        theorem exists_homeomorph_image_eq {E : Type u_1} [AddCommGroup E] [Module E] [TopologicalSpace E] [T1Space E] [TopologicalAddGroup E] [ContinuousSMul E] {s : Set E} {t : Set E} (hsc : Convex s) (hsne : Set.Nonempty (interior s)) (hsb : Bornology.IsVonNBounded s) (hst : Convex t) (htne : Set.Nonempty (interior t)) (htb : Bornology.IsVonNBounded t) :
        ∃ (e : E ≃ₜ E), e '' interior s = interior t e '' closure s = closure t e '' frontier s = frontier t

        Given two convex bounded sets in a topological vector space with nonempty interiors, there exists a homeomorphism of the ambient space that sends the interior, the closure, and the frontier of one set to the interior, the closure, and the frontier of the other set.

        In particular, if both s and t are open set or both s and t are closed sets, then e maps s to t.

        If s is a convex bounded set with a nonempty interior in a real normed space, then there is a homeomorphism of the ambient space to itself that sends the interior of s to the unit open ball and the closure of s to the unit closed ball.