src/Pure/Pure.thy
changeset 67386 998e01d6f8fd
parent 67283 0493be7f2d9b
child 67446 1f4d167b6ac9
--- a/src/Pure/Pure.thy	Tue Jan 09 15:18:41 2018 +0100
+++ b/src/Pure/Pure.thy	Tue Jan 09 15:40:12 2018 +0100
@@ -1145,7 +1145,7 @@
   Outer_Syntax.command \<^command_keyword>\<open>print_antiquotations\<close>
     "print document antiquotations"
     (Parse.opt_bang >> (fn b =>
-      Toplevel.keep (Thy_Output.print_antiquotations b o Toplevel.context_of)));
+      Toplevel.keep (Document_Antiquotation.print_antiquotations b o Toplevel.context_of)));
 
 val _ =
   Outer_Syntax.command \<^command_keyword>\<open>print_ML_antiquotations\<close>