src/HOL/TPTP/ATP_Export.thy
author blanchet
Fri, 26 Aug 2011 10:12:17 +0200
changeset 44508 5438d88b2cb7
parent 44402 f0bc74b9161e
child 45305 3e09961326ce
permissions -rw-r--r--
comment

theory ATP_Export
imports Complex_Main
uses "atp_export.ML"
begin

ML {*
val do_it = false; (* switch to "true" to generate the files *)
val thy = @{theory Complex_Main};
val ctxt = @{context}
*}

ML {*
if do_it then
  ATP_Export.generate_tptp_inference_file_for_theory ctxt thy "poly_preds"
      "/tmp/infs_poly_preds.tptp"
else
  ()
*}

ML {*
if do_it then
  ATP_Export.generate_tptp_inference_file_for_theory ctxt thy "poly_tags"
      "/tmp/infs_poly_tags.tptp"
else
  ()
*}

ML {*
if do_it then
  ATP_Export.generate_tptp_inference_file_for_theory ctxt thy "poly_tags_uniform"
      "/tmp/infs_poly_tags_uniform.tptp"
else
  ()
*}

ML {*
if do_it then
  ATP_Export.generate_tptp_graph_file_for_theory ctxt thy
      "/tmp/graph.out"
else
  ()
*}

end