avoid clash of Misc/pairs.thy and Types/Pairs.thy on case-insensible file-system;
--- a/doc-src/TutorialI/IsaMakefile Thu Jul 26 19:07:28 2012 +0200
+++ b/doc-src/TutorialI/IsaMakefile Thu Jul 26 19:08:14 2012 +0200
@@ -41,7 +41,7 @@
Inductive/Advanced.thy Types/Numbers.thy Types/Pairs.thy \
Types/Records.thy Types/Typedefs.thy Types/Overloading.thy \
Types/Axioms.thy Misc/Tree.thy Misc/Tree2.thy Misc/Plus.thy \
- Misc/fakenat.thy Misc/natsum.thy Misc/pairs.thy Misc/Option2.thy \
+ Misc/fakenat.thy Misc/natsum.thy Misc/pairs2.thy Misc/Option2.thy \
Misc/types.thy Misc/prime_def.thy Misc/case_exprs.thy Misc/simp.thy \
Misc/Itrev.thy Misc/AdvancedInd.thy Misc/appendix.thy \
Protocol/Message.thy Protocol/Event.thy Protocol/Public.thy \
--- a/doc-src/TutorialI/Misc/pairs.thy Thu Jul 26 19:07:28 2012 +0200
+++ /dev/null Thu Jan 01 00:00:00 1970 +0000
@@ -1,35 +0,0 @@
-(*<*)
-theory pairs imports Main begin;
-(*>*)
-text{*\label{sec:pairs}\index{pairs and tuples}
-HOL also has ordered 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 functions \cdx{fst} and
-\cdx{snd} extract the components of a pair:
- \isa{fst($x$,$y$) = $x$} and \isa{snd($x$,$y$) = $y$}. Tuples
-are simulated by pairs nested to the right: \isa{($a@1$,$a@2$,$a@3$)} stands
-for \isa{($a@1$,($a@2$,$a@3$))} and $\tau@1 \times \tau@2 \times \tau@3$ for
-$\tau@1 \times (\tau@2 \times \tau@3)$. Therefore we have
-\isa{fst(snd($a@1$,$a@2$,$a@3$)) = $a@2$}.
-
-Remarks:
-\begin{itemize}
-\item
-There is also the type \tydx{unit}, which contains exactly one
-element denoted by~\cdx{()}. This type can be viewed
-as a degenerate product with 0 components.
-\item
-Products, like type @{typ nat}, are datatypes, which means
-in particular that @{text induct_tac} and @{text case_tac} are applicable to
-terms of product type.
-Both split the term into a number of variables corresponding to the tuple structure
-(up to 7 components).
-\item
-Tuples with more than two or three components become unwieldy;
-records are preferable.
-\end{itemize}
-For more information on pairs and records see Chapter~\ref{ch:more-types}.
-*}
-(*<*)
-end
-(*>*)
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/TutorialI/Misc/pairs2.thy Thu Jul 26 19:08:14 2012 +0200
@@ -0,0 +1,35 @@
+(*<*)
+theory pairs2 imports Main begin;
+(*>*)
+text{*\label{sec:pairs}\index{pairs and tuples}
+HOL also has ordered 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 functions \cdx{fst} and
+\cdx{snd} extract the components of a pair:
+ \isa{fst($x$,$y$) = $x$} and \isa{snd($x$,$y$) = $y$}. Tuples
+are simulated by pairs nested to the right: \isa{($a@1$,$a@2$,$a@3$)} stands
+for \isa{($a@1$,($a@2$,$a@3$))} and $\tau@1 \times \tau@2 \times \tau@3$ for
+$\tau@1 \times (\tau@2 \times \tau@3)$. Therefore we have
+\isa{fst(snd($a@1$,$a@2$,$a@3$)) = $a@2$}.
+
+Remarks:
+\begin{itemize}
+\item
+There is also the type \tydx{unit}, which contains exactly one
+element denoted by~\cdx{()}. This type can be viewed
+as a degenerate product with 0 components.
+\item
+Products, like type @{typ nat}, are datatypes, which means
+in particular that @{text induct_tac} and @{text case_tac} are applicable to
+terms of product type.
+Both split the term into a number of variables corresponding to the tuple structure
+(up to 7 components).
+\item
+Tuples with more than two or three components become unwieldy;
+records are preferable.
+\end{itemize}
+For more information on pairs and records see Chapter~\ref{ch:more-types}.
+*}
+(*<*)
+end
+(*>*)
--- a/doc-src/TutorialI/ROOT.ML Thu Jul 26 19:07:28 2012 +0200
+++ b/doc-src/TutorialI/ROOT.ML Thu Jul 26 19:08:14 2012 +0200
@@ -33,7 +33,7 @@
use_thy "Misc/case_exprs";
use_thy "Misc/fakenat";
use_thy "Misc/natsum";
-use_thy "Misc/pairs";
+use_thy "Misc/pairs2";
use_thy "Misc/Option2";
use_thy "Misc/types";
use_thy "Misc/prime_def";
--- a/doc-src/TutorialI/document/pairs.tex Thu Jul 26 19:07:28 2012 +0200
+++ /dev/null Thu Jan 01 00:00:00 1970 +0000
@@ -1,66 +0,0 @@
-%
-\begin{isabellebody}%
-\def\isabellecontext{pairs}%
-%
-\isadelimtheory
-%
-\endisadelimtheory
-%
-\isatagtheory
-%
-\endisatagtheory
-{\isafoldtheory}%
-%
-\isadelimtheory
-%
-\endisadelimtheory
-%
-\begin{isamarkuptext}%
-\label{sec:pairs}\index{pairs and tuples}
-HOL also has ordered 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 functions \cdx{fst} and
-\cdx{snd} extract the components of a pair:
- \isa{fst($x$,$y$) = $x$} and \isa{snd($x$,$y$) = $y$}. Tuples
-are simulated by pairs nested to the right: \isa{($a@1$,$a@2$,$a@3$)} stands
-for \isa{($a@1$,($a@2$,$a@3$))} and $\tau@1 \times \tau@2 \times \tau@3$ for
-$\tau@1 \times (\tau@2 \times \tau@3)$. Therefore we have
-\isa{fst(snd($a@1$,$a@2$,$a@3$)) = $a@2$}.
-
-Remarks:
-\begin{itemize}
-\item
-There is also the type \tydx{unit}, which contains exactly one
-element denoted by~\cdx{()}. This type can be viewed
-as a degenerate product with 0 components.
-\item
-Products, like type \isa{nat}, are datatypes, which means
-in particular that \isa{induct{\isaliteral{5F}{\isacharunderscore}}tac} and \isa{case{\isaliteral{5F}{\isacharunderscore}}tac} are applicable to
-terms of product type.
-Both split the term into a number of variables corresponding to the tuple structure
-(up to 7 components).
-\item
-Tuples with more than two or three components become unwieldy;
-records are preferable.
-\end{itemize}
-For more information on pairs and records see Chapter~\ref{ch:more-types}.%
-\end{isamarkuptext}%
-\isamarkuptrue%
-%
-\isadelimtheory
-%
-\endisadelimtheory
-%
-\isatagtheory
-%
-\endisatagtheory
-{\isafoldtheory}%
-%
-\isadelimtheory
-%
-\endisadelimtheory
-\end{isabellebody}%
-%%% Local Variables:
-%%% mode: latex
-%%% TeX-master: "root"
-%%% End:
--- /dev/null Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/TutorialI/document/pairs2.tex Thu Jul 26 19:08:14 2012 +0200
@@ -0,0 +1,66 @@
+%
+\begin{isabellebody}%
+\def\isabellecontext{pairs{\isadigit{2}}}%
+%
+\isadelimtheory
+%
+\endisadelimtheory
+%
+\isatagtheory
+%
+\endisatagtheory
+{\isafoldtheory}%
+%
+\isadelimtheory
+%
+\endisadelimtheory
+%
+\begin{isamarkuptext}%
+\label{sec:pairs}\index{pairs and tuples}
+HOL also has ordered 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 functions \cdx{fst} and
+\cdx{snd} extract the components of a pair:
+ \isa{fst($x$,$y$) = $x$} and \isa{snd($x$,$y$) = $y$}. Tuples
+are simulated by pairs nested to the right: \isa{($a@1$,$a@2$,$a@3$)} stands
+for \isa{($a@1$,($a@2$,$a@3$))} and $\tau@1 \times \tau@2 \times \tau@3$ for
+$\tau@1 \times (\tau@2 \times \tau@3)$. Therefore we have
+\isa{fst(snd($a@1$,$a@2$,$a@3$)) = $a@2$}.
+
+Remarks:
+\begin{itemize}
+\item
+There is also the type \tydx{unit}, which contains exactly one
+element denoted by~\cdx{()}. This type can be viewed
+as a degenerate product with 0 components.
+\item
+Products, like type \isa{nat}, are datatypes, which means
+in particular that \isa{induct{\isaliteral{5F}{\isacharunderscore}}tac} and \isa{case{\isaliteral{5F}{\isacharunderscore}}tac} are applicable to
+terms of product type.
+Both split the term into a number of variables corresponding to the tuple structure
+(up to 7 components).
+\item
+Tuples with more than two or three components become unwieldy;
+records are preferable.
+\end{itemize}
+For more information on pairs and records see Chapter~\ref{ch:more-types}.%
+\end{isamarkuptext}%
+\isamarkuptrue%
+%
+\isadelimtheory
+%
+\endisadelimtheory
+%
+\isatagtheory
+%
+\endisatagtheory
+{\isafoldtheory}%
+%
+\isadelimtheory
+%
+\endisadelimtheory
+\end{isabellebody}%
+%%% Local Variables:
+%%% mode: latex
+%%% TeX-master: "root"
+%%% End:
--- a/doc-src/TutorialI/fp.tex Thu Jul 26 19:07:28 2012 +0200
+++ b/doc-src/TutorialI/fp.tex Thu Jul 26 19:08:14 2012 +0200
@@ -229,7 +229,7 @@
\subsection{Pairs}
-\input{document/pairs.tex}
+\input{document/pairs2.tex}
\subsection{Datatype {\tt\slshape option}}
\label{sec:option}