author | kleing |
Tue, 13 May 2003 08:59:21 +0200 | |
changeset 14024 | 213dcc39358f |
parent 10919 | 144ede948e58 |
child 14365 | 3d4df8c166ae |
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 + instance real :: number defs real_number_of_def "number_of v == real (number_of v :: int)" (*::bin=>real ::bin=>int*) end