src/HOL/Predicate_Compile_Examples/Hotel_Example.thy
changeset 38963 b5d126d7be4b
parent 38954 80ce658600b0
child 39189 d183bf90dabd
child 39198 f967a16dfcdd
--- a/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Tue Aug 31 15:07:51 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Hotel_Example.thy	Tue Aug 31 15:21:56 2010 +0200
@@ -89,6 +89,7 @@
   limited_types = [],
   limited_predicates = [],
   replacing = [],
+  manual_reorder = [],
   prolog_system = Code_Prolog.SWI_PROLOG}) *}
 
 values 40 "{s. hotel s}"
@@ -115,8 +116,9 @@
 setup {* Code_Prolog.map_code_options (K 
   {ensure_groundness = true,
    limited_types = [],
-   limited_predicates = [("hotel", 5)],
+   limited_predicates = [(["hotel"], 5)],
    replacing = [(("hotel", "limited_hotel"), "quickcheck")],
+   manual_reorder = [],
    prolog_system = Code_Prolog.SWI_PROLOG}) *}
 
 lemma