doc-src/TutorialI/Types/Pairs.thy
changeset 15905 0a4cc9b113c7
parent 12815 1f073030b97a
child 17914 99ead7a7eb42
--- a/doc-src/TutorialI/Types/Pairs.thy	Mon May 02 10:56:13 2005 +0200
+++ b/doc-src/TutorialI/Types/Pairs.thy	Mon May 02 11:03:27 2005 +0200
@@ -138,7 +138,7 @@
 lemma "swap(swap p) = p"
 
 txt{*\noindent
-simplification will do nothing, because the defining equation for @{term swap}
+simplification will do nothing, because the defining equation for @{const swap}
 expects a pair. Again, we need to turn @{term p} into a pair first, but this
 time there is no @{term split} in sight. In this case the only thing we can do
 is to split the term by hand: