src/HOL/TPTP/ATP_Problem_Import.thy
author blanchet
Wed, 25 Apr 2012 22:00:33 +0200
changeset 47766 9f7cdd5fff7c
parent 47765 18f37b7aa6a6
child 47770 53e30966b4b6
permissions -rw-r--r--
more work on TPTP Isabelle and Sledgehammer tactics

(*  Title:      HOL/TPTP/ATP_Problem_Import.thy
    Author:     Jasmin Blanchette, TU Muenchen
*)

header {* ATP Problem Importer *}

theory ATP_Problem_Import
imports Complex_Main TPTP_Interpret
uses "~~/src/HOL/ex/sledgehammer_tactics.ML"
     ("atp_problem_import.ML")
begin

ML {* Proofterm.proofs := 0 *}

declare [[show_consts]] (* for Refute *)
declare [[smt_oracle]]

use "atp_problem_import.ML"

end