src/HOL/TPTP/ATP_Problem_Import.thy
author huffman
Sat, 21 Apr 2012 10:59:52 +0200
changeset 47647 ec29cc09599d
parent 47557 32f35b3d9e42
child 47670 24babc4b1925
permissions -rw-r--r--
renamed contravariant relator set_rel to vset_rel, to make room for new covariant relator

(*  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 ("atp_problem_import.ML")
begin

typedecl iota (* for TPTP *)

use "atp_problem_import.ML"

end