changeset 32381 | 11542bebe4d4 |
child 32382 | 98674ac811c4 |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/ex/Mirabelle/Mirabelle.thy Mon Aug 17 10:59:12 2009 +0200 @@ -0,0 +1,14 @@ +(* Title: Mirabelle.thy + Author: Jasmin Blanchette and Sascha Boehme +*) + +theory Mirabelle +imports Main +uses "mirabelle.ML" +begin + +(* FIXME: use a logfile for each theory file *) + +setup Mirabelle.setup + +end