src/HOL/Main.thy
changeset 14350 41b32020d0b3
parent 14192 d6cb80cc1d20
child 14443 75910c7557c5
--- a/src/HOL/Main.thy	Sat Jan 10 12:34:50 2004 +0100
+++ b/src/HOL/Main.thy	Sat Jan 10 13:35:10 2004 +0100
@@ -1,12 +1,12 @@
 (*  Title:      HOL/Main.thy
     ID:         $Id$
-    Author:     Stefan Berghofer, Tobias Nipkow and Markus Wenzel, TU Muenchen
+    Author:     Stefan Berghofer, Tobias Nipkow, Tjark Weber, Markus Wenzel (TU Muenchen)
     License:    GPL (GNU GENERAL PUBLIC LICENSE)
 *)
 
 header {* Main HOL *}
 
-theory Main = Map + Hilbert_Choice + Extraction:
+theory Main = Map + Hilbert_Choice + Extraction + Refute:
 
 text {*
   Theory @{text Main} includes everything.  Note that theory @{text
@@ -91,4 +91,26 @@
 lemma [code]: "(0 < Suc n) = True" by simp
 lemmas [code] = Suc_less_eq imp_conv_disj
 
+subsection {* Configuration of the 'refute' command *}
+
+text {*
+  The following are reasonable default parameters (for use with
+  ZChaff 2003.12.04).  For an explanation of these parameters,
+  see 'HOL/Refute.thy'.
+
+  \emph{Note}: If you want to use a different SAT solver (or
+  install ZChaff to a different location), you will need to
+  override at least the values for 'command' and (probably)
+  'success' in your own theory file.
+*}
+
+refute_params [minsize=1,
+               maxsize=8,
+               maxvars=200,
+               satfile="refute.cnf",
+               satformat="defcnf",
+               resultfile="refute.out",
+               success="Verify Solution successful. Instance satisfiable",
+               command="$HOME/bin/zchaff refute.cnf 60 > refute.out"]
+
 end