| author | wenzelm | 
| Sat, 30 May 2015 23:30:54 +0200 | |
| changeset 60318 | ab785001b51d | 
| parent 59574 | de392405a851 | 
| child 63167 | 0909deb8059b | 
| 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 | ||
| 32385 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
changeset | 12 | ML {* Toplevel.add_hook Mirabelle.step_hook *}
 | 
| 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
changeset | 13 | |
| 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
changeset | 14 | ML {*
 | 
| 
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 | 
| 32385 
594890623c46
split actions from Mirabelle core (Mirabelle may thus be applied to basic theories in HOL)
 boehmes parents: 
32383diff
changeset | 19 | *} | 
| 
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 |