src/HOL/Real.thy
author blanchet
Tue, 07 Dec 2010 11:56:01 +0100
changeset 41045 2a41709f34c1
parent 36899 bcd6fce5bf06
child 48891 c0eafbd55de3
permissions -rw-r--r--
use heuristic to determine whether to keep or drop an existing "let" -- and drop all higher-order lets

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

setup {* SMT_Real.setup *}

end