src/HOL/Real/RealArith.thy
author wenzelm
Tue, 25 Jul 2000 00:06:46 +0200
changeset 9436 62bb04ab4b01
child 10574 8f98f0301d67
permissions -rw-r--r--
rearranged setup of arithmetic procedures, avoiding global reference values;


theory RealArith = RealBin
files "real_arith.ML":

setup real_arith_setup

end