doc-src/IsarImplementation/Thy/Tactic.thy
changeset 46274 67139209b548
parent 46271 e1b5460f1725
child 46276 8f1f33faf24e
equal deleted inserted replaced
46273:48cf461535cf 46274:67139209b548
   400   of \secref{sec:struct-goals} allows to refer to internal goal
   400   of \secref{sec:struct-goals} allows to refer to internal goal
   401   structure with explicit context management.
   401   structure with explicit context management.
   402 *}
   402 *}
   403 
   403 
   404 
   404 
       
   405 subsection {* Rearranging goal states *}
       
   406 
       
   407 text {* In rare situations there is a need to rearrange goal states:
       
   408   either the overall collection of subgoals, or the local structure of
       
   409   a subgoal.  Various administrative tactics allow to operate on the
       
   410   concrete presentation these conceptual sets of formulae. *}
       
   411 
       
   412 text %mlref {*
       
   413   \begin{mldecls}
       
   414   @{index_ML rotate_tac: "int -> int -> tactic"} \\
       
   415   \end{mldecls}
       
   416 
       
   417   \begin{description}
       
   418 
       
   419   \item @{ML rotate_tac}~@{text "n i"} rotates the premises of subgoal
       
   420   @{text i} by @{text n} positions: from right to left if @{text n} is
       
   421   positive, and from left to right if @{text n} is negative.
       
   422 
       
   423   \end{description}
       
   424 *}
       
   425 
   405 section {* Tacticals \label{sec:tacticals} *}
   426 section {* Tacticals \label{sec:tacticals} *}
   406 
   427 
   407 text {* A \emph{tactical} is a functional combinator for building up
   428 text {* A \emph{tactical} is a functional combinator for building up
   408   complex tactics from simpler ones.  Common tacticals perform
   429   complex tactics from simpler ones.  Common tacticals perform
   409   sequential composition, disjunctive choice, iteration, or goal
   430   sequential composition, disjunctive choice, iteration, or goal