author | desharna |
Mon, 01 Sep 2014 13:53:39 +0200 | |
changeset 58107 | f3c5360711e9 |
parent 58105 | 42c09d2ac48b |
child 58121 | d7550665da31 |
permissions | -rw-r--r-- |
52792 | 1 |
(* Title: Doc/Datatypes/Datatypes.thy |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
57079 | 3 |
Author: Martin Desharnais, Ecole de technologie superieure |
53617 | 4 |
Author: Lorenz Panny, TU Muenchen |
5 |
Author: Andrei Popescu, TU Muenchen |
|
6 |
Author: Dmitriy Traytel, TU Muenchen |
|
52792 | 7 |
|
8 |
Tutorial for (co)datatype definitions with the new package. |
|
9 |
*) |
|
10 |
||
11 |
theory Datatypes |
|
55073 | 12 |
imports |
13 |
Setup |
|
56942 | 14 |
"~~/src/HOL/Library/BNF_Axiomatization" |
55350 | 15 |
"~~/src/HOL/Library/Cardinal_Notations" |
55129
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
16 |
"~~/src/HOL/Library/FSet" |
55073 | 17 |
"~~/src/HOL/Library/Simps_Case_Conv" |
52792 | 18 |
begin |
19 |
||
52828 | 20 |
section {* Introduction |
21 |
\label{sec:introduction} *} |
|
52792 | 22 |
|
23 |
text {* |
|
53028 | 24 |
The 2013 edition of Isabelle introduced a new definitional package for freely |
25 |
generated datatypes and codatatypes. The datatype support is similar to that |
|
26 |
provided by the earlier package due to Berghofer and Wenzel |
|
27 |
\cite{Berghofer-Wenzel:1999:TPHOL}, documented in the Isar reference manual |
|
53535 | 28 |
\cite{isabelle-isar-ref}; indeed, replacing the keyword \keyw{datatype} by |
53028 | 29 |
@{command datatype_new} is usually all that is needed to port existing theories |
30 |
to use the new package. |
|
52840 | 31 |
|
52841 | 32 |
Perhaps the main advantage of the new package is that it supports recursion |
53619 | 33 |
through a large class of non-datatypes, such as finite sets: |
52792 | 34 |
*} |
35 |
||
53644 | 36 |
datatype_new 'a tree\<^sub>f\<^sub>s = Node\<^sub>f\<^sub>s (lbl\<^sub>f\<^sub>s: 'a) (sub\<^sub>f\<^sub>s: "'a tree\<^sub>f\<^sub>s fset") |
52792 | 37 |
|
38 |
text {* |
|
52794 | 39 |
\noindent |
53025 | 40 |
Another strong point is the support for local definitions: |
52792 | 41 |
*} |
42 |
||
52805 | 43 |
context linorder |
44 |
begin |
|
52841 | 45 |
datatype_new flag = Less | Eq | Greater |
52805 | 46 |
end |
52792 | 47 |
|
48 |
text {* |
|
52794 | 49 |
\noindent |
54187 | 50 |
Furthermore, the package provides a lot of convenience, including automatically |
51 |
generated discriminators, selectors, and relators as well as a wealth of |
|
52 |
properties about them. |
|
53 |
||
54 |
In addition to inductive datatypes, the new package supports coinductive |
|
55 |
datatypes, or \emph{codatatypes}, which allow infinite values. For example, the |
|
56 |
following command introduces the type of lazy lists, which comprises both finite |
|
57 |
and infinite values: |
|
52794 | 58 |
*} |
59 |
||
53623 | 60 |
(*<*) |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
61 |
locale early |
54072 | 62 |
locale late |
53623 | 63 |
(*>*) |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
64 |
codatatype (*<*)(in early) (*>*)'a llist = LNil | LCons 'a "'a llist" |
52794 | 65 |
|
66 |
text {* |
|
67 |
\noindent |
|
52840 | 68 |
Mixed inductive--coinductive recursion is possible via nesting. Compare the |
53028 | 69 |
following four Rose tree examples: |
52794 | 70 |
*} |
71 |
||
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
72 |
datatype_new (*<*)(in early) (*>*)'a tree\<^sub>f\<^sub>f = Node\<^sub>f\<^sub>f 'a "'a tree\<^sub>f\<^sub>f list" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
73 |
datatype_new (*<*)(in early) (*>*)'a tree\<^sub>f\<^sub>i = Node\<^sub>f\<^sub>i 'a "'a tree\<^sub>f\<^sub>i llist" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
74 |
codatatype (*<*)(in early) (*>*)'a tree\<^sub>i\<^sub>f = Node\<^sub>i\<^sub>f 'a "'a tree\<^sub>i\<^sub>f list" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
75 |
codatatype (*<*)(in early) (*>*)'a tree\<^sub>i\<^sub>i = Node\<^sub>i\<^sub>i 'a "'a tree\<^sub>i\<^sub>i llist" |
52792 | 76 |
|
52794 | 77 |
text {* |
54187 | 78 |
The first two tree types allow only paths of finite length, whereas the last two |
79 |
allow infinite paths. Orthogonally, the nodes in the first and third types have |
|
80 |
finitely many direct subtrees, whereas those of the second and fourth may have |
|
81 |
infinite branching. |
|
52840 | 82 |
|
55073 | 83 |
The package is part of @{theory Main}. Additional functionality is provided by |
56942 | 84 |
the theory @{theory BNF_Axiomatization}, located in the directory |
55129
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
85 |
\verb|~~/src/HOL/Library|. |
55073 | 86 |
|
52805 | 87 |
The package, like its predecessor, fully adheres to the LCF philosophy |
88 |
\cite{mgordon79}: The characteristic theorems associated with the specified |
|
89 |
(co)datatypes are derived rather than introduced axiomatically.% |
|
57542 | 90 |
\footnote{However, some of the |
91 |
internal constructions and most of the internal proof obligations are skipped |
|
92 |
if the @{text quick_and_dirty} option is enabled.} |
|
57575 | 93 |
The package is described in a number of papers |
57542 | 94 |
\cite{traytel-et-al-2012,blanchette-et-al-wit,blanchette-et-al-2014-impl,panny-et-al-2014}. |
95 |
The central notion is that of a \emph{bounded natural functor} (BNF)---a |
|
96 |
well-behaved type constructor for which nested (co)recursion is supported. |
|
52792 | 97 |
|
52794 | 98 |
This tutorial is organized as follows: |
99 |
||
52805 | 100 |
\begin{itemize} |
52822 | 101 |
\setlength{\itemsep}{0pt} |
102 |
||
52805 | 103 |
\item Section \ref{sec:defining-datatypes}, ``Defining Datatypes,'' |
52822 | 104 |
describes how to specify datatypes using the @{command datatype_new} command. |
52805 | 105 |
|
53018 | 106 |
\item Section \ref{sec:defining-recursive-functions}, ``Defining Recursive |
52805 | 107 |
Functions,'' describes how to specify recursive functions using |
56655 | 108 |
@{command primrec}. |
52805 | 109 |
|
110 |
\item Section \ref{sec:defining-codatatypes}, ``Defining Codatatypes,'' |
|
53829 | 111 |
describes how to specify codatatypes using the @{command codatatype} command. |
52805 | 112 |
|
53018 | 113 |
\item Section \ref{sec:defining-corecursive-functions}, ``Defining Corecursive |
52805 | 114 |
Functions,'' describes how to specify corecursive functions using the |
53826 | 115 |
@{command primcorec} and @{command primcorecursive} commands. |
52794 | 116 |
|
55351 | 117 |
\item Section \ref{sec:introducing-bounded-natural-functors}, ``Introducing |
53552 | 118 |
Bounded Natural Functors,'' explains how to use the @{command bnf} command |
119 |
to register arbitrary type constructors as BNFs. |
|
52805 | 120 |
|
53552 | 121 |
\item Section |
53617 | 122 |
\ref{sec:deriving-destructors-and-theorems-for-free-constructors}, |
123 |
``Deriving Destructors and Theorems for Free Constructors,'' explains how to |
|
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55460
diff
changeset
|
124 |
use the command @{command free_constructors} to derive destructor constants |
53552 | 125 |
and theorems for freely generated types, as performed internally by @{command |
53829 | 126 |
datatype_new} and @{command codatatype}. |
52794 | 127 |
|
53617 | 128 |
%\item Section \ref{sec:standard-ml-interface}, ``Standard ML Interface,'' |
129 |
%describes the package's programmatic interface. |
|
52794 | 130 |
|
53617 | 131 |
%\item Section \ref{sec:interoperability}, ``Interoperability,'' |
132 |
%is concerned with the packages' interaction with other Isabelle packages and |
|
133 |
%tools, such as the code generator and the counterexample generators. |
|
52805 | 134 |
|
53617 | 135 |
%\item Section \ref{sec:known-bugs-and-limitations}, ``Known Bugs and |
136 |
%Limitations,'' concludes with known open issues at the time of writing. |
|
52805 | 137 |
\end{itemize} |
52822 | 138 |
|
139 |
||
140 |
\newbox\boxA |
|
54185 | 141 |
\setbox\boxA=\hbox{\texttt{NOSPAM}} |
142 |
||
143 |
\newcommand\authoremaili{\texttt{blan{\color{white}NOSPAM}\kern-\wd\boxA{}chette@\allowbreak |
|
52822 | 144 |
in.\allowbreak tum.\allowbreak de}} |
57079 | 145 |
\newcommand\authoremailii{\texttt{desh{\color{white}NOSPAM}\kern-\wd\boxA{}arna@\allowbreak |
146 |
in.\allowbreak tum.\allowbreak de}} |
|
147 |
\newcommand\authoremailiii{\texttt{lore{\color{white}NOSPAM}\kern-\wd\boxA{}nz.panny@\allowbreak |
|
52822 | 148 |
in.\allowbreak tum.\allowbreak de}} |
57079 | 149 |
\newcommand\authoremailiv{\texttt{pope{\color{white}NOSPAM}\kern-\wd\boxA{}scua@\allowbreak |
150 |
in.\allowbreak tum.\allowbreak de}} |
|
151 |
\newcommand\authoremailv{\texttt{tray{\color{white}NOSPAM}\kern-\wd\boxA{}tel@\allowbreak |
|
52822 | 152 |
in.\allowbreak tum.\allowbreak de}} |
153 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
154 |
The command @{command datatype_new} is expected to replace \keyw{datatype} in a |
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
155 |
future release. Authors of new theories are encouraged to use the new commands, |
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
156 |
and maintainers of older theories may want to consider upgrading. |
52841 | 157 |
|
158 |
Comments and bug reports concerning either the tool or this tutorial should be |
|
53028 | 159 |
directed to the authors at \authoremaili, \authoremailii, \authoremailiii, |
57079 | 160 |
\authoremailiv, and \authoremailv. |
52794 | 161 |
*} |
162 |
||
53491 | 163 |
|
52827 | 164 |
section {* Defining Datatypes |
52805 | 165 |
\label{sec:defining-datatypes} *} |
166 |
||
167 |
text {* |
|
53646 | 168 |
Datatypes can be specified using the @{command datatype_new} command. |
52805 | 169 |
*} |
52792 | 170 |
|
52824 | 171 |
|
53617 | 172 |
subsection {* Introductory Examples |
173 |
\label{ssec:datatype-introductory-examples} *} |
|
52794 | 174 |
|
53646 | 175 |
text {* |
176 |
Datatypes are illustrated through concrete examples featuring different flavors |
|
177 |
of recursion. More examples can be found in the directory |
|
54185 | 178 |
\verb|~~/src/HOL/|\allowbreak\verb|BNF/Examples|. |
53646 | 179 |
*} |
53621 | 180 |
|
181 |
subsubsection {* Nonrecursive Types |
|
182 |
\label{sssec:datatype-nonrecursive-types} *} |
|
52794 | 183 |
|
52805 | 184 |
text {* |
53028 | 185 |
Datatypes are introduced by specifying the desired names and argument types for |
53491 | 186 |
their constructors. \emph{Enumeration} types are the simplest form of datatype. |
53028 | 187 |
All their constructors are nullary: |
52805 | 188 |
*} |
189 |
||
52828 | 190 |
datatype_new trool = Truue | Faalse | Perhaaps |
52805 | 191 |
|
192 |
text {* |
|
53028 | 193 |
\noindent |
53491 | 194 |
Here, @{const Truue}, @{const Faalse}, and @{const Perhaaps} have the type @{typ trool}. |
53028 | 195 |
|
196 |
Polymorphic types are possible, such as the following option type, modeled after |
|
197 |
its homologue from the @{theory Option} theory: |
|
52805 | 198 |
*} |
199 |
||
53025 | 200 |
(*<*) |
56995 | 201 |
hide_const None Some map_option |
54958
4933165fd112
do not use wrong constructor in auto-generated proof goal
panny
parents:
54955
diff
changeset
|
202 |
hide_type option |
53025 | 203 |
(*>*) |
204 |
datatype_new 'a option = None | Some 'a |
|
52805 | 205 |
|
206 |
text {* |
|
53028 | 207 |
\noindent |
53491 | 208 |
The constructors are @{text "None :: 'a option"} and |
209 |
@{text "Some :: 'a \<Rightarrow> 'a option"}. |
|
53028 | 210 |
|
211 |
The next example has three type parameters: |
|
52805 | 212 |
*} |
213 |
||
214 |
datatype_new ('a, 'b, 'c) triple = Triple 'a 'b 'c |
|
215 |
||
53028 | 216 |
text {* |
217 |
\noindent |
|
218 |
The constructor is |
|
53491 | 219 |
@{text "Triple :: 'a \<Rightarrow> 'b \<Rightarrow> 'c \<Rightarrow> ('a, 'b, 'c) triple"}. |
53028 | 220 |
Unlike in Standard ML, curried constructors are supported. The uncurried variant |
221 |
is also possible: |
|
222 |
*} |
|
223 |
||
224 |
datatype_new ('a, 'b, 'c) triple\<^sub>u = Triple\<^sub>u "'a * 'b * 'c" |
|
225 |
||
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
226 |
text {* |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
227 |
\noindent |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
228 |
Occurrences of nonatomic types on the right-hand side of the equal sign must be |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
229 |
enclosed in double quotes, as is customary in Isabelle. |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
230 |
*} |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
231 |
|
52824 | 232 |
|
53621 | 233 |
subsubsection {* Simple Recursion |
234 |
\label{sssec:datatype-simple-recursion} *} |
|
52794 | 235 |
|
52805 | 236 |
text {* |
53491 | 237 |
Natural numbers are the simplest example of a recursive type: |
52805 | 238 |
*} |
239 |
||
53332 | 240 |
datatype_new nat = Zero | Suc nat |
52805 | 241 |
|
242 |
text {* |
|
53491 | 243 |
\noindent |
54187 | 244 |
Lists were shown in the introduction. Terminated lists are a variant that |
245 |
stores a value of type @{typ 'b} at the very end: |
|
52805 | 246 |
*} |
247 |
||
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
248 |
datatype_new (*<*)(in early) (*>*)('a, 'b) tlist = TNil 'b | TCons 'a "('a, 'b) tlist" |
52805 | 249 |
|
52824 | 250 |
|
53621 | 251 |
subsubsection {* Mutual Recursion |
252 |
\label{sssec:datatype-mutual-recursion} *} |
|
52794 | 253 |
|
52805 | 254 |
text {* |
53552 | 255 |
\emph{Mutually recursive} types are introduced simultaneously and may refer to |
256 |
each other. The example below introduces a pair of types for even and odd |
|
257 |
natural numbers: |
|
52805 | 258 |
*} |
259 |
||
53623 | 260 |
datatype_new even_nat = Even_Zero | Even_Suc odd_nat |
261 |
and odd_nat = Odd_Suc even_nat |
|
52805 | 262 |
|
263 |
text {* |
|
53491 | 264 |
\noindent |
265 |
Arithmetic expressions are defined via terms, terms via factors, and factors via |
|
266 |
expressions: |
|
52805 | 267 |
*} |
268 |
||
52841 | 269 |
datatype_new ('a, 'b) exp = |
270 |
Term "('a, 'b) trm" | Sum "('a, 'b) trm" "('a, 'b) exp" |
|
52805 | 271 |
and ('a, 'b) trm = |
52841 | 272 |
Factor "('a, 'b) fct" | Prod "('a, 'b) fct" "('a, 'b) trm" |
273 |
and ('a, 'b) fct = |
|
274 |
Const 'a | Var 'b | Expr "('a, 'b) exp" |
|
52805 | 275 |
|
52824 | 276 |
|
53621 | 277 |
subsubsection {* Nested Recursion |
278 |
\label{sssec:datatype-nested-recursion} *} |
|
52794 | 279 |
|
52805 | 280 |
text {* |
53491 | 281 |
\emph{Nested recursion} occurs when recursive occurrences of a type appear under |
282 |
a type constructor. The introduction showed some examples of trees with nesting |
|
53675 | 283 |
through lists. A more complex example, that reuses our @{type option} type, |
53491 | 284 |
follows: |
52805 | 285 |
*} |
286 |
||
52843 | 287 |
datatype_new 'a btree = |
53025 | 288 |
BNode 'a "'a btree option" "'a btree option" |
52805 | 289 |
|
290 |
text {* |
|
53491 | 291 |
\noindent |
292 |
Not all nestings are admissible. For example, this command will fail: |
|
52805 | 293 |
*} |
294 |
||
54187 | 295 |
datatype_new 'a wrong = W1 | W2 (*<*)'a |
53542 | 296 |
typ (*>*)"'a wrong \<Rightarrow> 'a" |
52806 | 297 |
|
298 |
text {* |
|
53491 | 299 |
\noindent |
300 |
The issue is that the function arrow @{text "\<Rightarrow>"} allows recursion |
|
301 |
only through its right-hand side. This issue is inherited by polymorphic |
|
302 |
datatypes defined in terms of~@{text "\<Rightarrow>"}: |
|
303 |
*} |
|
304 |
||
55350 | 305 |
datatype_new ('a, 'b) fun_copy = Fun "'a \<Rightarrow> 'b" |
54187 | 306 |
datatype_new 'a also_wrong = W1 | W2 (*<*)'a |
55350 | 307 |
typ (*>*)"('a also_wrong, 'a) fun_copy" |
53491 | 308 |
|
309 |
text {* |
|
310 |
\noindent |
|
55129
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
311 |
The following definition of @{typ 'a}-branching trees is legal: |
53621 | 312 |
*} |
313 |
||
314 |
datatype_new 'a ftree = FTLeaf 'a | FTNode "'a \<Rightarrow> 'a ftree" |
|
315 |
||
316 |
text {* |
|
317 |
\noindent |
|
55129
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
318 |
And so is the definition of hereditarily finite sets: |
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
319 |
*} |
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
320 |
|
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
321 |
datatype_new hfset = HFSet "hfset fset" |
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
322 |
|
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
323 |
text {* |
26bd1cba3ab5
killed 'More_BNFs' by moving its various bits where they (now) belong
blanchet
parents:
55114
diff
changeset
|
324 |
\noindent |
53491 | 325 |
In general, type constructors @{text "('a\<^sub>1, \<dots>, 'a\<^sub>m) t"} |
326 |
allow recursion on a subset of their type arguments @{text 'a\<^sub>1}, \ldots, |
|
327 |
@{text 'a\<^sub>m}. These type arguments are called \emph{live}; the remaining |
|
328 |
type arguments are called \emph{dead}. In @{typ "'a \<Rightarrow> 'b"} and |
|
55350 | 329 |
@{typ "('a, 'b) fun_copy"}, the type variable @{typ 'a} is dead and |
330 |
@{typ 'b} is live. |
|
53552 | 331 |
|
53647 | 332 |
Type constructors must be registered as BNFs to have live arguments. This is |
333 |
done automatically for datatypes and codatatypes introduced by the @{command |
|
53829 | 334 |
datatype_new} and @{command codatatype} commands. |
55351 | 335 |
Section~\ref{sec:introducing-bounded-natural-functors} explains how to |
336 |
register arbitrary type constructors as BNFs. |
|
54187 | 337 |
|
338 |
Here is another example that fails: |
|
52806 | 339 |
*} |
340 |
||
54187 | 341 |
datatype_new 'a pow_list = PNil 'a (*<*)'a |
342 |
datatype_new 'a pow_list' = PNil' 'a (*>*)| PCons "('a * 'a) pow_list" |
|
343 |
||
344 |
text {* |
|
345 |
\noindent |
|
55351 | 346 |
This attempted definition features a different flavor of nesting, where the |
347 |
recursive call in the type specification occurs around (rather than inside) |
|
348 |
another type constructor. |
|
54187 | 349 |
*} |
350 |
||
351 |
subsubsection {* Auxiliary Constants and Properties |
|
352 |
\label{sssec:datatype-auxiliary-constants-and-properties} *} |
|
52805 | 353 |
|
354 |
text {* |
|
53491 | 355 |
The @{command datatype_new} command introduces various constants in addition to |
53617 | 356 |
the constructors. With each datatype are associated set functions, a map |
357 |
function, a relator, discriminators, and selectors, all of which can be given |
|
54187 | 358 |
custom names. In the example below, the familiar names @{text null}, @{text hd}, |
359 |
@{text tl}, @{text set}, @{text map}, and @{text list_all2}, override the |
|
360 |
default names @{text is_Nil}, @{text un_Cons1}, @{text un_Cons2}, |
|
54491 | 361 |
@{text set_list}, @{text map_list}, and @{text rel_list}: |
52822 | 362 |
*} |
363 |
||
52841 | 364 |
(*<*) |
365 |
no_translations |
|
366 |
"[x, xs]" == "x # [xs]" |
|
367 |
"[x]" == "x # []" |
|
368 |
||
369 |
no_notation |
|
370 |
Nil ("[]") and |
|
371 |
Cons (infixr "#" 65) |
|
372 |
||
53543 | 373 |
hide_type list |
56995 | 374 |
hide_const Nil Cons hd tl set map list_all2 rec_list size_list |
53025 | 375 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
376 |
context early begin |
52841 | 377 |
(*>*) |
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
378 |
datatype_new (set: 'a) list = |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
379 |
null: Nil |
53025 | 380 |
| Cons (hd: 'a) (tl: "'a list") |
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
381 |
for |
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
382 |
map: map |
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
383 |
rel: list_all2 |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
384 |
where |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
385 |
"tl Nil = Nil" |
52822 | 386 |
|
387 |
text {* |
|
388 |
\noindent |
|
55353 | 389 |
The types of the constants that appear in the specification are listed below. |
55351 | 390 |
|
391 |
\medskip |
|
54187 | 392 |
|
393 |
\begin{tabular}{@ {}ll@ {}} |
|
394 |
Constructors: & |
|
395 |
@{text "Nil \<Colon> 'a list"} \\ |
|
396 |
& |
|
397 |
@{text "Cons \<Colon> 'a \<Rightarrow> 'a list \<Rightarrow> 'a list"} \\ |
|
398 |
Discriminator: & |
|
399 |
@{text "null \<Colon> 'a list \<Rightarrow> bool"} \\ |
|
400 |
Selectors: & |
|
401 |
@{text "hd \<Colon> 'a list \<Rightarrow> 'a"} \\ |
|
402 |
& |
|
403 |
@{text "tl \<Colon> 'a list \<Rightarrow> 'a list"} \\ |
|
404 |
Set function: & |
|
405 |
@{text "set \<Colon> 'a list \<Rightarrow> 'a set"} \\ |
|
406 |
Map function: & |
|
407 |
@{text "map \<Colon> ('a \<Rightarrow> 'b) \<Rightarrow> 'a list \<Rightarrow> 'b list"} \\ |
|
408 |
Relator: & |
|
409 |
@{text "list_all2 \<Colon> ('a \<Rightarrow> 'b \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> 'b list \<Rightarrow> bool"} |
|
410 |
\end{tabular} |
|
411 |
||
55351 | 412 |
\medskip |
413 |
||
54187 | 414 |
The discriminator @{const null} and the selectors @{const hd} and @{const tl} |
55351 | 415 |
are characterized by the following conditional equations: |
52822 | 416 |
% |
53025 | 417 |
\[@{thm list.collapse(1)[of xs, no_vars]} |
418 |
\qquad @{thm list.collapse(2)[of xs, no_vars]}\] |
|
52822 | 419 |
% |
54187 | 420 |
For two-constructor datatypes, a single discriminator constant is sufficient. |
421 |
The discriminator associated with @{const Cons} is simply |
|
53491 | 422 |
@{term "\<lambda>xs. \<not> null xs"}. |
52822 | 423 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
424 |
The \keyw{where} clause at the end of the command specifies a default value for |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
425 |
selectors applied to constructors on which they are not a priori specified. |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
426 |
Here, it is used to ensure that the tail of the empty list is itself (instead of |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
427 |
being left unspecified). |
52822 | 428 |
|
53617 | 429 |
Because @{const Nil} is nullary, it is also possible to use |
57091 | 430 |
@{term "\<lambda>xs. xs = Nil"} as a discriminator. This is the default behavior |
431 |
if we omit the identifier @{const null} and the associated colon. Some users |
|
432 |
argue against this, because the mixture of constructors and selectors in the |
|
433 |
characteristic theorems can lead Isabelle's automation to switch between the |
|
434 |
constructor and the destructor view in surprising ways. |
|
52822 | 435 |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
436 |
The usual mixfix syntax annotations are available for both types and |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
437 |
constructors. For example: |
52805 | 438 |
*} |
52794 | 439 |
|
53025 | 440 |
(*<*) |
441 |
end |
|
442 |
(*>*) |
|
53552 | 443 |
datatype_new ('a, 'b) prod (infixr "*" 20) = Pair 'a 'b |
444 |
||
445 |
text {* \blankline *} |
|
52822 | 446 |
|
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
447 |
datatype_new (set: 'a) list = |
52822 | 448 |
null: Nil ("[]") |
52841 | 449 |
| Cons (hd: 'a) (tl: "'a list") (infixr "#" 65) |
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
450 |
for |
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
451 |
map: map |
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
452 |
rel: list_all2 |
52841 | 453 |
|
454 |
text {* |
|
53535 | 455 |
\noindent |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
456 |
Incidentally, this is how the traditional syntax can be set up: |
52841 | 457 |
*} |
458 |
||
459 |
syntax "_list" :: "args \<Rightarrow> 'a list" ("[(_)]") |
|
460 |
||
53552 | 461 |
text {* \blankline *} |
462 |
||
52841 | 463 |
translations |
464 |
"[x, xs]" == "x # [xs]" |
|
465 |
"[x]" == "x # []" |
|
52822 | 466 |
|
52824 | 467 |
|
53617 | 468 |
subsection {* Command Syntax |
469 |
\label{ssec:datatype-command-syntax} *} |
|
470 |
||
471 |
||
57542 | 472 |
subsubsection {* \keyw{datatype_new} |
53621 | 473 |
\label{sssec:datatype-new} *} |
52794 | 474 |
|
52822 | 475 |
text {* |
53829 | 476 |
\begin{matharray}{rcl} |
477 |
@{command_def "datatype_new"} & : & @{text "local_theory \<rightarrow> local_theory"} |
|
478 |
\end{matharray} |
|
52822 | 479 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
480 |
@{rail \<open> |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54958
diff
changeset
|
481 |
@@{command datatype_new} target? @{syntax dt_options}? \<newline> |
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
482 |
(@{syntax dt_name} '=' (@{syntax dt_ctor} + '|') \<newline> |
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
483 |
@{syntax map_rel}? (@'where' (prop + '|'))? + @'and') |
52828 | 484 |
; |
57094
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57092
diff
changeset
|
485 |
@{syntax_def dt_options}: '(' (('discs_sels' | 'no_code') + ',') ')' |
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
486 |
; |
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
487 |
@{syntax_def map_rel}: @'for' ((('map' | 'rel') ':' name) +) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
488 |
\<close>} |
52824 | 489 |
|
55351 | 490 |
\medskip |
491 |
||
492 |
\noindent |
|
55460
3f4efd7d950d
added a bit of documentation for the different commands
blanchet
parents:
55459
diff
changeset
|
493 |
The @{command datatype_new} command introduces a set of mutually recursive |
3f4efd7d950d
added a bit of documentation for the different commands
blanchet
parents:
55459
diff
changeset
|
494 |
datatypes specified by their constructors. |
3f4efd7d950d
added a bit of documentation for the different commands
blanchet
parents:
55459
diff
changeset
|
495 |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
496 |
The syntactic entity \synt{target} can be used to specify a local |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
497 |
context (e.g., @{text "(in linorder)"} \cite{isabelle-isar-ref}), |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
498 |
and \synt{prop} denotes a HOL proposition. |
55460
3f4efd7d950d
added a bit of documentation for the different commands
blanchet
parents:
55459
diff
changeset
|
499 |
|
56124 | 500 |
The optional target is optionally followed by one or both of the following |
501 |
options: |
|
52822 | 502 |
|
52824 | 503 |
\begin{itemize} |
504 |
\setlength{\itemsep}{0pt} |
|
505 |
||
506 |
\item |
|
57094
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57092
diff
changeset
|
507 |
The @{text "discs_sels"} option indicates that discriminators and selectors |
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57092
diff
changeset
|
508 |
should be generated. The option is implicitly enabled if names are specified for |
589ec121ce1a
don't generate discriminators and selectors for 'datatype_new' unless the user asked for it
blanchet
parents:
57092
diff
changeset
|
509 |
discriminators or selectors. |
52822 | 510 |
|
52824 | 511 |
\item |
54626 | 512 |
The @{text "no_code"} option indicates that the datatype should not be |
513 |
registered for code generation. |
|
52824 | 514 |
\end{itemize} |
52822 | 515 |
|
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
516 |
The optional \keyw{where} clause specifies default values for selectors. |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
517 |
Each proposition must be an equation of the form |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
518 |
@{text "un_D (C \<dots>) = \<dots>"}, where @{text C} is a constructor and |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
519 |
@{text un_D} is a selector. |
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
520 |
|
52827 | 521 |
The left-hand sides of the datatype equations specify the name of the type to |
53534 | 522 |
define, its type parameters, and additional information: |
52822 | 523 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
524 |
@{rail \<open> |
57206
d9be905d6283
changed syntax of map: and rel: arguments to BNF-based datatypes
blanchet
parents:
57200
diff
changeset
|
525 |
@{syntax_def dt_name}: @{syntax tyargs}? name mixfix? |
52824 | 526 |
; |
57092 | 527 |
@{syntax_def tyargs}: typefree | '(' (('dead' | name ':')? typefree + ',') ')' |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
528 |
\<close>} |
52822 | 529 |
|
55351 | 530 |
\medskip |
531 |
||
52827 | 532 |
\noindent |
55474 | 533 |
The syntactic entity \synt{name} denotes an identifier, \synt{mixfix} denotes |
534 |
the usual parenthesized mixfix notation, and \synt{typefree} denotes fixed type |
|
535 |
variable (@{typ 'a}, @{typ 'b}, \ldots) \cite{isabelle-isar-ref}. |
|
52822 | 536 |
|
52827 | 537 |
The optional names preceding the type variables allow to override the default |
57988 | 538 |
names of the set functions (@{text set\<^sub>1_t}, \ldots, @{text set\<^sub>m_t}). Type |
57092 | 539 |
arguments can be marked as dead by entering ``@{text dead}'' in front of the |
540 |
type variable (e.g., ``@{text "(dead 'a)"}''); otherwise, they are live or dead |
|
55705 | 541 |
(and a set function is generated or not) depending on where they occur in the |
542 |
right-hand sides of the definition. Declaring a type argument as dead can speed |
|
543 |
up the type definition but will prevent any later (co)recursion through that |
|
544 |
type argument. |
|
545 |
||
53647 | 546 |
Inside a mutually recursive specification, all defined datatypes must |
547 |
mention exactly the same type variables in the same order. |
|
52822 | 548 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
549 |
@{rail \<open> |
57200
aab87ffa60cc
use 'where' clause for selector default value syntax
blanchet
parents:
57153
diff
changeset
|
550 |
@{syntax_def dt_ctor}: (name ':')? name (@{syntax dt_ctor_arg} * ) mixfix? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
551 |
\<close>} |
52824 | 552 |
|
53535 | 553 |
\medskip |
554 |
||
52827 | 555 |
\noindent |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
556 |
The main constituents of a constructor specification are the name of the |
52827 | 557 |
constructor and the list of its argument types. An optional discriminator name |
57091 | 558 |
can be supplied at the front to override the default, which is |
559 |
@{text "\<lambda>x. x = C\<^sub>j"} for nullary constructors and |
|
560 |
@{text t.is_C\<^sub>j} otherwise. |
|
52822 | 561 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
562 |
@{rail \<open> |
55472
990651bfc65b
updated docs to reflect the new 'free_constructors' syntax
blanchet
parents:
55468
diff
changeset
|
563 |
@{syntax_def dt_ctor_arg}: type | '(' name ':' type ')' |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
564 |
\<close>} |
52827 | 565 |
|
53535 | 566 |
\medskip |
567 |
||
52827 | 568 |
\noindent |
55474 | 569 |
The syntactic entity \synt{type} denotes a HOL type \cite{isabelle-isar-ref}. |
570 |
||
52827 | 571 |
In addition to the type of a constructor argument, it is possible to specify a |
572 |
name for the corresponding selector to override the default name |
|
53554 | 573 |
(@{text un_C\<^sub>ji}). The same selector names can be reused for several |
574 |
constructors as long as they share the same type. |
|
52822 | 575 |
*} |
576 |
||
53617 | 577 |
|
57542 | 578 |
subsubsection {* \keyw{datatype_compat} |
56644 | 579 |
\label{sssec:datatype-compat} *} |
53617 | 580 |
|
581 |
text {* |
|
53829 | 582 |
\begin{matharray}{rcl} |
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
583 |
@{command_def "datatype_compat"} & : & @{text "local_theory \<rightarrow> local_theory"} |
53829 | 584 |
\end{matharray} |
585 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
586 |
@{rail \<open> |
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
587 |
@@{command datatype_compat} (name +) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
588 |
\<close>} |
53829 | 589 |
|
55351 | 590 |
\medskip |
591 |
||
53829 | 592 |
\noindent |
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
593 |
The @{command datatype_compat} command registers new-style datatypes as |
55474 | 594 |
old-style datatypes. For example: |
53621 | 595 |
*} |
596 |
||
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
597 |
datatype_compat even_nat odd_nat |
53621 | 598 |
|
599 |
text {* \blankline *} |
|
600 |
||
53623 | 601 |
ML {* Datatype_Data.get_info @{theory} @{type_name even_nat} *} |
53621 | 602 |
|
603 |
text {* |
|
55474 | 604 |
The syntactic entity \synt{name} denotes an identifier \cite{isabelle-isar-ref}. |
605 |
||
606 |
The command is interesting because the old datatype package provides some |
|
56655 | 607 |
functionality that is not yet replicated in the new package, such as the |
608 |
integration with Quickcheck. |
|
55474 | 609 |
|
610 |
A few remarks concern nested recursive datatypes: |
|
53748 | 611 |
|
612 |
\begin{itemize} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
613 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
614 |
|
55871 | 615 |
\item The old-style, nested-as-mutual induction rule and recursor theorems are |
616 |
generated under their usual names but with ``@{text "compat_"}'' prefixed |
|
617 |
(e.g., @{text compat_tree.induct}). |
|
53748 | 618 |
|
619 |
\item All types through which recursion takes place must be new-style datatypes |
|
620 |
or the function type. In principle, it should be possible to support old-style |
|
55474 | 621 |
datatypes as well, but this has not been implemented yet (and there is currently |
622 |
no way to register old-style datatypes as new-style datatypes). |
|
54184 | 623 |
|
624 |
\item The recursor produced for types that recurse through functions has a |
|
56655 | 625 |
different signature than with the old package. This might affect the behavior of |
626 |
some third-party extensions. |
|
53748 | 627 |
\end{itemize} |
628 |
||
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
629 |
An alternative to @{command datatype_compat} is to use the old package's |
57542 | 630 |
\keyw{rep_\allowbreak datatype} command. The associated proof obligations must then be |
53748 | 631 |
discharged manually. |
53617 | 632 |
*} |
633 |
||
634 |
||
635 |
subsection {* Generated Constants |
|
636 |
\label{ssec:datatype-generated-constants} *} |
|
637 |
||
638 |
text {* |
|
53623 | 639 |
Given a datatype @{text "('a\<^sub>1, \<dots>, 'a\<^sub>m) t"} |
53617 | 640 |
with $m > 0$ live type variables and $n$ constructors |
641 |
@{text "t.C\<^sub>1"}, \ldots, @{text "t.C\<^sub>n"}, the |
|
642 |
following auxiliary constants are introduced: |
|
643 |
||
55353 | 644 |
\medskip |
645 |
||
646 |
\begin{tabular}{@ {}ll@ {}} |
|
647 |
Case combinator: & |
|
648 |
@{text t.case_t} (rendered using the familiar @{text case}--@{text of} syntax) \\ |
|
649 |
Discriminators: & |
|
57988 | 650 |
@{text t.is_C\<^sub>1}$, \ldots, $@{text t.is_C\<^sub>n} \\ |
55353 | 651 |
Selectors: & |
652 |
@{text t.un_C\<^sub>11}$, \ldots, $@{text t.un_C\<^sub>1k\<^sub>1} \\ |
|
653 |
& \quad\vdots \\ |
|
654 |
& @{text t.un_C\<^sub>n1}$, \ldots, $@{text t.un_C\<^sub>nk\<^sub>n} \\ |
|
655 |
Set functions: & |
|
57988 | 656 |
@{text t.set\<^sub>1_t}, \ldots, @{text t.set\<^sub>m_t} \\ |
55353 | 657 |
Map function: & |
658 |
@{text t.map_t} \\ |
|
659 |
Relator: & |
|
660 |
@{text t.rel_t} \\ |
|
661 |
Recursor: & |
|
56655 | 662 |
@{text t.rec_t} \\ |
663 |
Size function: & |
|
664 |
@{text t.size_t} |
|
55353 | 665 |
\end{tabular} |
666 |
||
667 |
\medskip |
|
53617 | 668 |
|
669 |
\noindent |
|
670 |
The case combinator, discriminators, and selectors are collectively called |
|
671 |
\emph{destructors}. The prefix ``@{text "t."}'' is an optional component of the |
|
54491 | 672 |
names and is normally hidden. |
56655 | 673 |
|
674 |
In addition to the above, the @{class size} class is instantiated to overload the |
|
675 |
@{const size} function based on @{text t.size_t}. |
|
53617 | 676 |
*} |
677 |
||
678 |
||
52840 | 679 |
subsection {* Generated Theorems |
680 |
\label{ssec:datatype-generated-theorems} *} |
|
52828 | 681 |
|
682 |
text {* |
|
53544 | 683 |
The characteristic theorems generated by @{command datatype_new} are grouped in |
53623 | 684 |
three broad categories: |
53535 | 685 |
|
53543 | 686 |
\begin{itemize} |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
687 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
688 |
|
56655 | 689 |
\item The \emph{free constructor theorems} |
690 |
(Section~\ref{sssec:free-constructor-theorems}) are properties of the |
|
691 |
constructors and destructors that can be derived for any freely generated type. |
|
692 |
Internally, the derivation is performed by @{command free_constructors}. |
|
693 |
||
694 |
\item The \emph{functorial theorems} (Section~\ref{sssec:functorial-theorems}) |
|
695 |
are properties of datatypes related to their BNF nature. |
|
696 |
||
697 |
\item The \emph{inductive theorems} (Section~\ref{sssec:inductive-theorems}) |
|
698 |
are properties of datatypes related to their inductive nature. |
|
53552 | 699 |
|
53543 | 700 |
\end{itemize} |
53535 | 701 |
|
702 |
\noindent |
|
53542 | 703 |
The full list of named theorems can be obtained as usual by entering the |
57542 | 704 |
command \keyw{print_theorems} immediately after the datatype definition. |
53542 | 705 |
This list normally excludes low-level theorems that reveal internal |
53552 | 706 |
constructions. To make these accessible, add the line |
53542 | 707 |
*} |
53535 | 708 |
|
53542 | 709 |
declare [[bnf_note_all]] |
710 |
(*<*) |
|
711 |
declare [[bnf_note_all = false]] |
|
712 |
(*>*) |
|
53535 | 713 |
|
53552 | 714 |
text {* |
715 |
\noindent |
|
716 |
to the top of the theory file. |
|
717 |
*} |
|
53535 | 718 |
|
53621 | 719 |
subsubsection {* Free Constructor Theorems |
720 |
\label{sssec:free-constructor-theorems} *} |
|
53535 | 721 |
|
53543 | 722 |
(*<*) |
53837 | 723 |
consts nonnull :: 'a |
53543 | 724 |
(*>*) |
725 |
||
53535 | 726 |
text {* |
54621 | 727 |
The free constructor theorems are partitioned in three subgroups. The first |
728 |
subgroup of properties is concerned with the constructors. They are listed below |
|
729 |
for @{typ "'a list"}: |
|
53543 | 730 |
|
53552 | 731 |
\begin{indentblock} |
53543 | 732 |
\begin{description} |
53544 | 733 |
|
53642 | 734 |
\item[@{text "t."}\hthm{inject} @{text "[iff, induct_simp]"}\rm:] ~ \\ |
53544 | 735 |
@{thm list.inject[no_vars]} |
736 |
||
53642 | 737 |
\item[@{text "t."}\hthm{distinct} @{text "[simp, induct_simp]"}\rm:] ~ \\ |
53543 | 738 |
@{thm list.distinct(1)[no_vars]} \\ |
739 |
@{thm list.distinct(2)[no_vars]} |
|
740 |
||
53642 | 741 |
\item[@{text "t."}\hthm{exhaust} @{text "[cases t, case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
53543 | 742 |
@{thm list.exhaust[no_vars]} |
743 |
||
53642 | 744 |
\item[@{text "t."}\hthm{nchotomy}\rm:] ~ \\ |
53543 | 745 |
@{thm list.nchotomy[no_vars]} |
746 |
||
747 |
\end{description} |
|
53552 | 748 |
\end{indentblock} |
53543 | 749 |
|
750 |
\noindent |
|
53621 | 751 |
In addition, these nameless theorems are registered as safe elimination rules: |
752 |
||
753 |
\begin{indentblock} |
|
754 |
\begin{description} |
|
755 |
||
54386 | 756 |
\item[@{text "t."}\hthm{distinct {\upshape[}THEN notE}@{text ", elim!"}\hthm{\upshape]}\rm:] ~ \\ |
53621 | 757 |
@{thm list.distinct(1)[THEN notE, elim!, no_vars]} \\ |
758 |
@{thm list.distinct(2)[THEN notE, elim!, no_vars]} |
|
759 |
||
760 |
\end{description} |
|
761 |
\end{indentblock} |
|
762 |
||
763 |
\noindent |
|
53543 | 764 |
The next subgroup is concerned with the case combinator: |
765 |
||
53552 | 766 |
\begin{indentblock} |
53543 | 767 |
\begin{description} |
53544 | 768 |
|
53798 | 769 |
\item[@{text "t."}\hthm{case} @{text "[simp, code]"}\rm:] ~ \\ |
53543 | 770 |
@{thm list.case(1)[no_vars]} \\ |
771 |
@{thm list.case(2)[no_vars]} |
|
772 |
||
57542 | 773 |
\item[@{text "t."}\hthm{case_cong} @{text "[fundef_cong]"}\rm:] ~ \\ |
53543 | 774 |
@{thm list.case_cong[no_vars]} |
775 |
||
57983
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
776 |
\item[@{text "t."}\hthm{case_cong_weak} @{text "[cong]"}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
777 |
@{thm list.case_cong_weak[no_vars]} |
53543 | 778 |
|
53642 | 779 |
\item[@{text "t."}\hthm{split}\rm:] ~ \\ |
53543 | 780 |
@{thm list.split[no_vars]} |
781 |
||
57542 | 782 |
\item[@{text "t."}\hthm{split_asm}\rm:] ~ \\ |
53543 | 783 |
@{thm list.split_asm[no_vars]} |
784 |
||
53544 | 785 |
\item[@{text "t."}\hthm{splits} = @{text "split split_asm"}] |
53543 | 786 |
|
787 |
\end{description} |
|
53552 | 788 |
\end{indentblock} |
53543 | 789 |
|
790 |
\noindent |
|
54621 | 791 |
The third subgroup revolves around discriminators and selectors: |
53543 | 792 |
|
53552 | 793 |
\begin{indentblock} |
53543 | 794 |
\begin{description} |
53544 | 795 |
|
53694 | 796 |
\item[@{text "t."}\hthm{disc} @{text "[simp]"}\rm:] ~ \\ |
797 |
@{thm list.disc(1)[no_vars]} \\ |
|
798 |
@{thm list.disc(2)[no_vars]} |
|
799 |
||
53703 | 800 |
\item[@{text "t."}\hthm{discI}\rm:] ~ \\ |
801 |
@{thm list.discI(1)[no_vars]} \\ |
|
802 |
@{thm list.discI(2)[no_vars]} |
|
803 |
||
53805 | 804 |
\item[@{text "t."}\hthm{sel} @{text "[simp, code]"}\rm:] ~ \\ |
53694 | 805 |
@{thm list.sel(1)[no_vars]} \\ |
806 |
@{thm list.sel(2)[no_vars]} |
|
53543 | 807 |
|
53642 | 808 |
\item[@{text "t."}\hthm{collapse} @{text "[simp]"}\rm:] ~ \\ |
53543 | 809 |
@{thm list.collapse(1)[no_vars]} \\ |
810 |
@{thm list.collapse(2)[no_vars]} |
|
811 |
||
57983
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
812 |
\item[@{text "t."}\hthm{distinct_disc} @{text "[dest]"}\rm:] ~ \\ |
53543 | 813 |
These properties are missing for @{typ "'a list"} because there is only one |
814 |
proper discriminator. Had the datatype been introduced with a second |
|
53837 | 815 |
discriminator called @{const nonnull}, they would have read thusly: \\[\jot] |
816 |
@{prop "null list \<Longrightarrow> \<not> nonnull list"} \\ |
|
817 |
@{prop "nonnull list \<Longrightarrow> \<not> null list"} |
|
53543 | 818 |
|
57983
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
819 |
\item[@{text "t."}\hthm{exhaust_disc} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
820 |
@{thm list.exhaust_disc[no_vars]} |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
821 |
|
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
822 |
\item[@{text "t."}\hthm{exhaust_sel} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
823 |
@{thm list.exhaust_sel[no_vars]} |
53916 | 824 |
|
53642 | 825 |
\item[@{text "t."}\hthm{expand}\rm:] ~ \\ |
53543 | 826 |
@{thm list.expand[no_vars]} |
827 |
||
57983
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
828 |
\item[@{text "t."}\hthm{split_sel}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
829 |
@{thm list.split_sel[no_vars]} |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
830 |
|
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
831 |
\item[@{text "t."}\hthm{split_sel_asm}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
832 |
@{thm list.split_sel_asm[no_vars]} |
53917 | 833 |
|
57984
cbe9a16f8e11
added collection theorem for consistency and convenience
blanchet
parents:
57983
diff
changeset
|
834 |
\item[@{text "t."}\hthm{split_sels} = @{text "split_sel split_sel_asm"}] |
cbe9a16f8e11
added collection theorem for consistency and convenience
blanchet
parents:
57983
diff
changeset
|
835 |
|
57542 | 836 |
\item[@{text "t."}\hthm{case_eq_if}\rm:] ~ \\ |
54491 | 837 |
@{thm list.case_eq_if[no_vars]} |
53543 | 838 |
|
839 |
\end{description} |
|
53552 | 840 |
\end{indentblock} |
54152 | 841 |
|
842 |
\noindent |
|
843 |
In addition, equational versions of @{text t.disc} are registered with the @{text "[code]"} |
|
844 |
attribute. |
|
53552 | 845 |
*} |
846 |
||
847 |
||
53621 | 848 |
subsubsection {* Functorial Theorems |
849 |
\label{sssec:functorial-theorems} *} |
|
53552 | 850 |
|
851 |
text {* |
|
54621 | 852 |
The functorial theorems are partitioned in two subgroups. The first subgroup |
56992 | 853 |
consists of properties involving the constructors or the destructors and either |
854 |
a set function, the map function, or the relator: |
|
53552 | 855 |
|
856 |
\begin{indentblock} |
|
857 |
\begin{description} |
|
858 |
||
58094 | 859 |
\item[@{text "t."}\hthm{case_transfer}\rm:] ~ \\ |
860 |
@{thm list.case_transfer[no_vars]} |
|
861 |
||
58000 | 862 |
\item[@{text "t."}\hthm{ctr_transfer}\rm:] ~ \\ |
863 |
@{thm list.ctr_transfer(1)[no_vars]} \\ |
|
864 |
@{thm list.ctr_transfer(2)[no_vars]} |
|
865 |
||
58096 | 866 |
\item[@{text "t."}\hthm{disc_transfer}\rm:] ~ \\ |
867 |
@{thm list.disc_transfer(1)[no_vars]} \\ |
|
868 |
@{thm list.disc_transfer(2)[no_vars]} |
|
869 |
||
53798 | 870 |
\item[@{text "t."}\hthm{set} @{text "[simp, code]"}\rm:] ~ \\ |
53694 | 871 |
@{thm list.set(1)[no_vars]} \\ |
872 |
@{thm list.set(2)[no_vars]} |
|
53552 | 873 |
|
57988 | 874 |
\item[@{text "t."}\hthm{set_cases} @{text "[consumes 1, cases set: set\<^sub>i_t]"}\rm:] ~ \\ |
57894 | 875 |
@{thm list.set_cases[no_vars]} |
876 |
||
57892 | 877 |
\item[@{text "t."}\hthm{set_intros}\rm:] ~ \\ |
878 |
@{thm list.set_intros(1)[no_vars]} \\ |
|
879 |
@{thm list.set_intros(2)[no_vars]} |
|
880 |
||
57983
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
881 |
\item[@{text "t."}\hthm{set_sel}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
882 |
@{thm list.set_sel[no_vars]} |
57153 | 883 |
|
53798 | 884 |
\item[@{text "t."}\hthm{map} @{text "[simp, code]"}\rm:] ~ \\ |
53552 | 885 |
@{thm list.map(1)[no_vars]} \\ |
886 |
@{thm list.map(2)[no_vars]} |
|
887 |
||
57983
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
888 |
\item[@{text "t."}\hthm{map_disc_iff} @{text "[simp]"}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
889 |
@{thm list.map_disc_iff[no_vars]} |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
890 |
|
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
891 |
\item[@{text "t."}\hthm{map_sel}\rm:] ~ \\ |
6edc3529bb4e
reordered some (co)datatype property names for more consistency
blanchet
parents:
57982
diff
changeset
|
892 |
@{thm list.map_sel[no_vars]} |
57047 | 893 |
|
57542 | 894 |
\item[@{text "t."}\hthm{rel_inject} @{text "[simp]"}\rm:] ~ \\ |
53552 | 895 |
@{thm list.rel_inject(1)[no_vars]} \\ |
896 |
@{thm list.rel_inject(2)[no_vars]} |
|
897 |
||
57542 | 898 |
\item[@{text "t."}\hthm{rel_distinct} @{text "[simp]"}\rm:] ~ \\ |
57526 | 899 |
@{thm list.rel_distinct(1)[no_vars]} \\ |
900 |
@{thm list.rel_distinct(2)[no_vars]} |
|
901 |
||
57542 | 902 |
\item[@{text "t."}\hthm{rel_intros}\rm:] ~ \\ |
57494 | 903 |
@{thm list.rel_intros(1)[no_vars]} \\ |
904 |
@{thm list.rel_intros(2)[no_vars]} |
|
905 |
||
57558
6bb3dd7f8097
took out 'rel_cases' for now because of failing tactic
blanchet
parents:
57542
diff
changeset
|
906 |
% FIXME (and add @ before antiquotation below) |
6bb3dd7f8097
took out 'rel_cases' for now because of failing tactic
blanchet
parents:
57542
diff
changeset
|
907 |
%\item[@{text "t."}\hthm{rel_cases} @{text "[consumes 1, case_names t\<^sub>1 \<dots> t\<^sub>m, cases pred]"}\rm:] ~ \\ |
6bb3dd7f8097
took out 'rel_cases' for now because of failing tactic
blanchet
parents:
57542
diff
changeset
|
908 |
%{thm list.rel_cases[no_vars]} |
53552 | 909 |
|
57564 | 910 |
\item[@{text "t."}\hthm{rel_sel}\rm:] ~ \\ |
911 |
@{thm list.rel_sel[no_vars]} |
|
912 |
||
53552 | 913 |
\end{description} |
914 |
\end{indentblock} |
|
54146 | 915 |
|
916 |
\noindent |
|
917 |
In addition, equational versions of @{text t.rel_inject} and @{text |
|
918 |
rel_distinct} are registered with the @{text "[code]"} attribute. |
|
54621 | 919 |
|
920 |
The second subgroup consists of more abstract properties of the set functions, |
|
921 |
the map function, and the relator: |
|
922 |
||
923 |
\begin{indentblock} |
|
924 |
\begin{description} |
|
925 |
||
57969 | 926 |
\item[@{text "t."}\hthm{inj_map}\rm:] ~ \\ |
927 |
@{thm list.inj_map[no_vars]} |
|
928 |
||
57971 | 929 |
\item[@{text "t."}\hthm{inj_map_strong}\rm:] ~ \\ |
930 |
@{thm list.inj_map_strong[no_vars]} |
|
931 |
||
57542 | 932 |
\item[@{text "t."}\hthm{set_map}\rm:] ~ \\ |
56992 | 933 |
@{thm list.set_map[no_vars]} |
934 |
||
58107 | 935 |
\item[@{text "t."}\hthm{set_transfer}\rm:] ~ \\ |
936 |
@{thm list.set_transfer[no_vars]} |
|
937 |
||
57982 | 938 |
\item[@{text "t."}\hthm{map_comg0}\rm:] ~ \\ |
54621 | 939 |
@{thm list.map_cong0[no_vars]} |
940 |
||
57542 | 941 |
\item[@{text "t."}\hthm{map_cong} @{text "[fundef_cong]"}\rm:] ~ \\ |
54621 | 942 |
@{thm list.map_cong[no_vars]} |
943 |
||
57982 | 944 |
\item[@{text "t."}\hthm{map_cong_simp}\rm:] ~ \\ |
945 |
@{thm list.map_cong_simp[no_vars]} |
|
946 |
||
57542 | 947 |
\item[@{text "t."}\hthm{map_id}\rm:] ~ \\ |
54621 | 948 |
@{thm list.map_id[no_vars]} |
949 |
||
57542 | 950 |
\item[@{text "t."}\hthm{map_id0}\rm:] ~ \\ |
56955 | 951 |
@{thm list.map_id0[no_vars]} |
952 |
||
57542 | 953 |
\item[@{text "t."}\hthm{map_ident}\rm:] ~ \\ |
56904 | 954 |
@{thm list.map_ident[no_vars]} |
955 |
||
58103 | 956 |
\item[@{text "t."}\hthm{map_transfer}\rm:] ~ \\ |
957 |
@{thm list.map_transfer[no_vars]} |
|
958 |
||
57542 | 959 |
\item[@{text "t."}\hthm{rel_compp}\rm:] ~ \\ |
54621 | 960 |
@{thm list.rel_compp[no_vars]} |
961 |
||
57542 | 962 |
\item[@{text "t."}\hthm{rel_conversep}\rm:] ~ \\ |
54621 | 963 |
@{thm list.rel_conversep[no_vars]} |
964 |
||
57542 | 965 |
\item[@{text "t."}\hthm{rel_eq}\rm:] ~ \\ |
54621 | 966 |
@{thm list.rel_eq[no_vars]} |
967 |
||
57542 | 968 |
\item[@{text "t."}\hthm{rel_flip}\rm:] ~ \\ |
54621 | 969 |
@{thm list.rel_flip[no_vars]} |
970 |
||
57933 | 971 |
\item[@{text "t."}\hthm{rel_map}\rm:] ~ \\ |
972 |
@{thm list.rel_map(1)[no_vars]} \\ |
|
973 |
@{thm list.rel_map(2)[no_vars]} |
|
974 |
||
57542 | 975 |
\item[@{text "t."}\hthm{rel_mono}\rm:] ~ \\ |
54621 | 976 |
@{thm list.rel_mono[no_vars]} |
977 |
||
58105 | 978 |
\item[@{text "t."}\hthm{rel_transfer}\rm:] ~ \\ |
979 |
@{thm list.rel_transfer[no_vars]} |
|
980 |
||
54621 | 981 |
\end{description} |
982 |
\end{indentblock} |
|
53535 | 983 |
*} |
984 |
||
985 |
||
53621 | 986 |
subsubsection {* Inductive Theorems |
987 |
\label{sssec:inductive-theorems} *} |
|
53535 | 988 |
|
989 |
text {* |
|
53623 | 990 |
The inductive theorems are as follows: |
53544 | 991 |
|
53552 | 992 |
\begin{indentblock} |
53544 | 993 |
\begin{description} |
994 |
||
57304 | 995 |
\item[@{text "t."}\hthm{induct} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n, induct t]"}\rm:] ~ \\ |
53544 | 996 |
@{thm list.induct[no_vars]} |
997 |
||
57542 | 998 |
\item[@{text "t."}\hthm{rel_induct} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n, induct pred]"}\rm:] ~ \\ |
57472 | 999 |
@{thm list.rel_induct[no_vars]} |
1000 |
||
57701 | 1001 |
\item[\begin{tabular}{@ {}l@ {}} |
1002 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{induct} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm: \\ |
|
1003 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{rel_induct} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm: \\ |
|
1004 |
\end{tabular}] ~ \\ |
|
57472 | 1005 |
Given $m > 1$ mutually recursive datatypes, this induction rule can be used to |
1006 |
prove $m$ properties simultaneously. |
|
1007 |
||
53798 | 1008 |
\item[@{text "t."}\hthm{rec} @{text "[simp, code]"}\rm:] ~ \\ |
53544 | 1009 |
@{thm list.rec(1)[no_vars]} \\ |
1010 |
@{thm list.rec(2)[no_vars]} |
|
1011 |
||
57542 | 1012 |
\item[@{text "t."}\hthm{rec_o_map}\rm:] ~ \\ |
56655 | 1013 |
@{thm list.rec_o_map[no_vars]} |
1014 |
||
1015 |
\item[@{text "t."}\hthm{size} @{text "[simp, code]"}\rm:] ~ \\ |
|
1016 |
@{thm list.size(1)[no_vars]} \\ |
|
1017 |
@{thm list.size(2)[no_vars]} \\ |
|
1018 |
@{thm list.size(3)[no_vars]} \\ |
|
1019 |
@{thm list.size(4)[no_vars]} |
|
1020 |
||
57542 | 1021 |
\item[@{text "t."}\hthm{size_o_map}\rm:] ~ \\ |
56655 | 1022 |
@{thm list.size_o_map[no_vars]} |
1023 |
||
53544 | 1024 |
\end{description} |
53552 | 1025 |
\end{indentblock} |
53544 | 1026 |
|
1027 |
\noindent |
|
1028 |
For convenience, @{command datatype_new} also provides the following collection: |
|
1029 |
||
53552 | 1030 |
\begin{indentblock} |
53544 | 1031 |
\begin{description} |
1032 |
||
55871 | 1033 |
\item[@{text "t."}\hthm{simps} = @{text t.inject} @{text t.distinct} @{text t.case} @{text t.rec} @{text t.map} @{text t.rel_inject}] ~ \\ |
53694 | 1034 |
@{text t.rel_distinct} @{text t.set} |
53544 | 1035 |
|
1036 |
\end{description} |
|
53552 | 1037 |
\end{indentblock} |
52828 | 1038 |
*} |
1039 |
||
52794 | 1040 |
|
52827 | 1041 |
subsection {* Compatibility Issues |
52824 | 1042 |
\label{ssec:datatype-compatibility-issues} *} |
52794 | 1043 |
|
52828 | 1044 |
text {* |
53997 | 1045 |
The command @{command datatype_new} has been designed to be highly compatible |
1046 |
with the old \keyw{datatype}, to ease migration. There are nonetheless a few |
|
53647 | 1047 |
incompatibilities that may arise when porting to the new package: |
1048 |
||
1049 |
\begin{itemize} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1050 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1051 |
|
53647 | 1052 |
\item \emph{The Standard ML interfaces are different.} Tools and extensions |
1053 |
written to call the old ML interfaces will need to be adapted to the new |
|
56655 | 1054 |
interfaces. This concerns Quickcheck in particular. Whenever possible, it is |
1055 |
recommended to use @{command datatype_compat} to register new-style datatypes |
|
1056 |
as old-style datatypes. |
|
53647 | 1057 |
|
56644 | 1058 |
\item \emph{The constants @{text t_case}, @{text t_rec}, and @{text t_size} are |
1059 |
now called @{text case_t}, @{text rec_t}, and @{text size_t}.} |
|
54537 | 1060 |
|
1061 |
\item \emph{The recursor @{text rec_t} has a different signature for nested |
|
54185 | 1062 |
recursive datatypes.} In the old package, nested recursion through non-functions |
1063 |
was internally reduced to mutual recursion. This reduction was visible in the |
|
1064 |
type of the recursor, used by \keyw{primrec}. Recursion through functions was |
|
1065 |
handled specially. In the new package, nested recursion (for functions and |
|
1066 |
non-functions) is handled in a more modular fashion. The old-style recursor can |
|
56655 | 1067 |
be generated on demand using @{command primrec} if the recursion is via |
1068 |
new-style datatypes, as explained in |
|
1069 |
Section~\ref{sssec:primrec-nested-as-mutual-recursion}. |
|
53647 | 1070 |
|
54287 | 1071 |
\item \emph{Accordingly, the induction rule is different for nested recursive |
1072 |
datatypes.} Again, the old-style induction rule can be generated on demand using |
|
56655 | 1073 |
@{command primrec} if the recursion is via new-style datatypes, as explained in |
1074 |
Section~\ref{sssec:primrec-nested-as-mutual-recursion}. |
|
52828 | 1075 |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1076 |
\item \emph{The internal constructions are completely different.} Proof texts |
53647 | 1077 |
that unfold the definition of constants introduced by \keyw{datatype} will be |
1078 |
difficult to port. |
|
1079 |
||
56644 | 1080 |
\item \emph{Some theorems have different names.} |
55641
5b466efedd2c
renamed 'recs' and 'cases' theorems 'rec' and 'case' in old datatype package, for consistency with new package
blanchet
parents:
55531
diff
changeset
|
1081 |
For non-mutually recursive datatypes, |
5b466efedd2c
renamed 'recs' and 'cases' theorems 'rec' and 'case' in old datatype package, for consistency with new package
blanchet
parents:
55531
diff
changeset
|
1082 |
the alias @{text t.inducts} for @{text t.induct} is no longer generated. |
53647 | 1083 |
For $m > 1$ mutually recursive datatypes, |
53997 | 1084 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m.inducts(i)"} has been renamed |
56644 | 1085 |
@{text "t\<^sub>i.induct"} for each @{text "i \<in> {1, \<dots>, t}"}, and similarly the |
1086 |
collection @{text "t\<^sub>1_\<dots>_t\<^sub>m.size"} has been divided into @{text "t\<^sub>1.size"}, |
|
1087 |
\ldots, @{text "t\<^sub>m.size"}. |
|
53647 | 1088 |
|
1089 |
\item \emph{The @{text t.simps} collection has been extended.} |
|
1090 |
Previously available theorems are available at the same index. |
|
1091 |
||
1092 |
\item \emph{Variables in generated properties have different names.} This is |
|
1093 |
rarely an issue, except in proof texts that refer to variable names in the |
|
1094 |
@{text "[where \<dots>]"} attribute. The solution is to use the more robust |
|
1095 |
@{text "[of \<dots>]"} syntax. |
|
1096 |
\end{itemize} |
|
1097 |
||
1098 |
In the other direction, there is currently no way to register old-style |
|
1099 |
datatypes as new-style datatypes. If the goal is to define new-style datatypes |
|
1100 |
with nested recursion through old-style datatypes, the old-style |
|
1101 |
datatypes can be registered as a BNF |
|
55351 | 1102 |
(Section~\ref{sec:introducing-bounded-natural-functors}). If the goal is |
55468
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55460
diff
changeset
|
1103 |
to derive discriminators and selectors, this can be achieved using |
98b25c51e9e5
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet
parents:
55460
diff
changeset
|
1104 |
@{command free_constructors} |
53647 | 1105 |
(Section~\ref{sec:deriving-destructors-and-theorems-for-free-constructors}). |
52828 | 1106 |
*} |
1107 |
||
52792 | 1108 |
|
52827 | 1109 |
section {* Defining Recursive Functions |
52805 | 1110 |
\label{sec:defining-recursive-functions} *} |
1111 |
||
1112 |
text {* |
|
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1113 |
Recursive functions over datatypes can be specified using the @{command primrec} |
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1114 |
command, which supports primitive recursion, or using the more general |
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1115 |
\keyw{fun} and \keyw{function} commands. Here, the focus is on |
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1116 |
@{command primrec}; the other two commands are described in a separate |
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1117 |
tutorial \cite{isabelle-function}. |
52828 | 1118 |
|
53621 | 1119 |
%%% TODO: partial_function |
52805 | 1120 |
*} |
52792 | 1121 |
|
52805 | 1122 |
|
53617 | 1123 |
subsection {* Introductory Examples |
1124 |
\label{ssec:primrec-introductory-examples} *} |
|
52828 | 1125 |
|
53646 | 1126 |
text {* |
1127 |
Primitive recursion is illustrated through concrete examples based on the |
|
1128 |
datatypes defined in Section~\ref{ssec:datatype-introductory-examples}. More |
|
55075 | 1129 |
examples can be found in the directory \verb|~~/src/HOL/BNF_Examples|. |
53646 | 1130 |
*} |
1131 |
||
53621 | 1132 |
|
1133 |
subsubsection {* Nonrecursive Types |
|
1134 |
\label{sssec:primrec-nonrecursive-types} *} |
|
52828 | 1135 |
|
52841 | 1136 |
text {* |
53621 | 1137 |
Primitive recursion removes one layer of constructors on the left-hand side in |
1138 |
each equation. For example: |
|
52841 | 1139 |
*} |
1140 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1141 |
primrec bool_of_trool :: "trool \<Rightarrow> bool" where |
53621 | 1142 |
"bool_of_trool Faalse \<longleftrightarrow> False" | |
1143 |
"bool_of_trool Truue \<longleftrightarrow> True" |
|
52841 | 1144 |
|
53621 | 1145 |
text {* \blankline *} |
52841 | 1146 |
|
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1147 |
primrec the_list :: "'a option \<Rightarrow> 'a list" where |
53025 | 1148 |
"the_list None = []" | |
1149 |
"the_list (Some a) = [a]" |
|
52841 | 1150 |
|
53621 | 1151 |
text {* \blankline *} |
1152 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1153 |
primrec the_default :: "'a \<Rightarrow> 'a option \<Rightarrow> 'a" where |
53025 | 1154 |
"the_default d None = d" | |
1155 |
"the_default _ (Some a) = a" |
|
52843 | 1156 |
|
53621 | 1157 |
text {* \blankline *} |
1158 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1159 |
primrec mirrror :: "('a, 'b, 'c) triple \<Rightarrow> ('c, 'b, 'a) triple" where |
52841 | 1160 |
"mirrror (Triple a b c) = Triple c b a" |
1161 |
||
53621 | 1162 |
text {* |
1163 |
\noindent |
|
1164 |
The equations can be specified in any order, and it is acceptable to leave out |
|
1165 |
some cases, which are then unspecified. Pattern matching on the left-hand side |
|
1166 |
is restricted to a single datatype, which must correspond to the same argument |
|
1167 |
in all equations. |
|
1168 |
*} |
|
52828 | 1169 |
|
53621 | 1170 |
|
1171 |
subsubsection {* Simple Recursion |
|
1172 |
\label{sssec:primrec-simple-recursion} *} |
|
52828 | 1173 |
|
52841 | 1174 |
text {* |
53621 | 1175 |
For simple recursive types, recursive calls on a constructor argument are |
1176 |
allowed on the right-hand side: |
|
52841 | 1177 |
*} |
1178 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1179 |
primrec replicate :: "nat \<Rightarrow> 'a \<Rightarrow> 'a list" where |
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1180 |
"replicate Zero _ = []" | |
53644 | 1181 |
"replicate (Suc n) x = x # replicate n x" |
52841 | 1182 |
|
53621 | 1183 |
text {* \blankline *} |
52843 | 1184 |
|
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1185 |
primrec at :: "'a list \<Rightarrow> nat \<Rightarrow> 'a" where |
53644 | 1186 |
"at (x # xs) j = |
52843 | 1187 |
(case j of |
53644 | 1188 |
Zero \<Rightarrow> x |
1189 |
| Suc j' \<Rightarrow> at xs j')" |
|
52843 | 1190 |
|
53621 | 1191 |
text {* \blankline *} |
1192 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1193 |
primrec (*<*)(in early) (*>*)tfold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> ('a, 'b) tlist \<Rightarrow> 'b" where |
53644 | 1194 |
"tfold _ (TNil y) = y" | |
1195 |
"tfold f (TCons x xs) = f x (tfold f xs)" |
|
52841 | 1196 |
|
53025 | 1197 |
text {* |
53621 | 1198 |
\noindent |
54402 | 1199 |
Pattern matching is only available for the argument on which the recursion takes |
1200 |
place. Fortunately, it is easy to generate pattern-maching equations using the |
|
57542 | 1201 |
\keyw{simps_of_case} command provided by the theory |
55290 | 1202 |
\verb|~~/src/HOL/|\allowbreak\verb|Library/|\allowbreak\verb|Simps_Case_Conv|. |
54402 | 1203 |
*} |
1204 |
||
1205 |
simps_of_case at_simps: at.simps |
|
1206 |
||
1207 |
text {* |
|
1208 |
This generates the lemma collection @{thm [source] at_simps}: |
|
1209 |
% |
|
1210 |
\[@{thm at_simps(1)[no_vars]} |
|
1211 |
\qquad @{thm at_simps(2)[no_vars]}\] |
|
1212 |
% |
|
54184 | 1213 |
The next example is defined using \keyw{fun} to escape the syntactic |
55254 | 1214 |
restrictions imposed on primitively recursive functions. The |
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
1215 |
@{command datatype_compat} command is needed to register new-style datatypes |
54184 | 1216 |
for use with \keyw{fun} and \keyw{function} |
56644 | 1217 |
(Section~\ref{sssec:datatype-compat}): |
53025 | 1218 |
*} |
52828 | 1219 |
|
55531
601ca8efa000
renamed 'datatype_new_compat' to 'datatype_compat'
blanchet
parents:
55530
diff
changeset
|
1220 |
datatype_compat nat |
53621 | 1221 |
|
1222 |
text {* \blankline *} |
|
1223 |
||
1224 |
fun at_least_two :: "nat \<Rightarrow> bool" where |
|
1225 |
"at_least_two (Suc (Suc _)) \<longleftrightarrow> True" | |
|
1226 |
"at_least_two _ \<longleftrightarrow> False" |
|
1227 |
||
1228 |
||
1229 |
subsubsection {* Mutual Recursion |
|
1230 |
\label{sssec:primrec-mutual-recursion} *} |
|
52828 | 1231 |
|
52841 | 1232 |
text {* |
53621 | 1233 |
The syntax for mutually recursive functions over mutually recursive datatypes |
1234 |
is straightforward: |
|
52841 | 1235 |
*} |
1236 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1237 |
primrec |
53623 | 1238 |
nat_of_even_nat :: "even_nat \<Rightarrow> nat" and |
1239 |
nat_of_odd_nat :: "odd_nat \<Rightarrow> nat" |
|
52841 | 1240 |
where |
53623 | 1241 |
"nat_of_even_nat Even_Zero = Zero" | |
1242 |
"nat_of_even_nat (Even_Suc n) = Suc (nat_of_odd_nat n)" | |
|
1243 |
"nat_of_odd_nat (Odd_Suc n) = Suc (nat_of_even_nat n)" |
|
52841 | 1244 |
|
53752 | 1245 |
text {* \blankline *} |
1246 |
||
55530
3dfb724db099
renamed 'primrec_new' to 'primrec', overriding the old command (which it still uses as a fallback for old-style datatypes)
blanchet
parents:
55474
diff
changeset
|
1247 |
primrec |
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1248 |
eval\<^sub>e :: "('a \<Rightarrow> int) \<Rightarrow> ('b \<Rightarrow> int) \<Rightarrow> ('a, 'b) exp \<Rightarrow> int" and |
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1249 |
eval\<^sub>t :: "('a \<Rightarrow> int) \<Rightarrow> ('b \<Rightarrow> int) \<Rightarrow> ('a, 'b) trm \<Rightarrow> int" and |