doc-src/IsarRef/Thy/Proof.thy
changeset 30510 4120fc59dd85
parent 30462 0b857a58b15e
child 30547 4c2514625873
equal deleted inserted replaced
30509:e19d5b459a61 30510:4120fc59dd85
   893   arguments, or a list of theorems, respectively.
   893   arguments, or a list of theorems, respectively.
   894 
   894 
   895 %FIXME proper antiquotations
   895 %FIXME proper antiquotations
   896 {\footnotesize
   896 {\footnotesize
   897 \begin{verbatim}
   897 \begin{verbatim}
   898  Method.no_args (Method.METHOD (fn facts => foobar_tac))
   898  Method.no_args (METHOD (fn facts => foobar_tac))
   899  Method.thms_args (fn thms => Method.METHOD (fn facts => foobar_tac))
   899  Method.thms_args (fn thms => METHOD (fn facts => foobar_tac))
   900  Method.ctxt_args (fn ctxt => Method.METHOD (fn facts => foobar_tac))
   900  Method.ctxt_args (fn ctxt => METHOD (fn facts => foobar_tac))
   901  Method.thms_ctxt_args (fn thms => fn ctxt =>
   901  Method.thms_ctxt_args (fn thms => fn ctxt => METHOD (fn facts => foobar_tac))
   902     Method.METHOD (fn facts => foobar_tac))
       
   903 \end{verbatim}
   902 \end{verbatim}
   904 }
   903 }
   905 
   904 
   906   Note that mere tactic emulations may ignore the @{text facts}
   905   Note that mere tactic emulations may ignore the @{text facts}
   907   parameter above.  Proper proof methods would do something
   906   parameter above.  Proper proof methods would do something