src/HOL/Nitpick_Examples/Record_Nits.thy
changeset 35075 6fd1052fe463
parent 35073 cc19e2aef17e
child 35284 9edc2bd6d2bd
     1.1 --- a/src/HOL/Nitpick_Examples/Record_Nits.thy	Tue Feb 09 16:05:49 2010 +0100
     1.2 +++ b/src/HOL/Nitpick_Examples/Record_Nits.thy	Tue Feb 09 16:07:51 2010 +0100
     1.3 @@ -11,7 +11,7 @@
     1.4  imports Main
     1.5  begin
     1.6  
     1.7 -nitpick_params [sat_solver = MiniSatJNI, max_threads = 1, timeout = 60 s]
     1.8 +nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60 s]
     1.9  
    1.10  record point2d =
    1.11    xc :: int