src/HOL/Real/RealAbs.thy
author oheimb
Mon, 06 Sep 1999 18:19:12 +0200
changeset 7497 a18f3bce7198
parent 7334 a90fc1e5fb19
child 7588 26384af93359
permissions -rw-r--r--
strengthened card_seteq

(*  Title       : RealAbs.thy
    ID          : $Id$
    Author      : Jacques D. Fleuriot
    Copyright   : 1998  University of Cambridge
    Description : Absolute value function for the reals
*) 

RealAbs = RealOrd +

constdefs
   rabs   :: real => real
   "rabs r      == if 0r<=r then r else -r" 

end