src/HOL/ATP_Linkup.thy
changeset 27368 9f90ac19e32b
parent 27182 9e4475b9d58c
child 28290 4cc2b6046258
equal deleted inserted replaced
27367:a75d71c73362 27368:9f90ac19e32b
     5 *)
     5 *)
     6 
     6 
     7 header{* The Isabelle-ATP Linkup *}
     7 header{* The Isabelle-ATP Linkup *}
     8 
     8 
     9 theory ATP_Linkup
     9 theory ATP_Linkup
    10 imports Record Presburger SAT Recdef Extraction Relation_Power Hilbert_Choice
    10 imports Record Hilbert_Choice
    11 uses
    11 uses
    12   "Tools/polyhash.ML"
    12   "Tools/polyhash.ML"
    13   "Tools/res_clause.ML"
    13   "Tools/res_clause.ML"
    14   ("Tools/res_hol_clause.ML")
    14   ("Tools/res_hol_clause.ML")
    15   ("Tools/res_axioms.ML")
    15   ("Tools/res_axioms.ML")
    86 apply (rule eq_reflection)
    86 apply (rule eq_reflection)
    87 apply (rule ext) 
    87 apply (rule ext) 
    88 apply (simp add: COMBC_def) 
    88 apply (simp add: COMBC_def) 
    89 done
    89 done
    90 
    90 
       
    91 
       
    92 subsection {* Setup of Vampire, E prover and SPASS *}
       
    93 
    91 use "Tools/res_axioms.ML"      --{*requires the combinators declared above*}
    94 use "Tools/res_axioms.ML"      --{*requires the combinators declared above*}
    92 setup ResAxioms.setup
    95 setup ResAxioms.setup
    93 
    96 
    94 use "Tools/res_hol_clause.ML"
    97 use "Tools/res_hol_clause.ML"
    95 use "Tools/res_reconstruct.ML"
    98 use "Tools/res_reconstruct.ML"
    96 use "Tools/watcher.ML"
    99 use "Tools/watcher.ML"
    97 use "Tools/res_atp.ML"
   100 use "Tools/res_atp.ML"
    98 
       
    99 
       
   100 subsection {* Setup for Vampire, E prover and SPASS *}
       
   101 
   101 
   102 use "Tools/res_atp_provers.ML"
   102 use "Tools/res_atp_provers.ML"
   103 
   103 
   104 oracle vampire_oracle ("string * int") = {* ResAtpProvers.vampire_o *}
   104 oracle vampire_oracle ("string * int") = {* ResAtpProvers.vampire_o *}
   105 oracle eprover_oracle ("string * int") = {* ResAtpProvers.eprover_o *}
   105 oracle eprover_oracle ("string * int") = {* ResAtpProvers.eprover_o *}