| author | Andreas Lochbihler <mail@andreas-lochbihler.de> | 
| Sun, 31 Jan 2021 12:10:20 +0100 | |
| changeset 73213 | bb35f7f60d6c | 
| parent 69605 | a96320074298 | 
| child 73684 | a63d76ba0a03 | 
| 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 | ||
| 69605 | 9 | ML_file \<open>Tools/mirabelle.ML\<close> | 
| 10 | ML_file \<open>../TPTP/sledgehammer_tactics.ML\<close> | |
| 48891 | 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: 
32383diff
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: 
32383diff
changeset | 15 | signature MIRABELLE_ACTION = | 
| 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
changeset | 16 | sig | 
| 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
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: 
32383diff
changeset | 20 | |
| 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
changeset | 21 | end |