Absolute values in linear ordered rings. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
abs
as a monoid_with_zero_hom
.
Equations
- abs_hom = {to_fun := has_abs.abs has_neg.to_has_abs, map_zero' := _, map_one' := _, map_mul' := _}
@[simp]
@[simp]
@[simp]
theorem
max_zero_add_max_neg_zero_eq_abs_self
{α : Type u_1}
[linear_ordered_ring α]
(a : α) :
linear_order.max a 0 + linear_order.max (-a) 0 = |a|