author | wenzelm |
Sun, 31 Jul 2016 17:25:38 +0200 | |
changeset 63569 | 7e0b0db5e9ac |
parent 63167 | 0909deb8059b |
child 69605 | a96320074298 |
permissions | -rw-r--r-- |
32564 | 1 |
(* Title: HOL/Mirabelle/Mirabelle.thy |
2 |
Author: Jasmin Blanchette and Sascha Boehme, TU Munich |
|
32381 | 3 |
*) |
4 |
||
5 |
theory Mirabelle |
|
59574 | 6 |
imports Main |
32381 | 7 |
begin |
8 |
||
48891 | 9 |
ML_file "Tools/mirabelle.ML" |
10 |
ML_file "../TPTP/sledgehammer_tactics.ML" |
|
11 |
||
63167 | 12 |
ML \<open>Toplevel.add_hook Mirabelle.step_hook\<close> |
32385
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
boehmes
parents:
32383
diff
changeset
|
13 |
|
63167 | 14 |
ML \<open> |
32385
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
boehmes
parents:
32383
diff
changeset
|
15 |
signature MIRABELLE_ACTION = |
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
boehmes
parents:
32383
diff
changeset
|
16 |
sig |
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
boehmes
parents:
32383
diff
changeset
|
17 |
val invoke : (string * string) list -> theory -> theory |
32381 | 18 |
end |
63167 | 19 |
\<close> |
32385
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
boehmes
parents:
32383
diff
changeset
|
20 |
|
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
boehmes
parents:
32383
diff
changeset
|
21 |
end |