doc-src/IsarRef/Thy/document/Proof.tex
changeset 40255 9ffbc25e1606
parent 37364 dfca6c4cd1e8
child 40406 313a24b66a8d
equal deleted inserted replaced
40254:6d1ebaa7a4ba 40255:9ffbc25e1606
   451   contexts of (essentially a big disjunction of eliminated parameters
   451   contexts of (essentially a big disjunction of eliminated parameters
   452   and assumptions, cf.\ \secref{sec:obtain}).
   452   and assumptions, cf.\ \secref{sec:obtain}).
   453 
   453 
   454   \begin{rail}
   454   \begin{rail}
   455     ('lemma' | 'theorem' | 'corollary' |
   455     ('lemma' | 'theorem' | 'corollary' |
   456      'schematic\_lemma' | 'schematic\_theorem' | 'schematic\_corollary') target? (goal | longgoal)
   456      'schematic_lemma' | 'schematic_theorem' | 'schematic_corollary') target? (goal | longgoal)
   457     ;
   457     ;
   458     ('have' | 'show' | 'hence' | 'thus') goal
   458     ('have' | 'show' | 'hence' | 'thus') goal
   459     ;
   459     ;
   460     'print\_statement' modes? thmrefs
   460     'print_statement' modes? thmrefs
   461     ;
   461     ;
   462   
   462   
   463     goal: (props + 'and')
   463     goal: (props + 'and')
   464     ;
   464     ;
   465     longgoal: thmdecl? (contextelem *) conclusion
   465     longgoal: thmdecl? (contextelem *) conclusion
   841     \indexdef{}{command}{prefer}\hypertarget{command.prefer}{\hyperlink{command.prefer}{\mbox{\isa{\isacommand{prefer}}}}}\isa{{\isachardoublequote}\isactrlsup {\isacharasterisk}{\isachardoublequote}} & : & \isa{{\isachardoublequote}proof\ {\isasymrightarrow}\ proof{\isachardoublequote}} \\
   841     \indexdef{}{command}{prefer}\hypertarget{command.prefer}{\hyperlink{command.prefer}{\mbox{\isa{\isacommand{prefer}}}}}\isa{{\isachardoublequote}\isactrlsup {\isacharasterisk}{\isachardoublequote}} & : & \isa{{\isachardoublequote}proof\ {\isasymrightarrow}\ proof{\isachardoublequote}} \\
   842     \indexdef{}{command}{back}\hypertarget{command.back}{\hyperlink{command.back}{\mbox{\isa{\isacommand{back}}}}}\isa{{\isachardoublequote}\isactrlsup {\isacharasterisk}{\isachardoublequote}} & : & \isa{{\isachardoublequote}proof\ {\isasymrightarrow}\ proof{\isachardoublequote}} \\
   842     \indexdef{}{command}{back}\hypertarget{command.back}{\hyperlink{command.back}{\mbox{\isa{\isacommand{back}}}}}\isa{{\isachardoublequote}\isactrlsup {\isacharasterisk}{\isachardoublequote}} & : & \isa{{\isachardoublequote}proof\ {\isasymrightarrow}\ proof{\isachardoublequote}} \\
   843   \end{matharray}
   843   \end{matharray}
   844 
   844 
   845   \begin{rail}
   845   \begin{rail}
   846     ( 'apply' | 'apply\_end' ) method
   846     ( 'apply' | 'apply_end' ) method
   847     ;
   847     ;
   848     'defer' nat?
   848     'defer' nat?
   849     ;
   849     ;
   850     'prefer' nat
   850     'prefer' nat
   851     ;
   851     ;
   901 \begin{matharray}{rcl}
   901 \begin{matharray}{rcl}
   902     \indexdef{}{command}{method\_setup}\hypertarget{command.method-setup}{\hyperlink{command.method-setup}{\mbox{\isa{\isacommand{method{\isacharunderscore}setup}}}}} & : & \isa{{\isachardoublequote}theory\ {\isasymrightarrow}\ theory{\isachardoublequote}} \\
   902     \indexdef{}{command}{method\_setup}\hypertarget{command.method-setup}{\hyperlink{command.method-setup}{\mbox{\isa{\isacommand{method{\isacharunderscore}setup}}}}} & : & \isa{{\isachardoublequote}theory\ {\isasymrightarrow}\ theory{\isachardoublequote}} \\
   903   \end{matharray}
   903   \end{matharray}
   904 
   904 
   905   \begin{rail}
   905   \begin{rail}
   906     'method\_setup' name '=' text text
   906     'method_setup' name '=' text text
   907     ;
   907     ;
   908   \end{rail}
   908   \end{rail}
   909 
   909 
   910   \begin{description}
   910   \begin{description}
   911 
   911 
  1190     'case' (caseref | '(' caseref ((name | underscore) +) ')')
  1190     'case' (caseref | '(' caseref ((name | underscore) +) ')')
  1191     ;
  1191     ;
  1192     caseref: nameref attributes?
  1192     caseref: nameref attributes?
  1193     ;
  1193     ;
  1194 
  1194 
  1195     'case\_names' (name +)
  1195     'case_names' (name +)
  1196     ;
  1196     ;
  1197     'case\_conclusion' name (name *)
  1197     'case_conclusion' name (name *)
  1198     ;
  1198     ;
  1199     'params' ((name *) + 'and')
  1199     'params' ((name *) + 'and')
  1200     ;
  1200     ;
  1201     'consumes' nat?
  1201     'consumes' nat?
  1202     ;
  1202     ;