src/HOL/Ring_and_Field.thy
changeset 23879 4776af8be741
parent 23550 d4f1d6ef119c
child 24286 7619080e49f0
--- a/src/HOL/Ring_and_Field.thy	Fri Jul 20 14:27:56 2007 +0200
+++ b/src/HOL/Ring_and_Field.thy	Fri Jul 20 14:28:01 2007 +0200
@@ -296,7 +296,7 @@
 
 instance lordered_ring \<subseteq> lordered_ab_group_join ..
 
-class abs_if = minus + ord + zero +
+class abs_if = minus + ord + zero + abs +
   assumes abs_if: "abs a = (if a \<sqsubset> 0 then (uminus a) else a)"
 
 (* The "strict" suffix can be seen as describing the combination of ordered_ring and no_zero_divisors.