doc-src/TutorialI/Misc/simp.thy
changeset 12582 b85acd66f715
parent 12533 e417bd7ca8a0
child 12631 7648ac4a6b95
--- a/doc-src/TutorialI/Misc/simp.thy	Fri Dec 21 17:31:45 2001 +0100
+++ b/doc-src/TutorialI/Misc/simp.thy	Fri Dec 21 19:55:39 2001 +0100
@@ -156,8 +156,7 @@
 Constant definitions (\S\ref{sec:ConstDefinitions}) can be used as
 simplification rules, but by default they are not: the simplifier does not
 expand them automatically.  Definitions are intended for introducing abstract
-concepts and not merely as abbreviations.  (Contrast with syntax
-translations, \S\ref{sec:def-translations}.)  Of course, we need to expand
+concepts and not merely as abbreviations.  Of course, we need to expand
 the definition initially, but once we have proved enough abstract properties
 of the new constant, we can forget its original definition.  This style makes
 proofs more robust: if the definition has to be changed,