Ordered scalar product #
In this file we define
- OrderedSMul R M: an ordered additive commutative monoid- Mis an- OrderedSMulover an- OrderedSemiring- Rif the scalar product respects the order relation on the monoid and on the ring. There is a correspondence between this structure and convex cones, which is proven in- Analysis/Convex/Cone.lean.
Implementation notes #
- We choose to define OrderedSMulas aProp-valued mixin, so that it can be used for actions, modules, and algebras (the axioms for an "ordered algebra" are exactly that the algebra is ordered as a module).
- To get ordered modules and ordered vector spaces, it suffices to replace the
OrderedAddCommMonoidand theOrderedSemiringas desired.
TODO #
This file is now mostly useless. We should try deleting OrderedSMul
References #
Tags #
ordered module, ordered scalar, ordered smul, ordered action, ordered vector space
The ordered scalar product property is when an ordered additive commutative monoid with a partial order has a scalar multiplication which is compatible with the order.
- Scalar multiplication by positive elements preserves the order. 
- If - c • a < c • bfor some positive- c, then- a < b.
Instances
Scalar multiplication by positive elements preserves the order.
If c • a < c • b for some positive c, then a < b.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
To prove that a linear ordered monoid is an ordered module, it suffices to verify only the first
axiom of OrderedSMul.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
To prove that a vector space over a linear ordered field is ordered, it suffices to verify only
the first axiom of OrderedSMul.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯