src/HOL/Real.thy
author wenzelm
Mon, 16 Aug 2010 16:24:22 +0200
changeset 38444 796904799f4d
parent 36899 bcd6fce5bf06
child 48891 c0eafbd55de3
permissions -rw-r--r--
HTML.spans: explicit flag for preservation of original data (which would be turned into org.w3c.dom user data in XML.document_node);

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

setup {* SMT_Real.setup *}

end