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