diff -r 3a86194d1534 -r 7ce0ed8dc4d6 src/HOL/Predicate_Compile_Examples/Lambda_Example.thy --- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Thu Sep 16 13:49:06 2010 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy Thu Sep 16 13:49:08 2010 +0200 @@ -79,7 +79,7 @@ section {* Manual setup to find counterexample *} -setup {* Quickcheck.add_generator ("prolog", Code_Prolog.quickcheck) *} +setup {* Context.theory_map (Quickcheck.add_generator ("prolog", Code_Prolog.quickcheck)) *} setup {* Code_Prolog.map_code_options (K { ensure_groundness = true, @@ -87,9 +87,7 @@ limited_predicates = [(["typing"], 2), (["nthel1"], 2)], replacing = [(("typing", "limited_typing"), "quickcheck"), (("nthel1", "limited_nthel1"), "lim_typing")], - manual_reorder = [], - timeout = Time.fromSeconds 10, - prolog_system = Code_Prolog.SWI_PROLOG}) *} + manual_reorder = []}) *} lemma "\ \ t : U \ t \\<^sub>\ t' \ \ \ t' : U"