| author | wenzelm |
| Wed, 04 Nov 2015 23:27:00 +0100 | |
| changeset 61578 | 6623c81cb15a |
| parent 59574 | de392405a851 |
| child 63167 | 0909deb8059b |
| permissions | -rw-r--r-- |
(* Title: HOL/Mirabelle/Mirabelle.thy Author: Jasmin Blanchette and Sascha Boehme, TU Munich *) theory Mirabelle imports Main begin ML_file "Tools/mirabelle.ML" ML_file "../TPTP/sledgehammer_tactics.ML" ML {* Toplevel.add_hook Mirabelle.step_hook *} ML {* signature MIRABELLE_ACTION = sig val invoke : (string * string) list -> theory -> theory end *} end