src/HOL/Real/RealAbs.thy
author wenzelm
Mon, 29 Nov 1999 15:52:49 +0100
changeset 8039 a901bafe4578
parent 7588 26384af93359
child 8856 435187ffc64e
permissions -rw-r--r--
Goal: tuned pris;

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

RealAbs = RealOrd + RealBin +

end