src/HOL/Nitpick_Examples/Typedef_Nits.thy
changeset 41278 8e1cde88aae6
parent 40590 b994d855dbd2
child 42142 d24a93025feb
--- a/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Sun Dec 19 00:13:25 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Sun Dec 19 11:48:42 2010 +0100
@@ -11,7 +11,7 @@
 imports Complex_Main
 begin
 
-nitpick_params [card = 1\<midarrow>4, sat_solver = MiniSat_JNI, max_threads = 1,
+nitpick_params [verbose, card = 1\<midarrow>4, sat_solver = MiniSat_JNI, max_threads = 1,
                 timeout = 60]
 
 typedef three = "{0\<Colon>nat, 1, 2}"