src/HOL/Sledgehammer.thy
changeset 56126 fc937e7ef4c6
parent 56081 72fad75baf7e
child 56128 c106ac2ff76d
equal deleted inserted replaced
56125:e03c0f6ad1b6 56126:fc937e7ef4c6
    32 ML_file "Tools/Sledgehammer/sledgehammer_mepo.ML"
    32 ML_file "Tools/Sledgehammer/sledgehammer_mepo.ML"
    33 ML_file "Tools/Sledgehammer/sledgehammer_mash.ML"
    33 ML_file "Tools/Sledgehammer/sledgehammer_mash.ML"
    34 ML_file "Tools/Sledgehammer/sledgehammer.ML"
    34 ML_file "Tools/Sledgehammer/sledgehammer.ML"
    35 ML_file "Tools/Sledgehammer/sledgehammer_commands.ML"
    35 ML_file "Tools/Sledgehammer/sledgehammer_commands.ML"
    36 
    36 
       
    37 definition plus1 where "plus1 x = x + (1::int)"
       
    38 
       
    39 ML {* print_depth 1000 *}
       
    40 
       
    41 lemma "map plus1 [0] = [1]"
       
    42 sledgehammer [z3_new, isar_proofs = true, mepo, debug, dont_preplay, dont_minimize, dont_try0_isar]
       
    43 (add: plus1_def)
       
    44 oops
       
    45 
    37 end
    46 end