src/HOL/Real/RealAbs.thy
author berghofe
Fri, 23 Oct 1998 22:36:15 +0200
changeset 5760 7e2cf2820684
parent 5588 a3ab526bb891
child 7219 4e3f386c2e37
permissions -rw-r--r--
Added theorems True_not_False and False_not_True (for rep_datatype).

(*  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