src/HOL/ex/ATP_Export.thy
author blanchet
Tue, 07 Jun 2011 07:04:53 +0200
changeset 43223 c9e87dc92d9e
parent 43110 src/HOL/ex/TPTP_Export.thy@99bf2b38d3ef
child 43400 3d03f4472883
permissions -rw-r--r--
renamed example theory to "ATP_Export", for consistency with its underlying "ATP_" modules

theory ATP_Export
imports Complex_Main
uses "atp_export.ML"
begin

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

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

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

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

end