src/Doc/Isar_Ref/Document_Preparation.thy
changeset 62969 9f394a16c557
parent 62965 5bf08c9aa036
child 63120 629a4c5e953e
equal deleted inserted replaced
62968:4e4738698db4 62969:9f394a16c557
   165   @{rail \<open>
   165   @{rail \<open>
   166     @{syntax_def antiquotation_body}:
   166     @{syntax_def antiquotation_body}:
   167       (@@{antiquotation text} | @@{antiquotation cartouche} | @@{antiquotation theory_text})
   167       (@@{antiquotation text} | @@{antiquotation cartouche} | @@{antiquotation theory_text})
   168         options @{syntax text} |
   168         options @{syntax text} |
   169       @@{antiquotation theory} options @{syntax name} |
   169       @@{antiquotation theory} options @{syntax name} |
   170       @@{antiquotation thm} options styles @{syntax thmrefs} |
   170       @@{antiquotation thm} options styles @{syntax thms} |
   171       @@{antiquotation lemma} options @{syntax prop} @'by' @{syntax method} @{syntax method}? |
   171       @@{antiquotation lemma} options @{syntax prop} @'by' @{syntax method} @{syntax method}? |
   172       @@{antiquotation prop} options styles @{syntax prop} |
   172       @@{antiquotation prop} options styles @{syntax prop} |
   173       @@{antiquotation term} options styles @{syntax term} |
   173       @@{antiquotation term} options styles @{syntax term} |
   174       @@{antiquotation (HOL) value} options styles @{syntax term} |
   174       @@{antiquotation (HOL) value} options styles @{syntax term} |
   175       @@{antiquotation term_type} options styles @{syntax term} |
   175       @@{antiquotation term_type} options styles @{syntax term} |
   183         options @{syntax name}
   183         options @{syntax name}
   184     ;
   184     ;
   185     @{syntax antiquotation}:
   185     @{syntax antiquotation}:
   186       @@{antiquotation goals} options |
   186       @@{antiquotation goals} options |
   187       @@{antiquotation subgoals} options |
   187       @@{antiquotation subgoals} options |
   188       @@{antiquotation prf} options @{syntax thmrefs} |
   188       @@{antiquotation prf} options @{syntax thms} |
   189       @@{antiquotation full_prf} options @{syntax thmrefs} |
   189       @@{antiquotation full_prf} options @{syntax thms} |
   190       @@{antiquotation ML} options @{syntax text} |
   190       @@{antiquotation ML} options @{syntax text} |
   191       @@{antiquotation ML_op} options @{syntax text} |
   191       @@{antiquotation ML_op} options @{syntax text} |
   192       @@{antiquotation ML_type} options @{syntax text} |
   192       @@{antiquotation ML_type} options @{syntax text} |
   193       @@{antiquotation ML_structure} options @{syntax text} |
   193       @@{antiquotation ML_structure} options @{syntax text} |
   194       @@{antiquotation ML_functor} options @{syntax text} |
   194       @@{antiquotation ML_functor} options @{syntax text} |
   195       @@{antiquotation emph} options @{syntax text} |
   195       @@{antiquotation emph} options @{syntax text} |
   196       @@{antiquotation bold} options @{syntax text} |
   196       @@{antiquotation bold} options @{syntax text} |
   197       @@{antiquotation verbatim} options @{syntax text} |
   197       @@{antiquotation verbatim} options @{syntax text} |
   198       @@{antiquotation "file"} options @{syntax xname} |
   198       @@{antiquotation "file"} options @{syntax name} |
   199       @@{antiquotation file_unchecked} options @{syntax xname} |
   199       @@{antiquotation file_unchecked} options @{syntax name} |
   200       @@{antiquotation url} options @{syntax name} |
   200       @@{antiquotation url} options @{syntax name} |
   201       @@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and')
   201       @@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and')
   202     ;
   202     ;
   203     styles: '(' (style + ',') ')'
   203     styles: '(' (style + ',') ')'
   204     ;
   204     ;
   611   \begin{matharray}{rcl}
   611   \begin{matharray}{rcl}
   612     @{command_def "display_drafts"}\<open>\<^sup>*\<close> & : & \<open>any \<rightarrow>\<close> \\
   612     @{command_def "display_drafts"}\<open>\<^sup>*\<close> & : & \<open>any \<rightarrow>\<close> \\
   613   \end{matharray}
   613   \end{matharray}
   614 
   614 
   615   @{rail \<open>
   615   @{rail \<open>
   616     @@{command display_drafts} (@{syntax xname} +)
   616     @@{command display_drafts} (@{syntax name} +)
   617   \<close>}
   617   \<close>}
   618 
   618 
   619   \<^descr> @{command "display_drafts"}~\<open>paths\<close> performs simple output of a given list
   619   \<^descr> @{command "display_drafts"}~\<open>paths\<close> performs simple output of a given list
   620   of raw source files. Only those symbols that do not require additional
   620   of raw source files. Only those symbols that do not require additional
   621   {\LaTeX} packages are displayed properly, everything else is left verbatim.
   621   {\LaTeX} packages are displayed properly, everything else is left verbatim.