src/HOL/Predicate_Compile_Examples/Lambda_Example.thy
changeset 69597 ff784d5a5bfb
parent 66453 cc19f7ca2ed6
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
    85 \<close>
    85 \<close>
    86 
    86 
    87 setup \<open>Code_Prolog.map_code_options (K 
    87 setup \<open>Code_Prolog.map_code_options (K 
    88   { ensure_groundness = true,
    88   { ensure_groundness = true,
    89     limit_globally = NONE,
    89     limit_globally = NONE,
    90     limited_types = [(@{typ nat}, 1), (@{typ "type"}, 1), (@{typ dB}, 1), (@{typ "type list"}, 1)],
    90     limited_types = [(\<^typ>\<open>nat\<close>, 1), (\<^typ>\<open>type\<close>, 1), (\<^typ>\<open>dB\<close>, 1), (\<^typ>\<open>type list\<close>, 1)],
    91     limited_predicates = [(["typing"], 2), (["nthel1"], 2)],
    91     limited_predicates = [(["typing"], 2), (["nthel1"], 2)],
    92     replacing = [(("typing", "limited_typing"), "quickcheck"),
    92     replacing = [(("typing", "limited_typing"), "quickcheck"),
    93                  (("nthel1", "limited_nthel1"), "lim_typing")],
    93                  (("nthel1", "limited_nthel1"), "lim_typing")],
    94     manual_reorder = []})\<close>
    94     manual_reorder = []})\<close>
    95 
    95