src/Doc/Isar_Ref/Document_Preparation.thy
changeset 59917 9830c944670f
parent 59783 00b62aa9f430
child 59937 6eccb133d4e6
--- a/src/Doc/Isar_Ref/Document_Preparation.thy	Fri Apr 03 18:36:19 2015 +0200
+++ b/src/Doc/Isar_Ref/Document_Preparation.thy	Fri Apr 03 19:56:51 2015 +0200
@@ -85,6 +85,7 @@
 
 text \<open>
   \begin{matharray}{rcl}
+    @{command_def "print_antiquotations"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow> "} \\
     @{antiquotation_def "theory"} & : & @{text antiquotation} \\
     @{antiquotation_def "thm"} & : & @{text antiquotation} \\
     @{antiquotation_def "lemma"} & : & @{text antiquotation} \\
@@ -132,6 +133,10 @@
   antiquotations are checked within the current theory or proof
   context.
 
+  @{rail \<open>
+    @@{command print_antiquotations} ('!'?)
+  \<close>}
+
   %% FIXME less monolithic presentation, move to individual sections!?
   @{rail \<open>
     '@{' antiquotation '}'
@@ -182,7 +187,11 @@
   text @{verbatim "{*"}~@{text "\<dots>"}~@{verbatim "*}"}.
 
   \begin{description}
-  
+
+  \item @{command "print_antiquotations"} prints all document antiquotations
+  that are defined in the current context; the ``@{text "!"}'' option
+  indicates extra verbosity.
+
   \item @{text "@{theory A}"} prints the name @{text "A"}, which is
   guaranteed to refer to a valid ancestor theory in the current
   context.