src/HOL/Real/RealAbs.thy
author nipkow
Mon, 04 Jan 1999 15:07:47 +0100
changeset 6055 fdf4638bf726
parent 5588 a3ab526bb891
child 7219 4e3f386c2e37
permissions -rw-r--r--
Version 1.0 of linear nat arithmetic.

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

RealAbs = Real +

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

end