| author | oheimb |
| Mon, 06 Sep 1999 18:19:12 +0200 | |
| changeset 7497 | a18f3bce7198 |
| parent 7334 | a90fc1e5fb19 |
| child 7588 | 26384af93359 |
| 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 |
||
| 7334 | 8 |
RealAbs = RealOrd + |
| 5078 | 9 |
|
10 |
constdefs |
|
11 |
rabs :: real => real |
|
| 5588 | 12 |
"rabs r == if 0r<=r then r else -r" |
| 5078 | 13 |
|
14 |
end |