Absolute values in ordered groups #
The absolute value of an element in a group which is also a lattice is its supremum with its
negation. This generalizes the usual absolute value on real numbers (|x| = max x (-x)).
Notations #
- |a|: The absolute value of an element- aof an additive lattice ordered group
- |a|ₘ: The absolute value of an element- aof a multiplicative lattice ordered group
mabs a, denoted |a|ₘ, is the absolute value of a.
Equations
- One or more equations did not get rendered due to their size.
Instances For
abs a, denoted |a|, is the absolute value of a
Equations
- One or more equations did not get rendered due to their size.
Instances For
Unexpander for the notation |a|ₘ for mabs a.
Tries to add discretionary parentheses in unparsable cases.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Unexpander for the notation |a| for abs a.
Tries to add discretionary parentheses in unparsable cases.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
theorem
abs_nonneg
{α : Type u_1}
[Lattice α]
[AddGroup α]
[AddLeftMono α]
[AddRightMono α]
(a : α)
 :
The absolute value satisfies the triangle inequality.
theorem
sup_div_inf_eq_mabs_div
{α : Type u_1}
[Lattice α]
[CommGroup α]
[MulLeftMono α]
(a b : α)
 :
theorem
sup_sub_inf_eq_abs_sub
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
[AddLeftMono α]
(a b : α)
 :
theorem
two_nsmul_sup_eq_add_add_abs_sub
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
[AddLeftMono α]
(a b : α)
 :
theorem
two_nsmul_inf_eq_add_sub_abs_sub
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
[AddLeftMono α]
(a b : α)
 :
theorem
abs_sup_sub_sup_le_abs
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
[AddLeftMono α]
(a b c : α)
 :
theorem
abs_inf_sub_inf_le_abs
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
[AddLeftMono α]
(a b c : α)
 :
theorem
mabs_by_cases
{α : Type u_1}
[Group α]
[LinearOrder α]
{a : α}
(P : α → Prop)
(h1 : P a)
(h2 : P a⁻¹)
 :
P (mabs a)
theorem
abs_by_cases
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
{a : α}
(P : α → Prop)
(h1 : P a)
(h2 : P (-a))
 :
@[simp]
theorem
one_lt_mabs_pos_of_one_lt
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a : α}
(h : 1 < a)
 :
theorem
abs_pos_of_pos
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a : α}
(h : 0 < a)
 :
theorem
one_lt_mabs_of_lt_one
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a : α}
(h : a < 1)
 :
theorem
abs_pos_of_neg
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a : α}
(h : a < 0)
 :
theorem
mabs_ne_one
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a : α}
[MulRightMono α]
 :
theorem
abs_ne_zero
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a : α}
[AddRightMono α]
 :
@[simp]
theorem
mabs_eq_one
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a : α}
[MulRightMono α]
 :
@[simp]
theorem
abs_eq_zero
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a : α}
[AddRightMono α]
 :
@[simp]
theorem
mabs_le_one
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a : α}
[MulRightMono α]
 :
@[simp]
theorem
abs_nonpos_iff
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a : α}
[AddRightMono α]
 :
theorem
mabs_le_mabs_of_le_one
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a b : α}
[MulRightMono α]
(ha : a ≤ 1)
(hab : b ≤ a)
 :
theorem
abs_le_abs_of_nonpos
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a b : α}
[AddRightMono α]
(ha : a ≤ 0)
(hab : b ≤ a)
 :
theorem
mabs_lt
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a b : α}
[MulRightMono α]
 :
theorem
abs_lt
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a b : α}
[AddRightMono α]
 :
theorem
inv_lt_of_mabs_lt
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
{a b : α}
[MulRightMono α]
(h : mabs a < b)
 :
theorem
neg_lt_of_abs_lt
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
{a b : α}
[AddRightMono α]
(h : |a| < b)
 :
theorem
max_div_min_eq_mabs'
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
[MulRightMono α]
(a b : α)
 :
theorem
max_sub_min_eq_abs'
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
[AddRightMono α]
(a b : α)
 :
theorem
max_div_min_eq_mabs
{α : Type u_1}
[Group α]
[LinearOrder α]
[MulLeftMono α]
[MulRightMono α]
(a b : α)
 :
theorem
max_sub_min_eq_abs
{α : Type u_1}
[AddGroup α]
[LinearOrder α]
[AddLeftMono α]
[AddRightMono α]
(a b : α)
 :
A set s in a lattice ordered group is solid if for all x ∈ s and all y ∈ α such that
|y| ≤ |x|, then y ∈ s.
Instances For
theorem
LatticeOrderedAddCommGroup.isSolid_solidClosure
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
(s : Set α)
 :
IsSolid (solidClosure s)
theorem
LatticeOrderedAddCommGroup.solidClosure_min
{α : Type u_1}
[Lattice α]
[AddCommGroup α]
{s t : Set α}
(hst : s ⊆ t)
(ht : IsSolid t)
 :