src/HOL/Real.thy
author wenzelm
Thu, 28 Oct 2010 22:39:59 +0200
changeset 40239 c4336e45f199
parent 36899 bcd6fce5bf06
child 48891 c0eafbd55de3
permissions -rw-r--r--
moved FOL/ex/Iff_Oracle.thy to HOL/ex where it is more accessible to most readers of isar-ref; tuned;

theory Real
imports RComplete RealVector
uses "Tools/SMT/smt_real.ML"
begin

setup {* SMT_Real.setup *}

end