doc-src/TutorialI/Misc/simp.thy
changeset 10971 6852682eaf16
parent 10885 90695f46440b
child 10983 59961d32b1ae
--- a/doc-src/TutorialI/Misc/simp.thy	Wed Jan 24 11:59:15 2001 +0100
+++ b/doc-src/TutorialI/Misc/simp.thy	Wed Jan 24 12:29:10 2001 +0100
@@ -49,7 +49,7 @@
 where the list of \emph{modifiers} fine tunes the behaviour and may
 be empty. Most if not all of the proofs seen so far could have been performed
 with @{text simp} instead of \isa{auto}, except that @{text simp} attacks
-only the first subgoal and may thus need to be repeated---use
+only the first subgoal and may thus need to be repeated --- use
 \isaindex{simp_all} to simplify all subgoals.
 Note that @{text simp} fails if nothing changes.
 *}
@@ -106,7 +106,7 @@
 done
 
 text{*\noindent
-There are three options that influence the treatment of assumptions:
+There are three modifiers that influence the treatment of assumptions:
 \begin{description}
 \item[@{text"(no_asm)"}]\indexbold{*no_asm}
  means that assumptions are completely ignored.
@@ -119,7 +119,7 @@
 \end{description}
 Both @{text"(no_asm_simp)"} and @{text"(no_asm_use)"} run forever on
 the problematic subgoal above.
-Note that only one of the options is allowed, and it must precede all
+Note that only one of the modifiers is allowed, and it must precede all
 other arguments.
 *}
 
@@ -165,13 +165,14 @@
 rule because this defeats the whole purpose of an abbreviation.
 
 \begin{warn}
-  If you have defined $f\,x\,y~\isasymequiv~t$ then you can only expand
-  occurrences of $f$ with at least two arguments. Thus it is safer to define
-  $f$~\isasymequiv~\isasymlambda$x\,y.\;t$.
+  If you have defined $f\,x\,y~\isasymequiv~t$ then you can only unfold
+  occurrences of $f$ with at least two arguments. This may be helpful for unfolding
+  $f$ selectively, but it may also get in the way. Defining
+  $f$~\isasymequiv~\isasymlambda$x\,y.\;t$ allows to unfold all occurrences of $f$.
 \end{warn}
 *}
 
-subsubsection{*Simplifying Let-Expressions*}
+subsubsection{*Simplifying {\tt\slshape let}-Expressions*}
 
 text{*\index{simplification!of let-expressions}
 Proving a goal containing \isaindex{let}-expressions almost invariably
@@ -370,7 +371,7 @@
 Applying instance of rewrite rule:
 rev (?x1 \# ?xs1) == rev ?xs1 @ [?x1]
 Rewriting:
-rev [x] == rev [] @ [x]
+rev [a] == rev [] @ [a]
 Applying instance of rewrite rule:
 rev [] == []
 Rewriting:
@@ -378,11 +379,11 @@
 Applying instance of rewrite rule:
 [] @ ?y == ?y
 Rewriting:
-[] @ [x] == [x]
+[] @ [a] == [a]
 Applying instance of rewrite rule:
 ?x3 \# ?t3 = ?t3 == False
 Rewriting:
-[x] = [] == False
+[a] = [] == False
 \end{ttbox}
 
 In more complicated cases, the trace can be quite lenghty, especially since