| author | haftmann | 
| Sat, 24 Dec 2011 16:14:58 +0100 | |
| changeset 45982 | 989b1eede03c | 
| parent 42616 | 92715b528e78 | 
| child 47477 | 3fabf352243e | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Mirabelle/Mirabelle.thy Author: Jasmin Blanchette and Sascha Boehme, TU Munich *) theory Mirabelle imports Sledgehammer uses "Tools/mirabelle.ML" "../ex/sledgehammer_tactics.ML" begin (* no multithreading, no parallel proofs *) (* FIXME *) ML {* Multithreading.max_threads := 1 *} ML {* Goal.parallel_proofs := 0 *} ML {* Toplevel.add_hook Mirabelle.step_hook *} ML {* signature MIRABELLE_ACTION = sig val invoke : (string * string) list -> theory -> theory end *} end