src/HOL/TPTP/ATP_Export.thy
author wenzelm
Sat, 13 Aug 2011 15:59:26 +0200
changeset 44182 ecb51b457064
parent 43804 eb9be23db2b7
child 44402 f0bc74b9161e
permissions -rw-r--r--
clarified node header -- exclude master_dir;

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_heavy"
      "/tmp/infs_poly_tags_heavy.tptp"
else
  ()
*}

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

end