src/HOL/Nitpick_Examples/Refute_Nits.thy
changeset 56006 86e0b402994c
parent 50849 b27bbb021df1
child 56022 93f6d33a754e
     1.1 --- a/src/HOL/Nitpick_Examples/Refute_Nits.thy	Thu Dec 05 13:22:00 2013 +0100
     1.2 +++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy	Thu Dec 05 13:38:20 2013 +0100
     1.3 @@ -12,7 +12,7 @@
     1.4  begin
     1.5  
     1.6  nitpick_params [verbose, card = 1\<emdash>6, max_potential = 0,
     1.7 -                sat_solver = MiniSat_JNI, max_threads = 1, timeout = 240]
     1.8 +                sat_solver = Riss3g, max_threads = 1, timeout = 240]
     1.9  
    1.10  lemma "P \<and> Q"
    1.11  apply (rule conjI)