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