src/Doc/JEdit/Base.thy
changeset 53769 036e80175bdd
child 54354 4e6defdc24ac
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Doc/JEdit/Base.thy	Sat Sep 21 13:05:54 2013 +0200
@@ -0,0 +1,8 @@
+theory Base
+imports Pure
+begin
+
+ML_file "../antiquote_setup.ML"
+setup Antiquote_Setup.setup
+
+end