author | wenzelm |
Tue, 24 Aug 1999 11:50:58 +0200 | |
changeset 7333 | 6cb15c6f1d9f |
parent 7292 | dff3470c5c62 |
child 7588 | 26384af93359 |
permissions | -rw-r--r-- |
7292 | 1 |
(* Title: HOL/RealBin.thy |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1999 University of Cambridge |
|
5 |
||
6 |
Binary arithmetic for the reals |
|
7 |
||
8 |
This case is reduced to that for the integers |
|
9 |
*) |
|
10 |
||
11 |
RealBin = RealInt + Bin + RealPow + |
|
12 |
||
13 |
instance |
|
14 |
real :: number |
|
15 |
||
16 |
defs |
|
17 |
real_number_of_def |
|
18 |
"number_of v == real_of_int (number_of v)" |
|
19 |
(*::bin=>real ::bin=>int*) |
|
20 |
||
21 |
end |