Documentation

Mathlib.Topology.Bornology.BoundedOperation

Bounded operations #

This file introduces type classes for bornologically bounded operations.

In particular, when combined with type classes which guarantee continuity of the same operations, we can equip bounded continuous functions with the corresponding operations.

Main definitions #

TODO:

Bounded subtraction #

class BoundedSub (R : Type u_1) [Bornology R] [Sub R] :

A typeclass saying that (p : R × R) ↦ p.1 - p.2 maps any pair of bounded sets to a bounded set. This property automatically holds for seminormed additive groups, but it also holds, e.g., for ℝ≥0.

Instances
    theorem BoundedSub.isBounded_sub {R : Type u_1} [Bornology R] [Sub R] [self : BoundedSub R] {s : Set R} {t : Set R} :
    theorem isBounded_sub {R : Type u_1} [Bornology R] [Sub R] [BoundedSub R] {s : Set R} {t : Set R} (hs : Bornology.IsBounded s) (ht : Bornology.IsBounded t) :
    theorem sub_bounded_of_bounded_of_bounded {R : Type u_1} {X : Type u_2} [PseudoMetricSpace R] [Sub R] [BoundedSub R] {f : XR} {g : XR} (f_bdd : ∃ (C : ), ∀ (x y : X), dist (f x) (f y) C) (g_bdd : ∃ (C : ), ∀ (x y : X), dist (g x) (g y) C) :
    ∃ (C : ), ∀ (x y : X), dist ((f - g) x) ((f - g) y) C

    Bounded operations in seminormed additive commutative groups #

    Equations
    • =

    Bounded operations in ℝ≥0 #