src/HOL/Real.thy
author wenzelm
Sat, 20 Aug 2011 23:35:30 +0200
changeset 44338 700008399ee5
parent 36899 bcd6fce5bf06
child 48891 c0eafbd55de3
permissions -rw-r--r--
refined Graph implementation: more abstract/scalable Graph.Keys instead of plain lists -- order of adjacency is now standardized wrt. Key.ord;

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

setup {* SMT_Real.setup *}

end