doc-src/IsarRef/Thy/Generic.thy
changeset 27239 f2f42f9fa09d
parent 27223 8546e2407b31
child 27248 3c17b824650b
equal deleted inserted replaced
27238:d2bf12727c8a 27239:f2f42f9fa09d
   306 
   306 
   307 \begin{descr}
   307 \begin{descr}
   308 
   308 
   309   \item [@{method rule_tac} etc.] do resolution of rules with explicit
   309   \item [@{method rule_tac} etc.] do resolution of rules with explicit
   310   instantiation.  This works the same way as the ML tactics @{ML
   310   instantiation.  This works the same way as the ML tactics @{ML
   311   Tactic.res_inst_tac} etc. (see \cite[\S3]{isabelle-ref})
   311   res_inst_tac} etc. (see \cite[\S3]{isabelle-ref})
   312 
   312 
   313   Multiple rules may be only given if there is no instantiation; then
   313   Multiple rules may be only given if there is no instantiation; then
   314   @{method rule_tac} is the same as @{ML resolve_tac} in ML (see
   314   @{method rule_tac} is the same as @{ML resolve_tac} in ML (see
   315   \cite[\S3]{isabelle-ref}).
   315   \cite[\S3]{isabelle-ref}).
   316 
   316 
   321   may be given as well, see also ML tactic @{ML Tactic.cut_inst_tac}
   321   may be given as well, see also ML tactic @{ML Tactic.cut_inst_tac}
   322   in \cite[\S3]{isabelle-ref}.
   322   in \cite[\S3]{isabelle-ref}.
   323 
   323 
   324   \item [@{method thin_tac}~@{text \<phi>}] deletes the specified
   324   \item [@{method thin_tac}~@{text \<phi>}] deletes the specified
   325   assumption from a subgoal; note that @{text \<phi>} may contain schematic
   325   assumption from a subgoal; note that @{text \<phi>} may contain schematic
   326   variables.  See also @{ML Tactic.thin_tac} in
   326   variables.  See also @{ML thin_tac} in
   327   \cite[\S3]{isabelle-ref}.
   327   \cite[\S3]{isabelle-ref}.
   328 
   328 
   329   \item [@{method subgoal_tac}~@{text \<phi>}] adds @{text \<phi>} as an
   329   \item [@{method subgoal_tac}~@{text \<phi>}] adds @{text \<phi>} as an
   330   assumption to a subgoal.  See also @{ML Tactic.subgoal_tac} and @{ML
   330   assumption to a subgoal.  See also @{ML subgoal_tac} and @{ML
   331   Tactic.subgoals_tac} in \cite[\S3]{isabelle-ref}.
   331   subgoals_tac} in \cite[\S3]{isabelle-ref}.
   332 
   332 
   333   \item [@{method rename_tac}~@{text "x\<^sub>1 \<dots> x\<^sub>n"}] renames
   333   \item [@{method rename_tac}~@{text "x\<^sub>1 \<dots> x\<^sub>n"}] renames
   334   parameters of a goal according to the list @{text "x\<^sub>1, \<dots>,
   334   parameters of a goal according to the list @{text "x\<^sub>1, \<dots>,
   335   x\<^sub>n"}, which refers to the \emph{suffix} of variables.
   335   x\<^sub>n"}, which refers to the \emph{suffix} of variables.
   336 
   336