author | wenzelm |
Mon, 29 Nov 1999 15:52:49 +0100 | |
changeset 8039 | a901bafe4578 |
parent 7588 | 26384af93359 |
child 8856 | 435187ffc64e |
permissions | -rw-r--r-- |
5078 | 1 |
(* Title : RealAbs.thy |
7219 | 2 |
ID : $Id$ |
5078 | 3 |
Author : Jacques D. Fleuriot |
4 |
Copyright : 1998 University of Cambridge |
|
5 |
Description : Absolute value function for the reals |
|
6 |
*) |
|
7 |
||
7588
26384af93359
Tidying to exploit the new arith_tac. RealBin no longer imports RealPow or
paulson
parents:
7334
diff
changeset
|
8 |
RealAbs = RealOrd + RealBin + |
5078 | 9 |
|
7588
26384af93359
Tidying to exploit the new arith_tac. RealBin no longer imports RealPow or
paulson
parents:
7334
diff
changeset
|
10 |
end |