src/HOL/Predicate_Compile_Examples/Lambda_Example.thy
changeset 39800 17e29ddd538e
parent 39463 7ce0ed8dc4d6
child 40924 a9be7f26b4e6
--- a/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy	Thu Sep 30 10:48:12 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Lambda_Example.thy	Thu Sep 30 10:48:12 2010 +0200
@@ -83,6 +83,7 @@
 
 setup {* Code_Prolog.map_code_options (K 
   { ensure_groundness = true,
+    limit_globally = NONE,
     limited_types = [(@{typ nat}, 1), (@{typ "type"}, 1), (@{typ dB}, 1), (@{typ "type list"}, 1)],
     limited_predicates = [(["typing"], 2), (["nthel1"], 2)],
     replacing = [(("typing", "limited_typing"), "quickcheck"),