src/HOL/Predicate_Compile_Examples/Lambda_Example.thy
changeset 38958 08eb0ffa2413
parent 38950 62578950e748
child 38963 b5d126d7be4b
--- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy	Tue Aug 31 10:51:49 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy	Tue Aug 31 11:49:15 2010 +0200
@@ -84,9 +84,9 @@
 setup {* Code_Prolog.map_code_options (K 
   { ensure_groundness = true,
     limited_types = [(@{typ nat}, 1), (@{typ "type"}, 1), (@{typ dB}, 1), (@{typ "type list"}, 1)],
-    limited_predicates = [("typing", 2), ("nth_el1", 2)],
+    limited_predicates = [("typing", 2), ("nthel1", 2)],
     replacing = [(("typing", "limited_typing"), "quickcheck"),
-                 (("nth_el1", "limited_nth_el1"), "lim_typing")],
+                 (("nthel1", "limited_nthel1"), "lim_typing")],
     prolog_system = Code_Prolog.SWI_PROLOG}) *}
 
 lemma