src/Doc/System/Base.thy
changeset 48985 5386df44a037
parent 48937 e7418f8d49fe
child 56059 2390391584c2
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Doc/System/Base.thy	Tue Aug 28 18:57:32 2012 +0200
@@ -0,0 +1,8 @@
+theory Base
+imports Pure
+begin
+
+ML_file "../antiquote_setup.ML"
+setup Antiquote_Setup.setup
+
+end