src/HOL/TPTP/TPTP_Proof_Reconstruction.thy
changeset 69605 a96320074298
parent 69597 ff784d5a5bfb
child 74282 c2ee8d993d6a
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
    73 declare [[
    73 declare [[
    74   tptp_unexceptional_reconstruction = false, (*NOTE should be "false" while testing*)
    74   tptp_unexceptional_reconstruction = false, (*NOTE should be "false" while testing*)
    75   tptp_informative_failure = true
    75   tptp_informative_failure = true
    76 ]]
    76 ]]
    77 
    77 
    78 ML_file "TPTP_Parser/tptp_reconstruct_library.ML"
    78 ML_file \<open>TPTP_Parser/tptp_reconstruct_library.ML\<close>
    79 ML "open TPTP_Reconstruct_Library"
    79 ML "open TPTP_Reconstruct_Library"
    80 ML_file "TPTP_Parser/tptp_reconstruct.ML"
    80 ML_file \<open>TPTP_Parser/tptp_reconstruct.ML\<close>
    81 
    81 
    82 (*FIXME fudge*)
    82 (*FIXME fudge*)
    83 declare [[
    83 declare [[
    84   blast_depth_limit = 10,
    84   blast_depth_limit = 10,
    85   unify_search_bound = 5
    85   unify_search_bound = 5