src/HOL/Nitpick_Examples/Manual_Nits.thy
changeset 41278 8e1cde88aae6
parent 40341 03156257040f
child 41413 64cd30d6b0b8
--- a/src/HOL/Nitpick_Examples/Manual_Nits.thy	Sun Dec 19 00:13:25 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Manual_Nits.thy	Sun Dec 19 11:48:42 2010 +0100
@@ -17,7 +17,8 @@
 
 chapter {* 3. First Steps *}
 
-nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60]
+nitpick_params [verbose, sat_solver = MiniSat_JNI, max_threads = 1,
+                timeout = 60]
 
 subsection {* 3.1. Propositional Logic *}