src/HOL/Real/RealAbs.thy
changeset 8856 435187ffc64e
parent 7588 26384af93359
child 9013 9dd0274f76af
--- a/src/HOL/Real/RealAbs.thy	Wed May 10 21:04:16 2000 +0200
+++ b/src/HOL/Real/RealAbs.thy	Wed May 10 22:34:30 2000 +0200
@@ -5,6 +5,6 @@
     Description : Absolute value function for the reals
 *) 
 
-RealAbs = RealOrd + RealBin +
+RealAbs = RealBin +
 
 end