--- a/src/HOL/Nitpick_Examples/Typedef_Nits.thy Fri Apr 01 09:29:58 2011 +0200
+++ b/src/HOL/Nitpick_Examples/Typedef_Nits.thy Fri Apr 01 09:48:01 2011 +0200
@@ -159,7 +159,7 @@
by (rule Rep_Nat_inverse)
lemma "0 \<equiv> Abs_Integ (intrel `` {(0, 0)})"
-nitpick [card = 1, unary_ints, max_potential = 0, timeout = 120, expect = none]
+nitpick [card = 1, unary_ints, max_potential = 0, timeout = 240, expect = none]
by (rule Zero_int_def_raw)
lemma "Abs_list (Rep_list a) = a"
--- a/src/HOL/Predicate_Compile_Examples/Examples.thy Fri Apr 01 09:29:58 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Examples.thy Fri Apr 01 09:48:01 2011 +0200
@@ -2,6 +2,8 @@
imports Main "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs"
begin
+declare [[values_timeout = 240.0]]
+
section {* Formal Languages *}
subsection {* General Context Free Grammars *}
--- a/src/HOL/Predicate_Compile_Examples/Specialisation_Examples.thy Fri Apr 01 09:29:58 2011 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Specialisation_Examples.thy Fri Apr 01 09:48:01 2011 +0200
@@ -2,7 +2,7 @@
imports Main "~~/src/HOL/Library/Predicate_Compile_Alternative_Defs"
begin
-declare [[values_timeout = 240.0]]
+declare [[values_timeout = 480.0]]
section {* Specialisation Examples *}