doc-src/TutorialI/Advanced/simp.thy
changeset 10795 9e888d60d3e5
parent 10281 9554ce1c2e54
child 10845 3696bc935bbd
--- a/doc-src/TutorialI/Advanced/simp.thy	Fri Jan 05 18:32:33 2001 +0100
+++ b/doc-src/TutorialI/Advanced/simp.thy	Fri Jan 05 18:32:57 2001 +0100
@@ -78,7 +78,7 @@
 once they apply, they can be used forever. The simplifier is aware of this
 danger and treats permutative rules by means of a special strategy, called
 \bfindex{ordered rewriting}: a permutative rewrite
-rule is only applied if the term becomes ``smaller'' (w.r.t.\ some fixed
+rule is only applied if the term becomes ``smaller'' (with respect to a fixed
 lexicographic ordering on terms). For example, commutativity rewrites
 @{term"b+a"} to @{term"a+b"}, but then stops because @{term"a+b"} is strictly
 smaller than @{term"b+a"}.  Permutative rewrite rules can be turned into