src/HOL/ex/Mirabelle/Mirabelle.thy
changeset 32383 521065a499c6
parent 32382 98674ac811c4
child 32384 8629581acc0b
--- a/src/HOL/ex/Mirabelle/Mirabelle.thy	Fri Aug 21 09:44:55 2009 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,12 +0,0 @@
-(* Title: Mirabelle.thy
-   Author: Jasmin Blanchette and Sascha Boehme
-*)
-
-theory Mirabelle
-imports Plain
-uses "Tools/mirabelle.ML"
-begin
-
-setup Mirabelle.setup
-
-end