src/HOL/ex/SAT_Examples.thy
changeset 19236 150e8b0fb991
parent 17809 195045659c06
child 19534 1724ec4032c5
--- a/src/HOL/ex/SAT_Examples.thy	Fri Mar 10 16:21:49 2006 +0100
+++ b/src/HOL/ex/SAT_Examples.thy	Fri Mar 10 16:31:50 2006 +0100
@@ -1,7 +1,7 @@
 (*  Title:      HOL/ex/SAT_Examples.thy
     ID:         $Id$
     Author:     Alwen Tiu, Tjark Weber
-    Copyright   2005
+    Copyright   2005-2006
 *)
 
 header {* Examples for the 'sat' and 'satx' tactic *}
@@ -11,6 +11,7 @@
 begin
 
 ML {* set sat.trace_sat; *}
+ML {* set quick_and_dirty; *}
 
 lemma "True"
 by sat
@@ -64,10 +65,9 @@
 by satx
 
 ML {* reset sat.trace_sat; *}
+ML {* reset quick_and_dirty; *}
 
-(*
 ML {* Toplevel.profiling := 1; *}
-*)
 
 (* Translated from TPTP problem library: PUZ015-2.006.dimacs *)
 
@@ -488,8 +488,6 @@
 200 201 202 203 204
 by sat
 
-(*
 ML {* Toplevel.profiling := 0; *}
-*)
 
 end