src/HOL/Nitpick_Examples/Core_Nits.thy
changeset 34082 61b7aa37f4b7
parent 33199 6c9b2a94a69c
child 34083 652719832159
--- a/src/HOL/Nitpick_Examples/Core_Nits.thy	Mon Dec 14 10:13:06 2009 +0100
+++ b/src/HOL/Nitpick_Examples/Core_Nits.thy	Mon Dec 14 10:31:35 2009 +0100
@@ -11,6 +11,8 @@
 imports Main
 begin
 
+nitpick_params [sat_solver = MiniSatJNI]
+
 subsection {* Curry in a Hurry *}
 
 lemma "(\<lambda>f x y. (curry o split) f x y) = (\<lambda>f x y. (\<lambda>x. x) f x y)"
@@ -135,7 +137,7 @@
 by (auto simp: Id_def Collect_def)
 
 lemma "Id ((a\<Colon>'a, b\<Colon>'a), (a, b))"
-nitpick [card = 1\<midarrow>20, expect = none]
+nitpick [card = 1\<midarrow>10, expect = none]
 by (auto simp: Id_def Collect_def)
 
 lemma "UNIV (x\<Colon>'a\<times>'a)"