src/HOL/Nitpick_Examples/Typedef_Nits.thy
changeset 54633 86e0b402994c
parent 51706 0a4b4735d8bd
child 54680 93f6d33a754e
--- a/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Thu Dec 05 13:22:00 2013 +0100
+++ b/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Thu Dec 05 13:38:20 2013 +0100
@@ -11,7 +11,7 @@
 imports Complex_Main
 begin
 
-nitpick_params [verbose, card = 1\<emdash>4, sat_solver = MiniSat_JNI, max_threads = 1,
+nitpick_params [verbose, card = 1\<emdash>4, sat_solver = Riss3g, max_threads = 1,
                 timeout = 240]
 
 definition "three = {0\<Colon>nat, 1, 2}"