src/HOL/SMT.thy
changeset 41121 5c5d05963f93
parent 41059 d2b1fc1b8e19
child 41124 1de17a2de5ad
--- a/src/HOL/SMT.thy	Tue Dec 14 00:16:30 2010 +0100
+++ b/src/HOL/SMT.thy	Wed Dec 15 08:39:24 2010 +0100
@@ -205,6 +205,13 @@
 declare [[ smt_timeout = 20 ]]
 
 text {*
+SMT solvers apply randomized heuristics.  In case a problem is not
+solvable by an SMT solver, changing the following option might help.
+*}
+
+declare [[ smt_random_seed = 1 ]]
+
+text {*
 In general, the binding to SMT solvers runs as an oracle, i.e, the SMT
 solvers are fully trusted without additional checks.  The following
 option can cause the SMT solver to run in proof-producing mode, giving