src/HOL/Nitpick_Examples/Special_Nits.thy
changeset 35284 9edc2bd6d2bd
parent 35075 6fd1052fe463
child 35312 99cd1f96b400
     1.1 --- a/src/HOL/Nitpick_Examples/Special_Nits.thy	Mon Feb 22 14:36:10 2010 +0100
     1.2 +++ b/src/HOL/Nitpick_Examples/Special_Nits.thy	Mon Feb 22 19:31:00 2010 +0100
     1.3 @@ -11,8 +11,8 @@
     1.4  imports Main
     1.5  begin
     1.6  
     1.7 -nitpick_params [sat_solver = MiniSat_JNI, max_threads = 1, timeout = 60 s,
     1.8 -                card = 4]
     1.9 +nitpick_params [card = 4, sat_solver = MiniSat_JNI, max_threads = 1,
    1.10 +                timeout = 60 s]
    1.11  
    1.12  fun f1 :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> nat" where
    1.13  "f1 a b c d e = a + b + c + d + e"