src/Pure/Thy/thy_output.ML
changeset 50201 c26369c9eda6
parent 49847 ed5080c03165
child 50301 56b4c9afd7be
--- a/src/Pure/Thy/thy_output.ML	Sun Nov 25 18:50:13 2012 +0100
+++ b/src/Pure/Thy/thy_output.ML	Sun Nov 25 19:49:24 2012 +0100
@@ -83,8 +83,8 @@
     (Args.src -> Toplevel.state -> Proof.context -> string) Name_Space.table *
       (string -> Proof.context -> Proof.context) Name_Space.table;
   val empty : T =
-    (Name_Space.empty_table Isabelle_Markup.document_antiquotationN,
-      Name_Space.empty_table Isabelle_Markup.document_antiquotation_optionN);
+    (Name_Space.empty_table Markup.document_antiquotationN,
+      Name_Space.empty_table Markup.document_antiquotation_optionN);
   val extend = I;
   fun merge ((commands1, options1), (commands2, options2)) : T =
     (Name_Space.merge_tables (commands1, commands2),
@@ -205,7 +205,7 @@
 
 
 fun check_text (txt, pos) state =
- (Position.report pos Isabelle_Markup.doc_source;
+ (Position.report pos Markup.doc_source;
   ignore (eval_antiquote (#1 (Keyword.get_lexicons ())) state (txt, pos)));