src/HOL/SMT.thy
changeset 40424 7550b2cba1cb
parent 40277 4e3a3461c1a6
child 40662 798aad2229c0
--- a/src/HOL/SMT.thy	Mon Nov 08 11:49:28 2010 +0100
+++ b/src/HOL/SMT.thy	Mon Nov 08 12:13:44 2010 +0100
@@ -8,7 +8,9 @@
 imports List
 uses
   "Tools/Datatype/datatype_selectors.ML"
-  ("Tools/SMT/smt_monomorph.ML")
+  "Tools/SMT/smt_failure.ML"
+  "Tools/SMT/smt_config.ML"
+  "Tools/SMT/smt_monomorph.ML"
   ("Tools/SMT/smt_builtin.ML")
   ("Tools/SMT/smt_normalize.ML")
   ("Tools/SMT/smt_translate.ML")
@@ -126,7 +128,6 @@
 
 subsection {* Setup *}
 
-use "Tools/SMT/smt_monomorph.ML"
 use "Tools/SMT/smt_builtin.ML"
 use "Tools/SMT/smt_normalize.ML"
 use "Tools/SMT/smt_translate.ML"
@@ -141,6 +142,7 @@
 use "Tools/SMT/smt_setup_solvers.ML"
 
 setup {*
+  SMT_Config.setup #>
   SMT_Solver.setup #>
   Z3_Proof_Reconstruction.setup #>
   SMT_Setup_Solvers.setup
@@ -241,6 +243,13 @@
 subsection {* Tracing *}
 
 text {*
+The SMT method, when applied, traces important information.  To
+make it entirely silent, set the following option to @{text false}.
+*}
+
+declare [[ smt_verbose = true ]]
+
+text {*
 For tracing the generated problem file given to the SMT solver as
 well as the returned result of the solver, the option
 @{text smt_trace} should be set to @{text true}.