src/Doc/IsarRef/Outer_Syntax.thy
changeset 50213 7b73c0509835
parent 48985 5386df44a037
child 51058 98c48d023136
equal deleted inserted replaced
50212:4fb06c22c5ec 50213:7b73c0509835
    60     (in conjunction with @{verbatim "-l ZF"}, to specify the default
    60     (in conjunction with @{verbatim "-l ZF"}, to specify the default
    61     logic image).  Note that option @{verbatim "-L"} does both
    61     logic image).  Note that option @{verbatim "-L"} does both
    62     of this at the same time.
    62     of this at the same time.
    63   \end{warn}
    63   \end{warn}
    64 *}
    64 *}
       
    65 
       
    66 
       
    67 section {* Commands *}
       
    68 
       
    69 text {*
       
    70   \begin{matharray}{rcl}
       
    71     @{command_def "print_commands"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
       
    72     @{command_def "help"}@{text "\<^sup>*"} & : & @{text "any \<rightarrow>"} \\
       
    73   \end{matharray}
       
    74 
       
    75   @{rail "
       
    76     @@{command help} (@{syntax name} * )
       
    77   "}
       
    78 
       
    79   \begin{description}
       
    80 
       
    81   \item @{command "print_commands"} prints all outer syntax keywords
       
    82   and commands.
       
    83 
       
    84   \item @{command "help"}~@{text "pats"} retrieves outer syntax
       
    85   commands according to the specified name patterns.
       
    86 
       
    87   \end{description}
       
    88 *}
       
    89 
       
    90 
       
    91 subsubsection {* Examples *}
       
    92 
       
    93 text {* Some common diagnostic commands are retrieved like this
       
    94   (according to usual naming conventions): *}
       
    95 
       
    96 help "print"
       
    97 help "find"
    65 
    98 
    66 
    99 
    67 section {* Lexical matters \label{sec:outer-lex} *}
   100 section {* Lexical matters \label{sec:outer-lex} *}
    68 
   101 
    69 text {* The outer lexical syntax consists of three main categories of
   102 text {* The outer lexical syntax consists of three main categories of