src/HOL/TPTP/ATP_Theory_Export.thy
changeset 48129 933d43c31689
parent 46435 e9c90516bc0d
child 48141 1b864c4a3306
equal deleted inserted replaced
48128:bf172a5929bb 48129:933d43c31689
    21 *}
    21 *}
    22 
    22 
    23 ML {*
    23 ML {*
    24 if do_it then
    24 if do_it then
    25   "/tmp/axs_mono_native.dfg"
    25   "/tmp/axs_mono_native.dfg"
    26   |> generate_tptp_inference_file_for_theory ctxt thy (DFG DFG_Sorted)
    26   |> generate_tptp_inference_file_for_theory ctxt thy DFG "mono_native"
    27          "mono_native"
       
    28 else
    27 else
    29   ()
    28   ()
    30 *}
    29 *}
    31 
    30 
    32 ML {*
    31 ML {*