author | wenzelm |
Mon, 29 Nov 1999 15:52:49 +0100 | |
changeset 8039 | a901bafe4578 |
parent 7588 | 26384af93359 |
child 8838 | 4eaa99f0d223 |
permissions | -rw-r--r-- |
7334 | 1 |
(* Title: Real/RealOrd.thy |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C. Paulson |
|
4 |
Jacques D. Fleuriot |
|
5 |
Copyright: 1998 University of Cambridge |
|
6 |
Description: Type "real" is a linear order |
|
7 |
*) |
|
8 |
||
9 |
RealOrd = RealDef + |
|
10 |
||
11 |
instance real :: order (real_le_refl,real_le_trans,real_le_anti_sym,real_less_le) |
|
12 |
instance real :: linorder (real_le_linear) |
|
13 |
||
7588
26384af93359
Tidying to exploit the new arith_tac. RealBin no longer imports RealPow or
paulson
parents:
7334
diff
changeset
|
14 |
constdefs |
26384af93359
Tidying to exploit the new arith_tac. RealBin no longer imports RealPow or
paulson
parents:
7334
diff
changeset
|
15 |
rabs :: real => real |
26384af93359
Tidying to exploit the new arith_tac. RealBin no longer imports RealPow or
paulson
parents:
7334
diff
changeset
|
16 |
"rabs r == if 0r<=r then r else -r" |
26384af93359
Tidying to exploit the new arith_tac. RealBin no longer imports RealPow or
paulson
parents:
7334
diff
changeset
|
17 |
|
7334 | 18 |
end |