doc-src/TutorialI/Recdef/Nested2.thy
changeset 10171 59d6633835fa
parent 9940 102f2430cef9
child 10186 499637e8f2c6
--- a/doc-src/TutorialI/Recdef/Nested2.thy	Mon Oct 09 09:33:45 2000 +0200
+++ b/doc-src/TutorialI/Recdef/Nested2.thy	Mon Oct 09 10:18:21 2000 +0200
@@ -78,7 +78,7 @@
 recdef dummy "{}"
 "dummy n = n"
 (*>*)
-(hints cong: map_cong)
+(hints recdef_cong: map_cong)
 
 text{*\noindent
 or declare them globally
@@ -88,11 +88,11 @@
 declare map_cong[recdef_cong];
 
 text{*
-Note that the global @{text cong} and @{text recdef_cong} attributes are
+Note that the @{text cong} and @{text recdef_cong} attributes are
 intentionally kept apart because they control different activities, namely
-simplification and making recursive definitions. The local @{text cong} in
-the hints section of \isacommand{recdef} is merely short for @{text
-recdef_cong}.
+simplification and making recursive definitions.
+% The local @{text cong} in
+% the hints section of \isacommand{recdef} is merely short for @{text recdef_cong}.
 %The simplifier's congruence rules cannot be used by recdef.
 %For example the weak congruence rules for if and case would prevent
 %recdef from generating sensible termination conditions.