src/HOL/Nitpick_Examples/Datatype_Nits.thy
changeset 35078 6fd1052fe463
parent 35076 cc19e2aef17e
child 35284 9edc2bd6d2bd
--- a/src/HOL/Nitpick_Examples/Datatype_Nits.thy	Tue Feb 09 16:05:49 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Datatype_Nits.thy	Tue Feb 09 16:07:51 2010 +0100
@@ -11,7 +11,7 @@
 imports Main
 begin
 
-nitpick_params [sat_solver = MiniSatJNI, max_threads = 1, timeout = 60 s]
+nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60 s]
 
 primrec rot where
 "rot Nibble0 = Nibble1" | "rot Nibble1 = Nibble2" | "rot Nibble2 = Nibble3" |