1 (* Title: Doc/Datatypes/Datatypes.thy |
1 (* Title: Doc/Datatypes/Datatypes.thy |
2 Author: Jasmin Blanchette, TU Muenchen |
2 Author: Jasmin Blanchette, TU Muenchen |
|
3 Author: Martin Desharnais, Ecole de technologie superieure |
3 Author: Lorenz Panny, TU Muenchen |
4 Author: Lorenz Panny, TU Muenchen |
4 Author: Andrei Popescu, TU Muenchen |
5 Author: Andrei Popescu, TU Muenchen |
5 Author: Dmitriy Traytel, TU Muenchen |
6 Author: Dmitriy Traytel, TU Muenchen |
6 |
7 |
7 Tutorial for (co)datatype definitions with the new package. |
8 Tutorial for (co)datatype definitions with the new package. |
138 \newbox\boxA |
139 \newbox\boxA |
139 \setbox\boxA=\hbox{\texttt{NOSPAM}} |
140 \setbox\boxA=\hbox{\texttt{NOSPAM}} |
140 |
141 |
141 \newcommand\authoremaili{\texttt{blan{\color{white}NOSPAM}\kern-\wd\boxA{}chette@\allowbreak |
142 \newcommand\authoremaili{\texttt{blan{\color{white}NOSPAM}\kern-\wd\boxA{}chette@\allowbreak |
142 in.\allowbreak tum.\allowbreak de}} |
143 in.\allowbreak tum.\allowbreak de}} |
143 \newcommand\authoremailii{\texttt{lore{\color{white}NOSPAM}\kern-\wd\boxA{}nz.panny@\allowbreak |
144 \newcommand\authoremailii{\texttt{desh{\color{white}NOSPAM}\kern-\wd\boxA{}arna@\allowbreak |
144 \allowbreak tum.\allowbreak de}} |
|
145 \newcommand\authoremailiii{\texttt{pope{\color{white}NOSPAM}\kern-\wd\boxA{}scua@\allowbreak |
|
146 in.\allowbreak tum.\allowbreak de}} |
145 in.\allowbreak tum.\allowbreak de}} |
147 \newcommand\authoremailiv{\texttt{tray{\color{white}NOSPAM}\kern-\wd\boxA{}tel@\allowbreak |
146 \newcommand\authoremailiii{\texttt{lore{\color{white}NOSPAM}\kern-\wd\boxA{}nz.panny@\allowbreak |
|
147 in.\allowbreak tum.\allowbreak de}} |
|
148 \newcommand\authoremailiv{\texttt{pope{\color{white}NOSPAM}\kern-\wd\boxA{}scua@\allowbreak |
|
149 in.\allowbreak tum.\allowbreak de}} |
|
150 \newcommand\authoremailv{\texttt{tray{\color{white}NOSPAM}\kern-\wd\boxA{}tel@\allowbreak |
148 in.\allowbreak tum.\allowbreak de}} |
151 in.\allowbreak tum.\allowbreak de}} |
149 |
152 |
150 The command @{command datatype_new} is expected to replace \keyw{datatype} in a |
153 The command @{command datatype_new} is expected to replace \keyw{datatype} in a |
151 future release. Authors of new theories are encouraged to use the new commands, |
154 future release. Authors of new theories are encouraged to use the new commands, |
152 and maintainers of older theories may want to consider upgrading. |
155 and maintainers of older theories may want to consider upgrading. |
153 |
156 |
154 Comments and bug reports concerning either the tool or this tutorial should be |
157 Comments and bug reports concerning either the tool or this tutorial should be |
155 directed to the authors at \authoremaili, \authoremailii, \authoremailiii, |
158 directed to the authors at \authoremaili, \authoremailii, \authoremailiii, |
156 and \authoremailiv. |
159 \authoremailiv, and \authoremailv. |
157 *} |
160 *} |
158 |
161 |
159 |
162 |
160 section {* Defining Datatypes |
163 section {* Defining Datatypes |
161 \label{sec:defining-datatypes} *} |
164 \label{sec:defining-datatypes} *} |