Positive & negative parts #
Mathematical structures possessing an absolute value often also possess a unique decomposition of elements into "positive" and "negative" parts which are in some sense "disjoint" (e.g. the Jordan decomposition of a measure).
This file provides instances of PosPart
and NegPart
, the positive and negative parts of an
element in a lattice ordered group.
Main statements #
posPart_sub_negPart
: Every elementa
can be decomposed intoa⁺ - a⁻
, the difference of its positive and negative parts.posPart_inf_negPart_eq_zero
: The positive and negative parts are coprime.
References #
- Birkhoff, Lattice-ordered Groups
- Bourbaki, Algebra II
- Fuchs, Partially Ordered Algebraic Systems
- Zaanen, Lectures on "Riesz Spaces"
- Banasiak, Banach Lattices in Applications
Tags #
positive part, negative part
The positive part of an element a
in a lattice ordered group is a ⊔ 1
, denoted a⁺ᵐ
.
Equations
- Eq instOneLePart { oneLePart := fun (a : α) => Max.max a 1 }
Instances For
The positive part of an element a
in a lattice ordered group is a ⊔ 0
, denoted a⁺
.
Equations
- Eq instPosPart { posPart := fun (a : α) => Max.max a 0 }
Instances For
The negative part of an element a
in a lattice ordered group is a⁻¹ ⊔ 1
, denoted a⁻ᵐ
.
Equations
- Eq instLeOnePart { leOnePart := fun (a : α) => Max.max (Inv.inv a) 1 }
Instances For
The negative part of an element a
in a lattice ordered group is (-a) ⊔ 0
, denoted a⁻
.
Equations
- Eq instNegPart { negPart := fun (a : α) => Max.max (Neg.neg a) 0 }
Instances For
Alias of the reverse direction of oneLePart_eq_self
.
Alias of the reverse direction of oneLePart_eq_one
.
See also leOnePart_eq_inv
.
See also negPart_eq_neg
.
See also leOnePart_eq_one
.
See also negPart_eq_zero
.
See also leOnePart_le_one
.
See also negPart_nonpos
.
Alias of the reverse direction of leOnePart_eq_inv
.
Alias of the reverse direction of leOnePart_eq_one
.