src/HOL/Real/RealAbs.thy
author fleuriot
Thu, 01 Jun 2000 11:22:27 +0200
changeset 9013 9dd0274f76af
parent 8856 435187ffc64e
child 9429 8ebc549e9326
permissions -rw-r--r--
Updated files to remove 0r and 1r from theorems in descendant theories of RealBin. Some new theorems added.

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

RealAbs = RealBin +


defs
  abs_real_def "abs r == (if (#0::real) <= r then r else -r)"

end