doc-src/Ref/simplifier.tex
changeset 7990 0a604b2fc2b1
parent 7920 1ee85d4205b2
child 8136 8c65f3ca13f2
equal deleted inserted replaced
7989:50ca726466c6 7990:0a604b2fc2b1
   500 to prove the goal.  
   500 to prove the goal.  
   501 
   501 
   502 
   502 
   503 \subsection{*The subgoaler}\label{sec:simp-subgoaler}
   503 \subsection{*The subgoaler}\label{sec:simp-subgoaler}
   504 \begin{ttbox}
   504 \begin{ttbox}
   505 setsubgoaler : simpset *  (simpset -> int -> tactic) -> simpset \hfill{\bf infix 4}
   505 setsubgoaler :
       
   506   simpset *  (simpset -> int -> tactic) -> simpset \hfill{\bf infix 4}
   506 prems_of_ss  : simpset -> thm list
   507 prems_of_ss  : simpset -> thm list
   507 \end{ttbox}
   508 \end{ttbox}
   508 
   509 
   509 The subgoaler is the tactic used to solve subgoals arising out of
   510 The subgoaler is the tactic used to solve subgoals arising out of
   510 conditional rewrite rules or congruence rules.  The default should be
   511 conditional rewrite rules or congruence rules.  The default should be
   792   in ordinary proof scripts.  The main intention is to provide an
   793   in ordinary proof scripts.  The main intention is to provide an
   793   internal interface to the simplifier for special utilities.
   794   internal interface to the simplifier for special utilities.
   794 \end{warn}
   795 \end{warn}
   795 
   796 
   796 
   797 
   797 \section{Examples of using the simplifier}
   798 \section{Examples of using the Simplifier}
   798 \index{examples!of simplification} Assume we are working within {\tt
   799 \index{examples!of simplification} Assume we are working within {\tt
   799   FOL} (see the file \texttt{FOL/ex/Nat}) and that
   800   FOL} (see the file \texttt{FOL/ex/Nat}) and that
   800 \begin{ttdescription}
   801 \begin{ttdescription}
   801 \item[Nat.thy] 
   802 \item[Nat.thy] 
   802   is a theory including the constants $0$, $Suc$ and $+$,
   803   is a theory including the constants $0$, $Suc$ and $+$,
  1237 grained control over rule application, beyond higher-order pattern
  1238 grained control over rule application, beyond higher-order pattern
  1238 matching.  Usually, procedures would do some more work, in particular
  1239 matching.  Usually, procedures would do some more work, in particular
  1239 prove particular theorems depending on the current redex.
  1240 prove particular theorems depending on the current redex.
  1240 
  1241 
  1241 
  1242 
  1242 \section{*Setting up the simplifier}\label{sec:setting-up-simp}
  1243 \section{*Setting up the Simplifier}\label{sec:setting-up-simp}
  1243 \index{simplification!setting up}
  1244 \index{simplification!setting up}
  1244 
  1245 
  1245 Setting up the simplifier for new logics is complicated.  This section
  1246 Setting up the simplifier for new logics is complicated.  This section
  1246 describes how the simplifier is installed for intuitionistic
  1247 describes how the simplifier is installed for intuitionistic
  1247 first-order logic; the code is largely taken from {\tt
  1248 first-order logic; the code is largely taken from {\tt