doc-src/IsarImplementation/Thy/Base.thy
changeset 48891 c0eafbd55de3
parent 43564 9864182c6bad
--- a/doc-src/IsarImplementation/Thy/Base.thy	Wed Aug 22 22:47:16 2012 +0200
+++ b/doc-src/IsarImplementation/Thy/Base.thy	Wed Aug 22 22:55:41 2012 +0200
@@ -1,8 +1,8 @@
 theory Base
 imports Main
-uses "../../antiquote_setup.ML"
 begin
 
+ML_file "../../antiquote_setup.ML"
 setup {* Antiquote_Setup.setup *}
 
 end