src/HOL/TPTP/ATP_Problem_Import.thy
author blanchet
Fri, 27 Apr 2012 15:24:37 +0200
changeset 48661 2e1636e45770
parent 48659 44b33c1e702e
child 48665 4ad62c5f9f88
permissions -rw-r--r--
move file to where it belongs
     1 (*  Title:      HOL/TPTP/ATP_Problem_Import.thy
     2     Author:     Jasmin Blanchette, TU Muenchen
     3 *)
     4 
     5 header {* ATP Problem Importer *}
     6 theory ATP_Problem_Import
     7 imports Complex_Main TPTP_Interpret
     8 uses "sledgehammer_tactics.ML"
     9      "atp_problem_import.ML"
    10 begin
    11 
    12 ML {* Proofterm.proofs := 0 *}
    13 
    14 declare [[show_consts]] (* for Refute *)
    15 declare [[smt_oracle]]
    16 
    17 (*
    18 ML {* ATP_Problem_Import.isabelle_tptp_file 300 "$TPTP/Problems/PUZ/PUZ107^5.p" *}
    19 *)
    20 
    21 end