src/HOL/Predicate_Compile_Examples/Lambda_Example.thy
changeset 43937 768c70befd59
parent 41956 c15ef1b85035
child 52666 391913d17d15
equal deleted inserted replaced
43936:127749bbc639 43937:768c70befd59
    77 lemma [code_pred_inline]: "(x::nat) + 1 = Suc x"
    77 lemma [code_pred_inline]: "(x::nat) + 1 = Suc x"
    78 by simp
    78 by simp
    79 
    79 
    80 section {* Manual setup to find counterexample *}
    80 section {* Manual setup to find counterexample *}
    81 
    81 
    82 setup {* Context.theory_map (Quickcheck.add_generator ("prolog", Code_Prolog.quickcheck)) *}
    82 setup {* Context.theory_map (Quickcheck.add_tester ("prolog", (Code_Prolog.active, Code_Prolog.test_goals))) *}
    83 
    83 
    84 setup {* Code_Prolog.map_code_options (K 
    84 setup {* Code_Prolog.map_code_options (K 
    85   { ensure_groundness = true,
    85   { ensure_groundness = true,
    86     limit_globally = NONE,
    86     limit_globally = NONE,
    87     limited_types = [(@{typ nat}, 1), (@{typ "type"}, 1), (@{typ dB}, 1), (@{typ "type list"}, 1)],
    87     limited_types = [(@{typ nat}, 1), (@{typ "type"}, 1), (@{typ dB}, 1), (@{typ "type list"}, 1)],