diff -r 55c0f9a8df78 -r 59961d32b1ae doc-src/TutorialI/Types/Typedef.thy --- a/doc-src/TutorialI/Types/Typedef.thy Fri Jan 26 15:02:04 2001 +0100 +++ b/doc-src/TutorialI/Types/Typedef.thy Fri Jan 26 15:50:28 2001 +0100 @@ -96,8 +96,10 @@ @{term Abs_three} &::& @{typ"nat \ three"} \end{tabular} \end{center} -Constant @{term three} is just an abbreviation (@{thm[source]three_def}): -@{thm[display]three_def} +Constant @{term three} is explicitly defined as the representing set: +\begin{center} +@{thm three_def}\hfill(@{thm[source]three_def}) +\end{center} The situation is best summarized with the help of the following diagram, where squares are types and circles are sets: \begin{center} @@ -118,10 +120,10 @@ surjective on the subset @{term three} and @{term Abs_three} and @{term Rep_three} are inverses of each other: \begin{center} -\begin{tabular}{rl} -@{thm Rep_three[no_vars]} &~~ (@{thm[source]Rep_three}) \\ -@{thm Rep_three_inverse[no_vars]} &~~ (@{thm[source]Rep_three_inverse}) \\ -@{thm Abs_three_inverse[no_vars]} &~~ (@{thm[source]Abs_three_inverse}) +\begin{tabular}{@ {}r@ {\qquad\qquad}l@ {}} +@{thm Rep_three[no_vars]} & (@{thm[source]Rep_three}) \\ +@{thm Rep_three_inverse[no_vars]} & (@{thm[source]Rep_three_inverse}) \\ +@{thm Abs_three_inverse[no_vars]} & (@{thm[source]Abs_three_inverse}) \end{tabular} \end{center} %