src/HOL/Nitpick_Examples/Core_Nits.thy
changeset 38185 b51677438b3a
parent 37704 c6161bee8486
child 39221 70fd4a3c41ed
--- a/src/HOL/Nitpick_Examples/Core_Nits.thy	Tue Aug 03 17:29:54 2010 +0200
+++ b/src/HOL/Nitpick_Examples/Core_Nits.thy	Tue Aug 03 17:43:15 2010 +0200
@@ -11,8 +11,8 @@
 imports Main
 begin
 
-nitpick_params [unary_ints, max_potential = 0, sat_solver = MiniSat_JNI,
-                max_threads = 1, timeout = 60 s]
+nitpick_params [card = 1\<midarrow>6, unary_ints, max_potential = 0,
+                sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60 s]
 
 subsection {* Curry in a Hurry *}