author | wenzelm |
Mon, 29 Nov 1999 15:52:49 +0100 | |
changeset 8039 | a901bafe4578 |
parent 7706 | da41066983e5 |
child 8856 | 435187ffc64e |
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 + IntArith + instance real :: number defs real_number_of_def "number_of v == real_of_int (number_of v)" (*::bin=>real ::bin=>int*) end