--- a/doc-src/TutorialI/Misc/pairs.thy Wed Nov 29 18:42:40 2000 +0100
+++ b/doc-src/TutorialI/Misc/pairs.thy Thu Nov 30 13:56:46 2000 +0100
@@ -1,8 +1,7 @@
(*<*)
theory pairs = Main:;
(*>*)
-text{*\label{sec:pairs}\indexbold{product type}
-\index{pair|see{product type}}\index{tuple|see{product type}}
+text{*\label{sec:pairs}\indexbold{pair}
HOL also has pairs: \isa{($a@1$,$a@2$)} is of type $\tau@1$
\indexboldpos{\isasymtimes}{$Isatype} $\tau@2$ provided each $a@i$ is of type
$\tau@i$. The components of a pair are extracted by \isaindexbold{fst} and