src/HOL/Nitpick_Examples/Typedef_Nits.thy
changeset 40341 03156257040f
parent 39362 ee65900bfced
child 40590 b994d855dbd2
--- a/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Wed Nov 03 20:19:24 2010 +0100
+++ b/src/HOL/Nitpick_Examples/Typedef_Nits.thy	Wed Nov 03 22:26:53 2010 +0100
@@ -12,7 +12,7 @@
 begin
 
 nitpick_params [card = 1\<midarrow>4, sat_solver = MiniSat_JNI, max_threads = 1,
-                timeout = 60 s]
+                timeout = 60]
 
 typedef three = "{0\<Colon>nat, 1, 2}"
 by blast