| author | wenzelm |
| Sun, 07 Nov 2010 23:32:26 +0100 | |
| changeset 40405 | 42671298f037 |
| parent 39155 | 3e94ebe282f1 |
| child 41358 | d5e91925916e |
| permissions | -rw-r--r-- |
(* Title: HOL/Mirabelle/Mirabelle.thy Author: Jasmin Blanchette and Sascha Boehme, TU Munich *) theory Mirabelle imports Pure uses "Tools/mirabelle.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 *} setup Mirabelle.setup ML {* signature MIRABELLE_ACTION = sig val invoke : (string * string) list -> theory -> theory end *} end