doc-src/TutorialI/Types/Pairs.thy
changeset 11277 a2bff98d6e5d
parent 11161 166f7d87b37f
child 11428 332347b9b942
--- a/doc-src/TutorialI/Types/Pairs.thy	Tue May 01 17:16:32 2001 +0200
+++ b/doc-src/TutorialI/Types/Pairs.thy	Tue May 01 22:26:55 2001 +0200
@@ -109,9 +109,9 @@
 txt{*
 @{subgoals[display,indent=0]}
 Again, simplification produces a term suitable for @{thm[source]split_split}
-as above. If you are worried about the funny form of the premise:
-@{term"split (op =)"} is the same as @{text"\<lambda>(x,y). x=y"}.
-The same procedure works for
+as above. If you are worried about the strange form of the premise:
+@{term"split (op =)"} is short for @{text"\<lambda>(x,y). x=y"}.
+The same proof procedure works for
 *}
 
 (*<*)by(simp split:split_split)(*>*)