src/Doc/Isar_Ref/Document_Preparation.thy
changeset 61472 6458760261ca
parent 61463 8e46cea6a45a
child 61473 34d1913f0b20
--- a/src/Doc/Isar_Ref/Document_Preparation.thy	Sun Oct 18 17:24:24 2015 +0200
+++ b/src/Doc/Isar_Ref/Document_Preparation.thy	Sun Oct 18 18:09:48 2015 +0200
@@ -129,15 +129,24 @@
   antiquotations are checked within the current theory or proof
   context.
 
+  \<^medskip>
+  Antiquotations are in general written @{verbatim "@{"}@{text "name
+  [options] arguments"}@{verbatim "}"}. The short form @{verbatim
+  "\<^control>"}@{text "\<open>argument\<close>"} (without surrounding @{verbatim
+  "@{"}@{text "\<dots>"}@{verbatim "}"}) works where the name is a single control
+  symbol and the argument a single cartouche.
+
   @{rail \<open>
     @@{command print_antiquotations} ('!'?)
+    ;
+    @{syntax_def antiquotation}:
+      '@{' antiquotation_body '}' |
+      @{syntax_ref control_symbol} @{syntax_ref cartouche}
   \<close>}
 
   %% FIXME less monolithic presentation, move to individual sections!?
   @{rail \<open>
-    '@{' antiquotation '}'
-    ;
-    @{syntax_def antiquotation}:
+    @{syntax_def antiquotation_body}:
       @@{antiquotation theory} options @{syntax name} |
       @@{antiquotation thm} options styles @{syntax thmrefs} |
       @@{antiquotation lemma} options @{syntax prop} @'by' @{syntax method} @{syntax method}? |