src/HOL/Real.thy
author blanchet
Sat, 08 Sep 2012 21:30:31 +0200
changeset 49222 cbe8c859817c
parent 48891 c0eafbd55de3
child 51521 36fa825e0ea7
child 51539 625d2ec0bbff
permissions -rw-r--r--
for compatiblity with old datatype package: not only "recs" with "s", but also "iters" and their "fld_"/"unf_" variants

theory Real
imports RComplete RealVector
begin

ML_file "Tools/SMT/smt_real.ML"
setup SMT_Real.setup

end