author | wenzelm |
Tue, 06 Aug 2002 11:22:05 +0200 | |
changeset 13462 | 56610e2ba220 |
parent 10919 | 144ede948e58 |
child 14365 | 3d4df8c166ae |
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 |
||
8856 | 11 |
RealBin = RealInt + |
7292 | 12 |
|
13 |
instance |
|
14 |
real :: number |
|
15 |
||
16 |
defs |
|
17 |
real_number_of_def |
|
10919
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
8856
diff
changeset
|
18 |
"number_of v == real (number_of v :: int)" |
144ede948e58
renamings: real_of_nat, real_of_int -> (overloaded) real
paulson
parents:
8856
diff
changeset
|
19 |
(*::bin=>real ::bin=>int*) |
7292 | 20 |
|
21 |
end |