diff -r 3a86194d1534 -r 7ce0ed8dc4d6 src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy --- a/src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy Thu Sep 16 13:49:06 2010 +0200 +++ b/src/HOL/Predicate_Compile_Examples/Code_Prolog_Examples.thy Thu Sep 16 13:49:08 2010 +0200 @@ -15,9 +15,7 @@ limited_types = [], limited_predicates = [], replacing = [], - manual_reorder = [], - timeout = Time.fromSeconds 10, - prolog_system = Code_Prolog.SWI_PROLOG}) *} + manual_reorder = []}) *} values "{(x, y, z). append x y z}" @@ -28,9 +26,7 @@ limited_types = [], limited_predicates = [], replacing = [], - manual_reorder = [], - timeout = Time.fromSeconds 10, - prolog_system = Code_Prolog.YAP}) *} + manual_reorder = []}) *} values "{(x, y, z). append x y z}" @@ -39,9 +35,7 @@ limited_types = [], limited_predicates = [], replacing = [], - manual_reorder = [], - timeout = Time.fromSeconds 10, - prolog_system = Code_Prolog.SWI_PROLOG}) *} + manual_reorder = []}) *} section {* Example queens *} @@ -209,9 +203,7 @@ limited_types = [], limited_predicates = [], replacing = [], - manual_reorder = [], - timeout = Time.fromSeconds 10, - prolog_system = Code_Prolog.SWI_PROLOG}) *} + manual_reorder = []}) *} values 2 "{y. notB y}"