src/Pure/Thy/document_antiquotation.ML
changeset 67571 f858fe5531ac
parent 67474 90def2b06305
child 68223 88dd06301dd3
--- a/src/Pure/Thy/document_antiquotation.ML	Sat Feb 03 15:34:22 2018 +0100
+++ b/src/Pure/Thy/document_antiquotation.ML	Sat Feb 03 20:34:26 2018 +0100
@@ -29,7 +29,8 @@
   val setup_option: binding -> (string -> Proof.context -> Proof.context) -> theory -> theory
   val boolean: string -> bool
   val integer: string -> int
-  val evaluate: Proof.context -> Antiquote.text_antiquote -> Latex.text list
+  val evaluate: (Symbol_Pos.T list -> Latex.text list) -> Proof.context ->
+    Antiquote.text_antiquote -> Latex.text list
 end;
 
 structure Document_Antiquotation: DOCUMENT_ANTIQUOTATION =
@@ -167,9 +168,9 @@
 
 in
 
-fun evaluate ctxt antiq =
+fun evaluate eval_text ctxt antiq =
   (case antiq of
-    Antiquote.Text ss => [Latex.symbols ss]
+    Antiquote.Text ss => eval_text ss
   | Antiquote.Control {name, body, ...} =>
       eval ctxt ([], Token.make_src name (if null body then [] else [Token.read_cartouche body]))
   | Antiquote.Antiq {range = (pos, _), body, ...} =>