doc-src/TutorialI/Types/Typedefs.thy
changeset 12628 6a07c3bf4903
parent 12543 3e355f0f079f
child 12815 1f073030b97a
equal deleted inserted replaced
12627:08eee994bf99 12628:6a07c3bf4903
   100 @{thm three_def}\hfill(@{thm[source]three_def})
   100 @{thm three_def}\hfill(@{thm[source]three_def})
   101 \end{center}
   101 \end{center}
   102 The situation is best summarized with the help of the following diagram,
   102 The situation is best summarized with the help of the following diagram,
   103 where squares denote types and the irregular region denotes a set:
   103 where squares denote types and the irregular region denotes a set:
   104 \begin{center}
   104 \begin{center}
   105 \includegraphics[scale=.8]{Types/typedef}
   105 \includegraphics[scale=.8]{typedef}
   106 \end{center}
   106 \end{center}
   107 Finally, \isacommand{typedef} asserts that @{term Rep_three} is
   107 Finally, \isacommand{typedef} asserts that @{term Rep_three} is
   108 surjective on the subset @{term three} and @{term Abs_three} and @{term
   108 surjective on the subset @{term three} and @{term Abs_three} and @{term
   109 Rep_three} are inverses of each other:
   109 Rep_three} are inverses of each other:
   110 \begin{center}
   110 \begin{center}