src/HOL/Real/RealArith.thy
author nipkow
Fri, 01 Dec 2000 19:53:29 +0100
changeset 10574 8f98f0301d67
parent 9436 62bb04ab4b01
child 10722 55c8367bab05
permissions -rw-r--r--
Linear arithmetic now copes with mixed nat/int formulae.

theory RealArith = RealBin
files "real_arith.ML":

setup real_arith_setup

end