author | urbanc |
Wed, 01 Mar 2006 18:24:31 +0100 | |
changeset 19168 | c8faffc8e6fb |
parent 18201 | 6c63f0eb16d7 |
child 19193 | 45c8db82893d |
permissions | -rw-r--r-- |
17905
1574533861b1
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
mengj
parents:
diff
changeset
|
1 |
(* ID: $Id$ |
17907 | 2 |
Author: Jia Meng, NICTA |
17905
1574533861b1
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
mengj
parents:
diff
changeset
|
3 |
*) |
1574533861b1
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
mengj
parents:
diff
changeset
|
4 |
|
17958 | 5 |
header {* ATP setup (Vampire and E prover) *} |
17905
1574533861b1
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
mengj
parents:
diff
changeset
|
6 |
|
17958 | 7 |
theory ResAtpMethods |
8 |
imports Reconstruction |
|
9 |
uses |
|
10 |
"Tools/res_atp_setup.ML" |
|
11 |
"Tools/res_atp_provers.ML" |
|
12 |
("Tools/res_atp_methods.ML") |
|
17905
1574533861b1
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
mengj
parents:
diff
changeset
|
13 |
|
1574533861b1
Added files in order to use external ATPs as oracles and invoke these ATPs by calling Isabelle methods (currently "vampire" and "eprover").
mengj
parents:
diff
changeset
|
14 |
begin |
17939
3925ab7b8a18
Merged theory ResAtpOracle.thy into ResAtpMethods.thy
mengj
parents:
17907
diff
changeset
|
15 |
|
18201
6c63f0eb16d7
-- changed the interface of functions vampire_oracle and eprover_oracle.
mengj
parents:
17958
diff
changeset
|
16 |
oracle vampire_oracle ("(string list * string list) * int") = {* ResAtpProvers.vampire_o *} |
6c63f0eb16d7
-- changed the interface of functions vampire_oracle and eprover_oracle.
mengj
parents:
17958
diff
changeset
|
17 |
oracle eprover_oracle ("(string list * string list) * int") = {* ResAtpProvers.eprover_o *} |
17939
3925ab7b8a18
Merged theory ResAtpOracle.thy into ResAtpMethods.thy
mengj
parents:
17907
diff
changeset
|
18 |
|
17958 | 19 |
use "Tools/res_atp_methods.ML" |
20 |
setup ResAtpMethods.ResAtps_setup |
|
17939
3925ab7b8a18
Merged theory ResAtpOracle.thy into ResAtpMethods.thy
mengj
parents:
17907
diff
changeset
|
21 |
|
17907 | 22 |
end |