author | traytel |
Tue, 01 Oct 2013 17:06:35 +0200 | |
changeset 54014 | 21dac9a60f0c |
parent 53997 | 8ff43f638da2 |
child 54023 | cede3c1d2417 |
permissions | -rw-r--r-- |
52792 | 1 |
(* Title: Doc/Datatypes/Datatypes.thy |
2 |
Author: Jasmin Blanchette, TU Muenchen |
|
53617 | 3 |
Author: Lorenz Panny, TU Muenchen |
4 |
Author: Andrei Popescu, TU Muenchen |
|
5 |
Author: Dmitriy Traytel, TU Muenchen |
|
52792 | 6 |
|
7 |
Tutorial for (co)datatype definitions with the new package. |
|
8 |
*) |
|
9 |
||
10 |
theory Datatypes |
|
52824 | 11 |
imports Setup |
53644 | 12 |
keywords |
53826 | 13 |
"primcorec_notyet" :: thy_decl |
52792 | 14 |
begin |
15 |
||
53644 | 16 |
(*<*) |
53822 | 17 |
(* FIXME: Temporary setup until "primcorec" and "primcorecursive" are fully implemented. *) |
53644 | 18 |
ML_command {* |
19 |
fun add_dummy_cmd _ _ lthy = lthy; |
|
20 |
||
53826 | 21 |
val _ = Outer_Syntax.local_theory @{command_spec "primcorec_notyet"} "" |
53644 | 22 |
(Parse.fixes -- Parse_Spec.where_alt_specs >> uncurry add_dummy_cmd); |
23 |
*} |
|
24 |
(*>*) |
|
25 |
||
26 |
||
52828 | 27 |
section {* Introduction |
28 |
\label{sec:introduction} *} |
|
52792 | 29 |
|
30 |
text {* |
|
53028 | 31 |
The 2013 edition of Isabelle introduced a new definitional package for freely |
32 |
generated datatypes and codatatypes. The datatype support is similar to that |
|
33 |
provided by the earlier package due to Berghofer and Wenzel |
|
34 |
\cite{Berghofer-Wenzel:1999:TPHOL}, documented in the Isar reference manual |
|
53535 | 35 |
\cite{isabelle-isar-ref}; indeed, replacing the keyword \keyw{datatype} by |
53028 | 36 |
@{command datatype_new} is usually all that is needed to port existing theories |
37 |
to use the new package. |
|
52840 | 38 |
|
52841 | 39 |
Perhaps the main advantage of the new package is that it supports recursion |
53619 | 40 |
through a large class of non-datatypes, such as finite sets: |
52792 | 41 |
*} |
42 |
||
53644 | 43 |
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 | 44 |
|
45 |
text {* |
|
52794 | 46 |
\noindent |
53025 | 47 |
Another strong point is the support for local definitions: |
52792 | 48 |
*} |
49 |
||
52805 | 50 |
context linorder |
51 |
begin |
|
52841 | 52 |
datatype_new flag = Less | Eq | Greater |
52805 | 53 |
end |
52792 | 54 |
|
55 |
text {* |
|
52794 | 56 |
\noindent |
52840 | 57 |
The package also provides some convenience, notably automatically generated |
53543 | 58 |
discriminators and selectors. |
52794 | 59 |
|
53025 | 60 |
In addition to plain inductive datatypes, the new package supports coinductive |
52840 | 61 |
datatypes, or \emph{codatatypes}, which may have infinite values. For example, |
53028 | 62 |
the following command introduces the type of lazy lists, which comprises both |
63 |
finite and infinite values: |
|
52794 | 64 |
*} |
65 |
||
53623 | 66 |
(*<*) |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
67 |
locale early |
53623 | 68 |
(*>*) |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
69 |
codatatype (*<*)(in early) (*>*)'a llist = LNil | LCons 'a "'a llist" |
52794 | 70 |
|
71 |
text {* |
|
72 |
\noindent |
|
52840 | 73 |
Mixed inductive--coinductive recursion is possible via nesting. Compare the |
53028 | 74 |
following four Rose tree examples: |
52794 | 75 |
*} |
76 |
||
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
77 |
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
|
78 |
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
|
79 |
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
|
80 |
codatatype (*<*)(in early) (*>*)'a tree\<^sub>i\<^sub>i = Node\<^sub>i\<^sub>i 'a "'a tree\<^sub>i\<^sub>i llist" |
52792 | 81 |
|
52794 | 82 |
text {* |
52840 | 83 |
The first two tree types allow only finite branches, whereas the last two allow |
53028 | 84 |
branches of infinite length. Orthogonally, the nodes in the first and third |
85 |
types have finite branching, whereas those of the second and fourth may have |
|
86 |
infinitely many direct subtrees. |
|
52840 | 87 |
|
52794 | 88 |
To use the package, it is necessary to import the @{theory BNF} theory, which |
53552 | 89 |
can be precompiled into the \texttt{HOL-BNF} image. The following commands show |
52806 | 90 |
how to launch jEdit/PIDE with the image loaded and how to build the image |
91 |
without launching jEdit: |
|
52794 | 92 |
*} |
93 |
||
94 |
text {* |
|
95 |
\noindent |
|
52806 | 96 |
\ \ \ \ \texttt{isabelle jedit -l HOL-BNF} \\ |
52827 | 97 |
\noindent |
52828 | 98 |
\hbox{}\ \ \ \ \texttt{isabelle build -b HOL-BNF} |
52794 | 99 |
*} |
100 |
||
101 |
text {* |
|
52805 | 102 |
The package, like its predecessor, fully adheres to the LCF philosophy |
103 |
\cite{mgordon79}: The characteristic theorems associated with the specified |
|
104 |
(co)datatypes are derived rather than introduced axiomatically.% |
|
53543 | 105 |
\footnote{If the @{text quick_and_dirty} option is enabled, some of the |
52841 | 106 |
internal constructions and most of the internal proof obligations are skipped.} |
52805 | 107 |
The package's metatheory is described in a pair of papers |
53552 | 108 |
\cite{traytel-et-al-2012,blanchette-et-al-wit}. The central notion is that of a |
109 |
\emph{bounded natural functor} (BNF)---a well-behaved type constructor for which |
|
110 |
nested (co)recursion is supported. |
|
52792 | 111 |
|
52794 | 112 |
This tutorial is organized as follows: |
113 |
||
52805 | 114 |
\begin{itemize} |
52822 | 115 |
\setlength{\itemsep}{0pt} |
116 |
||
52805 | 117 |
\item Section \ref{sec:defining-datatypes}, ``Defining Datatypes,'' |
52822 | 118 |
describes how to specify datatypes using the @{command datatype_new} command. |
52805 | 119 |
|
53018 | 120 |
\item Section \ref{sec:defining-recursive-functions}, ``Defining Recursive |
52805 | 121 |
Functions,'' describes how to specify recursive functions using |
53535 | 122 |
@{command primrec_new}, \keyw{fun}, and \keyw{function}. |
52805 | 123 |
|
124 |
\item Section \ref{sec:defining-codatatypes}, ``Defining Codatatypes,'' |
|
53829 | 125 |
describes how to specify codatatypes using the @{command codatatype} command. |
52805 | 126 |
|
53018 | 127 |
\item Section \ref{sec:defining-corecursive-functions}, ``Defining Corecursive |
52805 | 128 |
Functions,'' describes how to specify corecursive functions using the |
53826 | 129 |
@{command primcorec} and @{command primcorecursive} commands. |
52794 | 130 |
|
53018 | 131 |
\item Section \ref{sec:registering-bounded-natural-functors}, ``Registering |
53552 | 132 |
Bounded Natural Functors,'' explains how to use the @{command bnf} command |
133 |
to register arbitrary type constructors as BNFs. |
|
52805 | 134 |
|
53552 | 135 |
\item Section |
53617 | 136 |
\ref{sec:deriving-destructors-and-theorems-for-free-constructors}, |
137 |
``Deriving Destructors and Theorems for Free Constructors,'' explains how to |
|
53552 | 138 |
use the command @{command wrap_free_constructors} to derive destructor constants |
139 |
and theorems for freely generated types, as performed internally by @{command |
|
53829 | 140 |
datatype_new} and @{command codatatype}. |
52794 | 141 |
|
53617 | 142 |
%\item Section \ref{sec:standard-ml-interface}, ``Standard ML Interface,'' |
143 |
%describes the package's programmatic interface. |
|
52794 | 144 |
|
53617 | 145 |
%\item Section \ref{sec:interoperability}, ``Interoperability,'' |
146 |
%is concerned with the packages' interaction with other Isabelle packages and |
|
147 |
%tools, such as the code generator and the counterexample generators. |
|
52805 | 148 |
|
53617 | 149 |
%\item Section \ref{sec:known-bugs-and-limitations}, ``Known Bugs and |
150 |
%Limitations,'' concludes with known open issues at the time of writing. |
|
52805 | 151 |
\end{itemize} |
52822 | 152 |
|
153 |
||
154 |
\newbox\boxA |
|
155 |
\setbox\boxA=\hbox{\texttt{nospam}} |
|
156 |
||
157 |
\newcommand\authoremaili{\texttt{blan{\color{white}nospam}\kern-\wd\boxA{}chette@\allowbreak |
|
158 |
in.\allowbreak tum.\allowbreak de}} |
|
53028 | 159 |
\newcommand\authoremailii{\texttt{lore{\color{white}nospam}\kern-\wd\boxA{}nz.panny@\allowbreak |
160 |
\allowbreak tum.\allowbreak de}} |
|
161 |
\newcommand\authoremailiii{\texttt{pope{\color{white}nospam}\kern-\wd\boxA{}scua@\allowbreak |
|
52822 | 162 |
in.\allowbreak tum.\allowbreak de}} |
53028 | 163 |
\newcommand\authoremailiv{\texttt{tray{\color{white}nospam}\kern-\wd\boxA{}tel@\allowbreak |
52822 | 164 |
in.\allowbreak tum.\allowbreak de}} |
165 |
||
53028 | 166 |
The commands @{command datatype_new} and @{command primrec_new} are expected to |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
167 |
replace \keyw{datatype} and \keyw{primrec} in a future release. Authors of new |
53535 | 168 |
theories are encouraged to use the new commands, and maintainers of older |
53028 | 169 |
theories may want to consider upgrading. |
52841 | 170 |
|
171 |
Comments and bug reports concerning either the tool or this tutorial should be |
|
53028 | 172 |
directed to the authors at \authoremaili, \authoremailii, \authoremailiii, |
173 |
and \authoremailiv. |
|
52822 | 174 |
|
175 |
\begin{framed} |
|
176 |
\noindent |
|
53646 | 177 |
\textbf{Warning:}\enskip This tutorial and the package it describes are under |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
178 |
construction. Please forgive their appearance. Should you have suggestions |
53646 | 179 |
or comments regarding either, please let the authors know. |
52822 | 180 |
\end{framed} |
52794 | 181 |
*} |
182 |
||
53491 | 183 |
|
52827 | 184 |
section {* Defining Datatypes |
52805 | 185 |
\label{sec:defining-datatypes} *} |
186 |
||
187 |
text {* |
|
53646 | 188 |
Datatypes can be specified using the @{command datatype_new} command. |
52805 | 189 |
*} |
52792 | 190 |
|
52824 | 191 |
|
53617 | 192 |
subsection {* Introductory Examples |
193 |
\label{ssec:datatype-introductory-examples} *} |
|
52794 | 194 |
|
53646 | 195 |
text {* |
196 |
Datatypes are illustrated through concrete examples featuring different flavors |
|
197 |
of recursion. More examples can be found in the directory |
|
198 |
\verb|~~/src/HOL/BNF/Examples|. |
|
199 |
*} |
|
53621 | 200 |
|
201 |
subsubsection {* Nonrecursive Types |
|
202 |
\label{sssec:datatype-nonrecursive-types} *} |
|
52794 | 203 |
|
52805 | 204 |
text {* |
53028 | 205 |
Datatypes are introduced by specifying the desired names and argument types for |
53491 | 206 |
their constructors. \emph{Enumeration} types are the simplest form of datatype. |
53028 | 207 |
All their constructors are nullary: |
52805 | 208 |
*} |
209 |
||
52828 | 210 |
datatype_new trool = Truue | Faalse | Perhaaps |
52805 | 211 |
|
212 |
text {* |
|
53028 | 213 |
\noindent |
53491 | 214 |
Here, @{const Truue}, @{const Faalse}, and @{const Perhaaps} have the type @{typ trool}. |
53028 | 215 |
|
216 |
Polymorphic types are possible, such as the following option type, modeled after |
|
217 |
its homologue from the @{theory Option} theory: |
|
52805 | 218 |
*} |
219 |
||
53025 | 220 |
(*<*) |
221 |
hide_const None Some |
|
222 |
(*>*) |
|
223 |
datatype_new 'a option = None | Some 'a |
|
52805 | 224 |
|
225 |
text {* |
|
53028 | 226 |
\noindent |
53491 | 227 |
The constructors are @{text "None :: 'a option"} and |
228 |
@{text "Some :: 'a \<Rightarrow> 'a option"}. |
|
53028 | 229 |
|
230 |
The next example has three type parameters: |
|
52805 | 231 |
*} |
232 |
||
233 |
datatype_new ('a, 'b, 'c) triple = Triple 'a 'b 'c |
|
234 |
||
53028 | 235 |
text {* |
236 |
\noindent |
|
237 |
The constructor is |
|
53491 | 238 |
@{text "Triple :: 'a \<Rightarrow> 'b \<Rightarrow> 'c \<Rightarrow> ('a, 'b, 'c) triple"}. |
53028 | 239 |
Unlike in Standard ML, curried constructors are supported. The uncurried variant |
240 |
is also possible: |
|
241 |
*} |
|
242 |
||
243 |
datatype_new ('a, 'b, 'c) triple\<^sub>u = Triple\<^sub>u "'a * 'b * 'c" |
|
244 |
||
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
245 |
text {* |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
246 |
\noindent |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
247 |
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
|
248 |
enclosed in double quotes, as is customary in Isabelle. |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
249 |
*} |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
250 |
|
52824 | 251 |
|
53621 | 252 |
subsubsection {* Simple Recursion |
253 |
\label{sssec:datatype-simple-recursion} *} |
|
52794 | 254 |
|
52805 | 255 |
text {* |
53491 | 256 |
Natural numbers are the simplest example of a recursive type: |
52805 | 257 |
*} |
258 |
||
53332 | 259 |
datatype_new nat = Zero | Suc nat |
52805 | 260 |
|
261 |
text {* |
|
53491 | 262 |
\noindent |
263 |
Lists were shown in the introduction. Terminated lists are a variant: |
|
52805 | 264 |
*} |
265 |
||
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
266 |
datatype_new (*<*)(in early) (*>*)('a, 'b) tlist = TNil 'b | TCons 'a "('a, 'b) tlist" |
52805 | 267 |
|
52824 | 268 |
|
53621 | 269 |
subsubsection {* Mutual Recursion |
270 |
\label{sssec:datatype-mutual-recursion} *} |
|
52794 | 271 |
|
52805 | 272 |
text {* |
53552 | 273 |
\emph{Mutually recursive} types are introduced simultaneously and may refer to |
274 |
each other. The example below introduces a pair of types for even and odd |
|
275 |
natural numbers: |
|
52805 | 276 |
*} |
277 |
||
53623 | 278 |
datatype_new even_nat = Even_Zero | Even_Suc odd_nat |
279 |
and odd_nat = Odd_Suc even_nat |
|
52805 | 280 |
|
281 |
text {* |
|
53491 | 282 |
\noindent |
283 |
Arithmetic expressions are defined via terms, terms via factors, and factors via |
|
284 |
expressions: |
|
52805 | 285 |
*} |
286 |
||
52841 | 287 |
datatype_new ('a, 'b) exp = |
288 |
Term "('a, 'b) trm" | Sum "('a, 'b) trm" "('a, 'b) exp" |
|
52805 | 289 |
and ('a, 'b) trm = |
52841 | 290 |
Factor "('a, 'b) fct" | Prod "('a, 'b) fct" "('a, 'b) trm" |
291 |
and ('a, 'b) fct = |
|
292 |
Const 'a | Var 'b | Expr "('a, 'b) exp" |
|
52805 | 293 |
|
52824 | 294 |
|
53621 | 295 |
subsubsection {* Nested Recursion |
296 |
\label{sssec:datatype-nested-recursion} *} |
|
52794 | 297 |
|
52805 | 298 |
text {* |
53491 | 299 |
\emph{Nested recursion} occurs when recursive occurrences of a type appear under |
300 |
a type constructor. The introduction showed some examples of trees with nesting |
|
53675 | 301 |
through lists. A more complex example, that reuses our @{type option} type, |
53491 | 302 |
follows: |
52805 | 303 |
*} |
304 |
||
52843 | 305 |
datatype_new 'a btree = |
53025 | 306 |
BNode 'a "'a btree option" "'a btree option" |
52805 | 307 |
|
308 |
text {* |
|
53491 | 309 |
\noindent |
310 |
Not all nestings are admissible. For example, this command will fail: |
|
52805 | 311 |
*} |
312 |
||
53491 | 313 |
datatype_new 'a wrong = Wrong (*<*)'a |
53542 | 314 |
typ (*>*)"'a wrong \<Rightarrow> 'a" |
52806 | 315 |
|
316 |
text {* |
|
53491 | 317 |
\noindent |
318 |
The issue is that the function arrow @{text "\<Rightarrow>"} allows recursion |
|
319 |
only through its right-hand side. This issue is inherited by polymorphic |
|
320 |
datatypes defined in terms of~@{text "\<Rightarrow>"}: |
|
321 |
*} |
|
322 |
||
323 |
datatype_new ('a, 'b) fn = Fn "'a \<Rightarrow> 'b" |
|
324 |
datatype_new 'a also_wrong = Also_Wrong (*<*)'a |
|
53542 | 325 |
typ (*>*)"('a also_wrong, 'a) fn" |
53491 | 326 |
|
327 |
text {* |
|
328 |
\noindent |
|
53621 | 329 |
This is legal: |
330 |
*} |
|
331 |
||
332 |
datatype_new 'a ftree = FTLeaf 'a | FTNode "'a \<Rightarrow> 'a ftree" |
|
333 |
||
334 |
text {* |
|
335 |
\noindent |
|
53491 | 336 |
In general, type constructors @{text "('a\<^sub>1, \<dots>, 'a\<^sub>m) t"} |
337 |
allow recursion on a subset of their type arguments @{text 'a\<^sub>1}, \ldots, |
|
338 |
@{text 'a\<^sub>m}. These type arguments are called \emph{live}; the remaining |
|
339 |
type arguments are called \emph{dead}. In @{typ "'a \<Rightarrow> 'b"} and |
|
340 |
@{typ "('a, 'b) fn"}, the type variable @{typ 'a} is dead and @{typ 'b} is live. |
|
53552 | 341 |
|
53647 | 342 |
Type constructors must be registered as BNFs to have live arguments. This is |
343 |
done automatically for datatypes and codatatypes introduced by the @{command |
|
53829 | 344 |
datatype_new} and @{command codatatype} commands. |
53552 | 345 |
Section~\ref{sec:registering-bounded-natural-functors} explains how to register |
346 |
arbitrary type constructors as BNFs. |
|
52806 | 347 |
*} |
348 |
||
349 |
||
53621 | 350 |
subsubsection {* Custom Names and Syntaxes |
351 |
\label{sssec:datatype-custom-names-and-syntaxes} *} |
|
52805 | 352 |
|
353 |
text {* |
|
53491 | 354 |
The @{command datatype_new} command introduces various constants in addition to |
53617 | 355 |
the constructors. With each datatype are associated set functions, a map |
356 |
function, a relator, discriminators, and selectors, all of which can be given |
|
357 |
custom names. In the example below, the traditional names |
|
358 |
@{text set}, @{text map}, @{text list_all2}, @{text null}, @{text hd}, and |
|
359 |
@{text tl} override the default names @{text list_set}, @{text list_map}, @{text |
|
360 |
list_rel}, @{text is_Nil}, @{text un_Cons1}, and @{text un_Cons2}: |
|
52822 | 361 |
*} |
362 |
||
52841 | 363 |
(*<*) |
364 |
no_translations |
|
365 |
"[x, xs]" == "x # [xs]" |
|
366 |
"[x]" == "x # []" |
|
367 |
||
368 |
no_notation |
|
369 |
Nil ("[]") and |
|
370 |
Cons (infixr "#" 65) |
|
371 |
||
53543 | 372 |
hide_type list |
53544 | 373 |
hide_const Nil Cons hd tl set map list_all2 list_case list_rec |
53025 | 374 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
375 |
context early begin |
52841 | 376 |
(*>*) |
53025 | 377 |
datatype_new (set: 'a) list (map: map rel: list_all2) = |
52822 | 378 |
null: Nil (defaults tl: Nil) |
53025 | 379 |
| Cons (hd: 'a) (tl: "'a list") |
52822 | 380 |
|
381 |
text {* |
|
382 |
\noindent |
|
383 |
The command introduces a discriminator @{const null} and a pair of selectors |
|
384 |
@{const hd} and @{const tl} characterized as follows: |
|
385 |
% |
|
53025 | 386 |
\[@{thm list.collapse(1)[of xs, no_vars]} |
387 |
\qquad @{thm list.collapse(2)[of xs, no_vars]}\] |
|
52822 | 388 |
% |
389 |
For two-constructor datatypes, a single discriminator constant suffices. The |
|
53491 | 390 |
discriminator associated with @{const Cons} is simply |
391 |
@{term "\<lambda>xs. \<not> null xs"}. |
|
52822 | 392 |
|
53553 | 393 |
The @{text defaults} clause following the @{const Nil} constructor specifies a |
394 |
default value for selectors associated with other constructors. Here, it is used |
|
395 |
to ensure that the tail of the empty list is itself (instead of being left |
|
53535 | 396 |
unspecified). |
52822 | 397 |
|
53617 | 398 |
Because @{const Nil} is nullary, it is also possible to use |
53491 | 399 |
@{term "\<lambda>xs. xs = Nil"} as a discriminator. This is specified by |
53534 | 400 |
entering ``@{text "="}'' instead of the identifier @{const null}. Although this |
53535 | 401 |
may look appealing, the mixture of constructors and selectors in the |
53534 | 402 |
characteristic theorems can lead Isabelle's automation to switch between the |
403 |
constructor and the destructor view in surprising ways. |
|
52822 | 404 |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
405 |
The usual mixfix syntax annotations are available for both types and |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
406 |
constructors. For example: |
52805 | 407 |
*} |
52794 | 408 |
|
53025 | 409 |
(*<*) |
410 |
end |
|
411 |
(*>*) |
|
53552 | 412 |
datatype_new ('a, 'b) prod (infixr "*" 20) = Pair 'a 'b |
413 |
||
414 |
text {* \blankline *} |
|
52822 | 415 |
|
52841 | 416 |
datatype_new (set: 'a) list (map: map rel: list_all2) = |
52822 | 417 |
null: Nil ("[]") |
52841 | 418 |
| Cons (hd: 'a) (tl: "'a list") (infixr "#" 65) |
419 |
||
420 |
text {* |
|
53535 | 421 |
\noindent |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
422 |
Incidentally, this is how the traditional syntax can be set up: |
52841 | 423 |
*} |
424 |
||
425 |
syntax "_list" :: "args \<Rightarrow> 'a list" ("[(_)]") |
|
426 |
||
53552 | 427 |
text {* \blankline *} |
428 |
||
52841 | 429 |
translations |
430 |
"[x, xs]" == "x # [xs]" |
|
431 |
"[x]" == "x # []" |
|
52822 | 432 |
|
52824 | 433 |
|
53617 | 434 |
subsection {* Command Syntax |
435 |
\label{ssec:datatype-command-syntax} *} |
|
436 |
||
437 |
||
53621 | 438 |
subsubsection {* \keyw{datatype\_new} |
439 |
\label{sssec:datatype-new} *} |
|
52794 | 440 |
|
52822 | 441 |
text {* |
53829 | 442 |
\begin{matharray}{rcl} |
443 |
@{command_def "datatype_new"} & : & @{text "local_theory \<rightarrow> local_theory"} |
|
444 |
\end{matharray} |
|
52822 | 445 |
|
52824 | 446 |
@{rail " |
53829 | 447 |
@@{command datatype_new} target? @{syntax dt_options}? \\ |
52824 | 448 |
(@{syntax dt_name} '=' (@{syntax ctor} + '|') + @'and') |
52828 | 449 |
; |
53623 | 450 |
@{syntax_def dt_options}: '(' (('no_discs_sels' | 'rep_compat') + ',') ')' |
52824 | 451 |
"} |
452 |
||
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
453 |
The syntactic entity \synt{target} can be used to specify a local |
53534 | 454 |
context---e.g., @{text "(in linorder)"}. It is documented in the Isar reference |
455 |
manual \cite{isabelle-isar-ref}. |
|
456 |
% |
|
457 |
The optional target is optionally followed by datatype-specific options: |
|
52822 | 458 |
|
52824 | 459 |
\begin{itemize} |
460 |
\setlength{\itemsep}{0pt} |
|
461 |
||
462 |
\item |
|
53623 | 463 |
The @{text "no_discs_sels"} option indicates that no discriminators or selectors |
53543 | 464 |
should be generated. |
52822 | 465 |
|
52824 | 466 |
\item |
53644 | 467 |
The @{text "rep_compat"} option indicates that the generated names should |
468 |
contain optional (and normally not displayed) ``@{text "new."}'' components to |
|
469 |
prevent clashes with a later call to \keyw{rep\_datatype}. See |
|
52824 | 470 |
Section~\ref{ssec:datatype-compatibility-issues} for details. |
471 |
\end{itemize} |
|
52822 | 472 |
|
52827 | 473 |
The left-hand sides of the datatype equations specify the name of the type to |
53534 | 474 |
define, its type parameters, and additional information: |
52822 | 475 |
|
52824 | 476 |
@{rail " |
53534 | 477 |
@{syntax_def dt_name}: @{syntax tyargs}? name @{syntax map_rel}? mixfix? |
52824 | 478 |
; |
53534 | 479 |
@{syntax_def tyargs}: typefree | '(' ((name ':')? typefree + ',') ')' |
52824 | 480 |
; |
53534 | 481 |
@{syntax_def map_rel}: '(' ((('map' | 'rel') ':' name) +) ')' |
52824 | 482 |
"} |
52822 | 483 |
|
52827 | 484 |
\noindent |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
485 |
The syntactic entity \synt{name} denotes an identifier, \synt{typefree} |
53534 | 486 |
denotes fixed type variable (@{typ 'a}, @{typ 'b}, \ldots), and \synt{mixfix} |
487 |
denotes the usual parenthesized mixfix notation. They are documented in the Isar |
|
488 |
reference manual \cite{isabelle-isar-ref}. |
|
52822 | 489 |
|
52827 | 490 |
The optional names preceding the type variables allow to override the default |
491 |
names of the set functions (@{text t_set1}, \ldots, @{text t_setM}). |
|
53647 | 492 |
Inside a mutually recursive specification, all defined datatypes must |
493 |
mention exactly the same type variables in the same order. |
|
52822 | 494 |
|
52824 | 495 |
@{rail " |
53534 | 496 |
@{syntax_def ctor}: (name ':')? name (@{syntax ctor_arg} * ) \\ |
497 |
@{syntax dt_sel_defaults}? mixfix? |
|
52824 | 498 |
"} |
499 |
||
53535 | 500 |
\medskip |
501 |
||
52827 | 502 |
\noindent |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
503 |
The main constituents of a constructor specification are the name of the |
52827 | 504 |
constructor and the list of its argument types. An optional discriminator name |
53554 | 505 |
can be supplied at the front to override the default name |
506 |
(@{text t.is_C\<^sub>j}). |
|
52822 | 507 |
|
52824 | 508 |
@{rail " |
53534 | 509 |
@{syntax_def ctor_arg}: type | '(' name ':' type ')' |
52827 | 510 |
"} |
511 |
||
53535 | 512 |
\medskip |
513 |
||
52827 | 514 |
\noindent |
515 |
In addition to the type of a constructor argument, it is possible to specify a |
|
516 |
name for the corresponding selector to override the default name |
|
53554 | 517 |
(@{text un_C\<^sub>ji}). The same selector names can be reused for several |
518 |
constructors as long as they share the same type. |
|
52827 | 519 |
|
520 |
@{rail " |
|
53621 | 521 |
@{syntax_def dt_sel_defaults}: '(' 'defaults' (name ':' term +) ')' |
52824 | 522 |
"} |
52827 | 523 |
|
524 |
\noindent |
|
525 |
Given a constructor |
|
526 |
@{text "C \<Colon> \<sigma>\<^sub>1 \<Rightarrow> \<dots> \<Rightarrow> \<sigma>\<^sub>p \<Rightarrow> \<sigma>"}, |
|
527 |
default values can be specified for any selector |
|
528 |
@{text "un_D \<Colon> \<sigma> \<Rightarrow> \<tau>"} |
|
53535 | 529 |
associated with other constructors. The specified default value must be of type |
52828 | 530 |
@{text "\<sigma>\<^sub>1 \<Rightarrow> \<dots> \<Rightarrow> \<sigma>\<^sub>p \<Rightarrow> \<tau>"} |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
531 |
(i.e., it may depend on @{text C}'s arguments). |
52822 | 532 |
*} |
533 |
||
53617 | 534 |
|
53621 | 535 |
subsubsection {* \keyw{datatype\_new\_compat} |
536 |
\label{sssec:datatype-new-compat} *} |
|
53617 | 537 |
|
538 |
text {* |
|
53829 | 539 |
\begin{matharray}{rcl} |
540 |
@{command_def "datatype_new_compat"} & : & @{text "local_theory \<rightarrow> local_theory"} |
|
541 |
\end{matharray} |
|
542 |
||
543 |
@{rail " |
|
544 |
@@{command datatype_new_compat} names |
|
545 |
"} |
|
546 |
||
547 |
\noindent |
|
53621 | 548 |
The old datatype package provides some functionality that is not yet replicated |
549 |
in the new package: |
|
550 |
||
551 |
\begin{itemize} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
552 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
553 |
|
53621 | 554 |
\item It is integrated with \keyw{fun} and \keyw{function} |
555 |
\cite{isabelle-function}, Nitpick \cite{isabelle-nitpick}, Quickcheck, |
|
556 |
and other packages. |
|
557 |
||
558 |
\item It is extended by various add-ons, notably to produce instances of the |
|
559 |
@{const size} function. |
|
560 |
\end{itemize} |
|
561 |
||
562 |
\noindent |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
563 |
New-style datatypes can in most cases be registered as old-style datatypes using |
53829 | 564 |
@{command datatype_new_compat}. The \textit{names} argument is a space-separated |
565 |
list of type names that are mutually recursive. For example: |
|
53621 | 566 |
*} |
567 |
||
53623 | 568 |
datatype_new_compat even_nat odd_nat |
53621 | 569 |
|
570 |
text {* \blankline *} |
|
571 |
||
53623 | 572 |
thm even_nat_odd_nat.size |
53621 | 573 |
|
574 |
text {* \blankline *} |
|
575 |
||
53623 | 576 |
ML {* Datatype_Data.get_info @{theory} @{type_name even_nat} *} |
53621 | 577 |
|
578 |
text {* |
|
53748 | 579 |
A few remarks concern nested recursive datatypes only: |
580 |
||
581 |
\begin{itemize} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
582 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
583 |
|
53748 | 584 |
\item The old-style, nested-as-mutual induction rule, iterator theorems, and |
585 |
recursor theorems are generated under their usual names but with ``@{text |
|
586 |
"compat_"}'' prefixed (e.g., @{text compat_tree.induct}). |
|
587 |
||
588 |
\item All types through which recursion takes place must be new-style datatypes |
|
589 |
or the function type. In principle, it should be possible to support old-style |
|
590 |
datatypes as well, but the command does not support this yet (and there is |
|
591 |
currently no way to register old-style datatypes as new-style datatypes). |
|
592 |
\end{itemize} |
|
593 |
||
594 |
An alternative to @{command datatype_new_compat} is to use the old package's |
|
595 |
\keyw{rep\_datatype} command. The associated proof obligations must then be |
|
596 |
discharged manually. |
|
53617 | 597 |
*} |
598 |
||
599 |
||
600 |
subsection {* Generated Constants |
|
601 |
\label{ssec:datatype-generated-constants} *} |
|
602 |
||
603 |
text {* |
|
53623 | 604 |
Given a datatype @{text "('a\<^sub>1, \<dots>, 'a\<^sub>m) t"} |
53617 | 605 |
with $m > 0$ live type variables and $n$ constructors |
606 |
@{text "t.C\<^sub>1"}, \ldots, @{text "t.C\<^sub>n"}, the |
|
607 |
following auxiliary constants are introduced: |
|
608 |
||
609 |
\begin{itemize} |
|
610 |
\setlength{\itemsep}{0pt} |
|
611 |
||
612 |
\item \relax{Case combinator}: @{text t_case} (rendered using the familiar |
|
613 |
@{text case}--@{text of} syntax) |
|
614 |
||
615 |
\item \relax{Discriminators}: @{text "t.is_C\<^sub>1"}, \ldots, |
|
616 |
@{text "t.is_C\<^sub>n"} |
|
617 |
||
618 |
\item \relax{Selectors}: |
|
619 |
@{text t.un_C\<^sub>11}$, \ldots, @{text t.un_C\<^sub>1k\<^sub>1}, \\ |
|
620 |
\phantom{\relax{Selectors:}} \quad\vdots \\ |
|
621 |
\phantom{\relax{Selectors:}} @{text t.un_C\<^sub>n1}$, \ldots, @{text t.un_C\<^sub>nk\<^sub>n}. |
|
622 |
||
623 |
\item \relax{Set functions} (or \relax{natural transformations}): |
|
624 |
@{text t_set1}, \ldots, @{text t_setm} |
|
625 |
||
626 |
\item \relax{Map function} (or \relax{functorial action}): @{text t_map} |
|
627 |
||
628 |
\item \relax{Relator}: @{text t_rel} |
|
629 |
||
630 |
\item \relax{Iterator}: @{text t_fold} |
|
631 |
||
632 |
\item \relax{Recursor}: @{text t_rec} |
|
633 |
||
634 |
\end{itemize} |
|
635 |
||
636 |
\noindent |
|
637 |
The case combinator, discriminators, and selectors are collectively called |
|
638 |
\emph{destructors}. The prefix ``@{text "t."}'' is an optional component of the |
|
639 |
name and is normally hidden. |
|
640 |
*} |
|
641 |
||
642 |
||
52840 | 643 |
subsection {* Generated Theorems |
644 |
\label{ssec:datatype-generated-theorems} *} |
|
52828 | 645 |
|
646 |
text {* |
|
53544 | 647 |
The characteristic theorems generated by @{command datatype_new} are grouped in |
53623 | 648 |
three broad categories: |
53535 | 649 |
|
53543 | 650 |
\begin{itemize} |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
651 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
652 |
|
53543 | 653 |
\item The \emph{free constructor theorems} are properties about the constructors |
654 |
and destructors that can be derived for any freely generated type. Internally, |
|
53542 | 655 |
the derivation is performed by @{command wrap_free_constructors}. |
53535 | 656 |
|
53552 | 657 |
\item The \emph{functorial theorems} are properties of datatypes related to |
658 |
their BNF nature. |
|
659 |
||
660 |
\item The \emph{inductive theorems} are properties of datatypes related to |
|
53544 | 661 |
their inductive nature. |
53552 | 662 |
|
53543 | 663 |
\end{itemize} |
53535 | 664 |
|
665 |
\noindent |
|
53542 | 666 |
The full list of named theorems can be obtained as usual by entering the |
53543 | 667 |
command \keyw{print\_theorems} immediately after the datatype definition. |
53542 | 668 |
This list normally excludes low-level theorems that reveal internal |
53552 | 669 |
constructions. To make these accessible, add the line |
53542 | 670 |
*} |
53535 | 671 |
|
53542 | 672 |
declare [[bnf_note_all]] |
673 |
(*<*) |
|
674 |
declare [[bnf_note_all = false]] |
|
675 |
(*>*) |
|
53535 | 676 |
|
53552 | 677 |
text {* |
678 |
\noindent |
|
679 |
to the top of the theory file. |
|
680 |
*} |
|
53535 | 681 |
|
53621 | 682 |
subsubsection {* Free Constructor Theorems |
683 |
\label{sssec:free-constructor-theorems} *} |
|
53535 | 684 |
|
53543 | 685 |
(*<*) |
53837 | 686 |
consts nonnull :: 'a |
53543 | 687 |
(*>*) |
688 |
||
53535 | 689 |
text {* |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
690 |
The first subgroup of properties is concerned with the constructors. |
53543 | 691 |
They are listed below for @{typ "'a list"}: |
692 |
||
53552 | 693 |
\begin{indentblock} |
53543 | 694 |
\begin{description} |
53544 | 695 |
|
53642 | 696 |
\item[@{text "t."}\hthm{inject} @{text "[iff, induct_simp]"}\rm:] ~ \\ |
53544 | 697 |
@{thm list.inject[no_vars]} |
698 |
||
53642 | 699 |
\item[@{text "t."}\hthm{distinct} @{text "[simp, induct_simp]"}\rm:] ~ \\ |
53543 | 700 |
@{thm list.distinct(1)[no_vars]} \\ |
701 |
@{thm list.distinct(2)[no_vars]} |
|
702 |
||
53642 | 703 |
\item[@{text "t."}\hthm{exhaust} @{text "[cases t, case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
53543 | 704 |
@{thm list.exhaust[no_vars]} |
705 |
||
53642 | 706 |
\item[@{text "t."}\hthm{nchotomy}\rm:] ~ \\ |
53543 | 707 |
@{thm list.nchotomy[no_vars]} |
708 |
||
709 |
\end{description} |
|
53552 | 710 |
\end{indentblock} |
53543 | 711 |
|
712 |
\noindent |
|
53621 | 713 |
In addition, these nameless theorems are registered as safe elimination rules: |
714 |
||
715 |
\begin{indentblock} |
|
716 |
\begin{description} |
|
717 |
||
53642 | 718 |
\item[@{text "t."}\hthm{list.distinct {\upshape[}THEN notE}@{text ", elim!"}\hthm{\upshape]}\rm:] ~ \\ |
53621 | 719 |
@{thm list.distinct(1)[THEN notE, elim!, no_vars]} \\ |
720 |
@{thm list.distinct(2)[THEN notE, elim!, no_vars]} |
|
721 |
||
722 |
\end{description} |
|
723 |
\end{indentblock} |
|
724 |
||
725 |
\noindent |
|
53543 | 726 |
The next subgroup is concerned with the case combinator: |
727 |
||
53552 | 728 |
\begin{indentblock} |
53543 | 729 |
\begin{description} |
53544 | 730 |
|
53798 | 731 |
\item[@{text "t."}\hthm{case} @{text "[simp, code]"}\rm:] ~ \\ |
53543 | 732 |
@{thm list.case(1)[no_vars]} \\ |
733 |
@{thm list.case(2)[no_vars]} |
|
734 |
||
53642 | 735 |
\item[@{text "t."}\hthm{case\_cong}\rm:] ~ \\ |
53543 | 736 |
@{thm list.case_cong[no_vars]} |
737 |
||
53642 | 738 |
\item[@{text "t."}\hthm{weak\_case\_cong} @{text "[cong]"}\rm:] ~ \\ |
53543 | 739 |
@{thm list.weak_case_cong[no_vars]} |
740 |
||
53642 | 741 |
\item[@{text "t."}\hthm{split}\rm:] ~ \\ |
53543 | 742 |
@{thm list.split[no_vars]} |
743 |
||
53642 | 744 |
\item[@{text "t."}\hthm{split\_asm}\rm:] ~ \\ |
53543 | 745 |
@{thm list.split_asm[no_vars]} |
746 |
||
53544 | 747 |
\item[@{text "t."}\hthm{splits} = @{text "split split_asm"}] |
53543 | 748 |
|
749 |
\end{description} |
|
53552 | 750 |
\end{indentblock} |
53543 | 751 |
|
752 |
\noindent |
|
753 |
The third and last subgroup revolves around discriminators and selectors: |
|
754 |
||
53552 | 755 |
\begin{indentblock} |
53543 | 756 |
\begin{description} |
53544 | 757 |
|
53694 | 758 |
\item[@{text "t."}\hthm{disc} @{text "[simp]"}\rm:] ~ \\ |
759 |
@{thm list.disc(1)[no_vars]} \\ |
|
760 |
@{thm list.disc(2)[no_vars]} |
|
761 |
||
53703 | 762 |
\item[@{text "t."}\hthm{discI}\rm:] ~ \\ |
763 |
@{thm list.discI(1)[no_vars]} \\ |
|
764 |
@{thm list.discI(2)[no_vars]} |
|
765 |
||
53805 | 766 |
\item[@{text "t."}\hthm{sel} @{text "[simp, code]"}\rm:] ~ \\ |
53694 | 767 |
@{thm list.sel(1)[no_vars]} \\ |
768 |
@{thm list.sel(2)[no_vars]} |
|
53543 | 769 |
|
53642 | 770 |
\item[@{text "t."}\hthm{collapse} @{text "[simp]"}\rm:] ~ \\ |
53543 | 771 |
@{thm list.collapse(1)[no_vars]} \\ |
772 |
@{thm list.collapse(2)[no_vars]} |
|
773 |
||
53837 | 774 |
\item[@{text "t."}\hthm{disc\_exclude} @{text "[dest]"}\rm:] ~ \\ |
53543 | 775 |
These properties are missing for @{typ "'a list"} because there is only one |
776 |
proper discriminator. Had the datatype been introduced with a second |
|
53837 | 777 |
discriminator called @{const nonnull}, they would have read thusly: \\[\jot] |
778 |
@{prop "null list \<Longrightarrow> \<not> nonnull list"} \\ |
|
779 |
@{prop "nonnull list \<Longrightarrow> \<not> null list"} |
|
53543 | 780 |
|
53642 | 781 |
\item[@{text "t."}\hthm{disc\_exhaust} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
53543 | 782 |
@{thm list.disc_exhaust[no_vars]} |
783 |
||
53916 | 784 |
\item[@{text "t."}\hthm{sel\_exhaust} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
785 |
@{thm list.sel_exhaust[no_vars]} |
|
786 |
||
53642 | 787 |
\item[@{text "t."}\hthm{expand}\rm:] ~ \\ |
53543 | 788 |
@{thm list.expand[no_vars]} |
789 |
||
53917 | 790 |
\item[@{text "t."}\hthm{sel\_split}\rm:] ~ \\ |
791 |
@{thm list.sel_split[no_vars]} |
|
792 |
||
793 |
\item[@{text "t."}\hthm{sel\_split\_asm}\rm:] ~ \\ |
|
794 |
@{thm list.sel_split_asm[no_vars]} |
|
795 |
||
53857 | 796 |
\item[@{text "t."}\hthm{case\_conv\_if}\rm:] ~ \\ |
797 |
@{thm list.case_conv_if[no_vars]} |
|
53543 | 798 |
|
799 |
\end{description} |
|
53552 | 800 |
\end{indentblock} |
801 |
*} |
|
802 |
||
803 |
||
53621 | 804 |
subsubsection {* Functorial Theorems |
805 |
\label{sssec:functorial-theorems} *} |
|
53552 | 806 |
|
807 |
text {* |
|
53623 | 808 |
The BNF-related theorem are as follows: |
53552 | 809 |
|
810 |
\begin{indentblock} |
|
811 |
\begin{description} |
|
812 |
||
53798 | 813 |
\item[@{text "t."}\hthm{set} @{text "[simp, code]"}\rm:] ~ \\ |
53694 | 814 |
@{thm list.set(1)[no_vars]} \\ |
815 |
@{thm list.set(2)[no_vars]} |
|
53552 | 816 |
|
53798 | 817 |
\item[@{text "t."}\hthm{map} @{text "[simp, code]"}\rm:] ~ \\ |
53552 | 818 |
@{thm list.map(1)[no_vars]} \\ |
819 |
@{thm list.map(2)[no_vars]} |
|
820 |
||
53798 | 821 |
\item[@{text "t."}\hthm{rel\_inject} @{text "[simp, code]"}\rm:] ~ \\ |
53552 | 822 |
@{thm list.rel_inject(1)[no_vars]} \\ |
823 |
@{thm list.rel_inject(2)[no_vars]} |
|
824 |
||
53798 | 825 |
\item[@{text "t."}\hthm{rel\_distinct} @{text "[simp, code]"}\rm:] ~ \\ |
53552 | 826 |
@{thm list.rel_distinct(1)[no_vars]} \\ |
827 |
@{thm list.rel_distinct(2)[no_vars]} |
|
828 |
||
829 |
\end{description} |
|
830 |
\end{indentblock} |
|
53535 | 831 |
*} |
832 |
||
833 |
||
53621 | 834 |
subsubsection {* Inductive Theorems |
835 |
\label{sssec:inductive-theorems} *} |
|
53535 | 836 |
|
837 |
text {* |
|
53623 | 838 |
The inductive theorems are as follows: |
53544 | 839 |
|
53552 | 840 |
\begin{indentblock} |
53544 | 841 |
\begin{description} |
842 |
||
53642 | 843 |
\item[@{text "t."}\hthm{induct} @{text "[induct t, case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
53544 | 844 |
@{thm list.induct[no_vars]} |
845 |
||
53642 | 846 |
\item[@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{induct} @{text "[case_names C\<^sub>1 \<dots> C\<^sub>n]"}\rm:] ~ \\ |
53544 | 847 |
Given $m > 1$ mutually recursive datatypes, this induction rule can be used to |
848 |
prove $m$ properties simultaneously. |
|
52828 | 849 |
|
53798 | 850 |
\item[@{text "t."}\hthm{fold} @{text "[simp, code]"}\rm:] ~ \\ |
53544 | 851 |
@{thm list.fold(1)[no_vars]} \\ |
852 |
@{thm list.fold(2)[no_vars]} |
|
853 |
||
53798 | 854 |
\item[@{text "t."}\hthm{rec} @{text "[simp, code]"}\rm:] ~ \\ |
53544 | 855 |
@{thm list.rec(1)[no_vars]} \\ |
856 |
@{thm list.rec(2)[no_vars]} |
|
857 |
||
858 |
\end{description} |
|
53552 | 859 |
\end{indentblock} |
53544 | 860 |
|
861 |
\noindent |
|
862 |
For convenience, @{command datatype_new} also provides the following collection: |
|
863 |
||
53552 | 864 |
\begin{indentblock} |
53544 | 865 |
\begin{description} |
866 |
||
867 |
\item[@{text "t."}\hthm{simps} = @{text t.inject} @{text t.distinct} @{text t.case} @{text t.rec} @{text t.fold} @{text t.map} @{text t.rel_inject}] ~ \\ |
|
53694 | 868 |
@{text t.rel_distinct} @{text t.set} |
53544 | 869 |
|
870 |
\end{description} |
|
53552 | 871 |
\end{indentblock} |
52828 | 872 |
*} |
873 |
||
52794 | 874 |
|
52827 | 875 |
subsection {* Compatibility Issues |
52824 | 876 |
\label{ssec:datatype-compatibility-issues} *} |
52794 | 877 |
|
52828 | 878 |
text {* |
53997 | 879 |
The command @{command datatype_new} has been designed to be highly compatible |
880 |
with the old \keyw{datatype}, to ease migration. There are nonetheless a few |
|
53647 | 881 |
incompatibilities that may arise when porting to the new package: |
882 |
||
883 |
\begin{itemize} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
884 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
885 |
|
53647 | 886 |
\item \emph{The Standard ML interfaces are different.} Tools and extensions |
887 |
written to call the old ML interfaces will need to be adapted to the new |
|
888 |
interfaces. Little has been done so far in this direction. Whenever possible, it |
|
889 |
is recommended to use @{command datatype_new_compat} or \keyw{rep\_datatype} |
|
890 |
to register new-style datatypes as old-style datatypes. |
|
891 |
||
892 |
\item \emph{The recursor @{text "t_rec"} has a different signature for nested |
|
893 |
recursive datatypes.} In the old package, nested recursion was internally |
|
894 |
reduced to mutual recursion. This reduction was visible in the type of the |
|
895 |
recursor, used by \keyw{primrec}. In the new package, nested recursion is |
|
896 |
handled in a more modular fashion. The old-style recursor can be generated on |
|
897 |
demand using @{command primrec_new}, as explained in |
|
898 |
Section~\ref{sssec:primrec-nested-as-mutual-recursion}, if the recursion is via |
|
899 |
new-style datatypes. |
|
900 |
||
901 |
\item \emph{Accordingly, the induction principle is different for nested |
|
902 |
recursive datatypes.} Again, the old-style induction principle can be generated |
|
903 |
on demand using @{command primrec_new}, as explained in |
|
904 |
Section~\ref{sssec:primrec-nested-as-mutual-recursion}, if the recursion is via |
|
905 |
new-style datatypes. |
|
52828 | 906 |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
907 |
\item \emph{The internal constructions are completely different.} Proof texts |
53647 | 908 |
that unfold the definition of constants introduced by \keyw{datatype} will be |
909 |
difficult to port. |
|
910 |
||
911 |
\item \emph{A few theorems have different names.} |
|
53997 | 912 |
The properties @{text t.cases} and @{text t.recs} have been renamed |
53647 | 913 |
@{text t.case} and @{text t.rec}. For non-mutually recursive datatypes, |
914 |
@{text t.inducts} is available as @{text t.induct}. |
|
915 |
For $m > 1$ mutually recursive datatypes, |
|
53997 | 916 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m.inducts(i)"} has been renamed |
53647 | 917 |
@{text "t\<^sub>i.induct"}. |
918 |
||
919 |
\item \emph{The @{text t.simps} collection has been extended.} |
|
920 |
Previously available theorems are available at the same index. |
|
921 |
||
922 |
\item \emph{Variables in generated properties have different names.} This is |
|
923 |
rarely an issue, except in proof texts that refer to variable names in the |
|
924 |
@{text "[where \<dots>]"} attribute. The solution is to use the more robust |
|
925 |
@{text "[of \<dots>]"} syntax. |
|
926 |
\end{itemize} |
|
927 |
||
928 |
In the other direction, there is currently no way to register old-style |
|
929 |
datatypes as new-style datatypes. If the goal is to define new-style datatypes |
|
930 |
with nested recursion through old-style datatypes, the old-style |
|
931 |
datatypes can be registered as a BNF |
|
932 |
(Section~\ref{sec:registering-bounded-natural-functors}). If the goal is |
|
933 |
to derive discriminators and selectors, this can be achieved using @{command |
|
934 |
wrap_free_constructors} |
|
935 |
(Section~\ref{sec:deriving-destructors-and-theorems-for-free-constructors}). |
|
52828 | 936 |
*} |
937 |
||
52792 | 938 |
|
52827 | 939 |
section {* Defining Recursive Functions |
52805 | 940 |
\label{sec:defining-recursive-functions} *} |
941 |
||
942 |
text {* |
|
53644 | 943 |
Recursive functions over datatypes can be specified using @{command |
944 |
primrec_new}, which supports primitive recursion, or using the more general |
|
945 |
\keyw{fun} and \keyw{function} commands. Here, the focus is on @{command |
|
946 |
primrec_new}; the other two commands are described in a separate tutorial |
|
53646 | 947 |
\cite{isabelle-function}. |
52828 | 948 |
|
53621 | 949 |
%%% TODO: partial_function |
52805 | 950 |
*} |
52792 | 951 |
|
52805 | 952 |
|
53617 | 953 |
subsection {* Introductory Examples |
954 |
\label{ssec:primrec-introductory-examples} *} |
|
52828 | 955 |
|
53646 | 956 |
text {* |
957 |
Primitive recursion is illustrated through concrete examples based on the |
|
958 |
datatypes defined in Section~\ref{ssec:datatype-introductory-examples}. More |
|
959 |
examples can be found in the directory \verb|~~/src/HOL/BNF/Examples|. |
|
960 |
*} |
|
961 |
||
53621 | 962 |
|
963 |
subsubsection {* Nonrecursive Types |
|
964 |
\label{sssec:primrec-nonrecursive-types} *} |
|
52828 | 965 |
|
52841 | 966 |
text {* |
53621 | 967 |
Primitive recursion removes one layer of constructors on the left-hand side in |
968 |
each equation. For example: |
|
52841 | 969 |
*} |
970 |
||
971 |
primrec_new bool_of_trool :: "trool \<Rightarrow> bool" where |
|
53621 | 972 |
"bool_of_trool Faalse \<longleftrightarrow> False" | |
973 |
"bool_of_trool Truue \<longleftrightarrow> True" |
|
52841 | 974 |
|
53621 | 975 |
text {* \blankline *} |
52841 | 976 |
|
53025 | 977 |
primrec_new the_list :: "'a option \<Rightarrow> 'a list" where |
978 |
"the_list None = []" | |
|
979 |
"the_list (Some a) = [a]" |
|
52841 | 980 |
|
53621 | 981 |
text {* \blankline *} |
982 |
||
53025 | 983 |
primrec_new the_default :: "'a \<Rightarrow> 'a option \<Rightarrow> 'a" where |
984 |
"the_default d None = d" | |
|
985 |
"the_default _ (Some a) = a" |
|
52843 | 986 |
|
53621 | 987 |
text {* \blankline *} |
988 |
||
52841 | 989 |
primrec_new mirrror :: "('a, 'b, 'c) triple \<Rightarrow> ('c, 'b, 'a) triple" where |
990 |
"mirrror (Triple a b c) = Triple c b a" |
|
991 |
||
53621 | 992 |
text {* |
993 |
\noindent |
|
994 |
The equations can be specified in any order, and it is acceptable to leave out |
|
995 |
some cases, which are then unspecified. Pattern matching on the left-hand side |
|
996 |
is restricted to a single datatype, which must correspond to the same argument |
|
997 |
in all equations. |
|
998 |
*} |
|
52828 | 999 |
|
53621 | 1000 |
|
1001 |
subsubsection {* Simple Recursion |
|
1002 |
\label{sssec:primrec-simple-recursion} *} |
|
52828 | 1003 |
|
52841 | 1004 |
text {* |
53621 | 1005 |
For simple recursive types, recursive calls on a constructor argument are |
1006 |
allowed on the right-hand side: |
|
52841 | 1007 |
*} |
1008 |
||
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1009 |
primrec_new replicate :: "nat \<Rightarrow> 'a \<Rightarrow> 'a list" where |
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1010 |
"replicate Zero _ = []" | |
53644 | 1011 |
"replicate (Suc n) x = x # replicate n x" |
52841 | 1012 |
|
53621 | 1013 |
text {* \blankline *} |
52843 | 1014 |
|
53332 | 1015 |
primrec_new at :: "'a list \<Rightarrow> nat \<Rightarrow> 'a" where |
53644 | 1016 |
"at (x # xs) j = |
52843 | 1017 |
(case j of |
53644 | 1018 |
Zero \<Rightarrow> x |
1019 |
| Suc j' \<Rightarrow> at xs j')" |
|
52843 | 1020 |
|
53621 | 1021 |
text {* \blankline *} |
1022 |
||
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1023 |
primrec_new (*<*)(in early) (*>*)tfold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> ('a, 'b) tlist \<Rightarrow> 'b" where |
53644 | 1024 |
"tfold _ (TNil y) = y" | |
1025 |
"tfold f (TCons x xs) = f x (tfold f xs)" |
|
52841 | 1026 |
|
53025 | 1027 |
text {* |
53621 | 1028 |
\noindent |
1029 |
The next example is not primitive recursive, but it can be defined easily using |
|
53644 | 1030 |
\keyw{fun}. The @{command datatype_new_compat} command is needed to register |
1031 |
new-style datatypes for use with \keyw{fun} and \keyw{function} |
|
53621 | 1032 |
(Section~\ref{sssec:datatype-new-compat}): |
53025 | 1033 |
*} |
52828 | 1034 |
|
53621 | 1035 |
datatype_new_compat nat |
1036 |
||
1037 |
text {* \blankline *} |
|
1038 |
||
1039 |
fun at_least_two :: "nat \<Rightarrow> bool" where |
|
1040 |
"at_least_two (Suc (Suc _)) \<longleftrightarrow> True" | |
|
1041 |
"at_least_two _ \<longleftrightarrow> False" |
|
1042 |
||
1043 |
||
1044 |
subsubsection {* Mutual Recursion |
|
1045 |
\label{sssec:primrec-mutual-recursion} *} |
|
52828 | 1046 |
|
52841 | 1047 |
text {* |
53621 | 1048 |
The syntax for mutually recursive functions over mutually recursive datatypes |
1049 |
is straightforward: |
|
52841 | 1050 |
*} |
1051 |
||
1052 |
primrec_new |
|
53623 | 1053 |
nat_of_even_nat :: "even_nat \<Rightarrow> nat" and |
1054 |
nat_of_odd_nat :: "odd_nat \<Rightarrow> nat" |
|
52841 | 1055 |
where |
53623 | 1056 |
"nat_of_even_nat Even_Zero = Zero" | |
1057 |
"nat_of_even_nat (Even_Suc n) = Suc (nat_of_odd_nat n)" | |
|
1058 |
"nat_of_odd_nat (Odd_Suc n) = Suc (nat_of_even_nat n)" |
|
52841 | 1059 |
|
53752 | 1060 |
text {* \blankline *} |
1061 |
||
52841 | 1062 |
primrec_new |
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1063 |
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
|
1064 |
eval\<^sub>t :: "('a \<Rightarrow> int) \<Rightarrow> ('b \<Rightarrow> int) \<Rightarrow> ('a, 'b) trm \<Rightarrow> int" and |
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1065 |
eval\<^sub>f :: "('a \<Rightarrow> int) \<Rightarrow> ('b \<Rightarrow> int) \<Rightarrow> ('a, 'b) fct \<Rightarrow> int" |
52841 | 1066 |
where |
1067 |
"eval\<^sub>e \<gamma> \<xi> (Term t) = eval\<^sub>t \<gamma> \<xi> t" | |
|
1068 |
"eval\<^sub>e \<gamma> \<xi> (Sum t e) = eval\<^sub>t \<gamma> \<xi> t + eval\<^sub>e \<gamma> \<xi> e" | |
|
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1069 |
"eval\<^sub>t \<gamma> \<xi> (Factor f) = eval\<^sub>f \<gamma> \<xi> f" | |
52841 | 1070 |
"eval\<^sub>t \<gamma> \<xi> (Prod f t) = eval\<^sub>f \<gamma> \<xi> f + eval\<^sub>t \<gamma> \<xi> t" | |
1071 |
"eval\<^sub>f \<gamma> _ (Const a) = \<gamma> a" | |
|
1072 |
"eval\<^sub>f _ \<xi> (Var b) = \<xi> b" | |
|
1073 |
"eval\<^sub>f \<gamma> \<xi> (Expr e) = eval\<^sub>e \<gamma> \<xi> e" |
|
1074 |
||
53621 | 1075 |
text {* |
1076 |
\noindent |
|
53647 | 1077 |
Mutual recursion is possible within a single type, using \keyw{fun}: |
53621 | 1078 |
*} |
52828 | 1079 |
|
53621 | 1080 |
fun |
1081 |
even :: "nat \<Rightarrow> bool" and |
|
1082 |
odd :: "nat \<Rightarrow> bool" |
|
1083 |
where |
|
1084 |
"even Zero = True" | |
|
1085 |
"even (Suc n) = odd n" | |
|
1086 |
"odd Zero = False" | |
|
1087 |
"odd (Suc n) = even n" |
|
1088 |
||
1089 |
||
1090 |
subsubsection {* Nested Recursion |
|
1091 |
\label{sssec:primrec-nested-recursion} *} |
|
1092 |
||
1093 |
text {* |
|
1094 |
In a departure from the old datatype package, nested recursion is normally |
|
1095 |
handled via the map functions of the nesting type constructors. For example, |
|
1096 |
recursive calls are lifted to lists using @{const map}: |
|
1097 |
*} |
|
52828 | 1098 |
|
52843 | 1099 |
(*<*) |
53644 | 1100 |
datatype_new 'a tree\<^sub>f\<^sub>f = Node\<^sub>f\<^sub>f (lbl\<^sub>f\<^sub>f: 'a) (sub\<^sub>f\<^sub>f: "'a tree\<^sub>f\<^sub>f list") |
52843 | 1101 |
(*>*) |
53028 | 1102 |
primrec_new at\<^sub>f\<^sub>f :: "'a tree\<^sub>f\<^sub>f \<Rightarrow> nat list \<Rightarrow> 'a" where |
1103 |
"at\<^sub>f\<^sub>f (Node\<^sub>f\<^sub>f a ts) js = |
|
52843 | 1104 |
(case js of |
1105 |
[] \<Rightarrow> a |
|
53028 | 1106 |
| j # js' \<Rightarrow> at (map (\<lambda>t. at\<^sub>f\<^sub>f t js') ts) j)" |
52843 | 1107 |
|
53025 | 1108 |
text {* |
53647 | 1109 |
\noindent |
53621 | 1110 |
The next example features recursion through the @{text option} type. Although |
53623 | 1111 |
@{text option} is not a new-style datatype, it is registered as a BNF with the |
53621 | 1112 |
map function @{const option_map}: |
53025 | 1113 |
*} |
52843 | 1114 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1115 |
primrec_new (*<*)(in early) (*>*)sum_btree :: "('a\<Colon>{zero,plus}) btree \<Rightarrow> 'a" where |
52843 | 1116 |
"sum_btree (BNode a lt rt) = |
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1117 |
a + the_default 0 (option_map sum_btree lt) + |
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1118 |
the_default 0 (option_map sum_btree rt)" |
52843 | 1119 |
|
53136 | 1120 |
text {* |
53621 | 1121 |
\noindent |
1122 |
The same principle applies for arbitrary type constructors through which |
|
1123 |
recursion is possible. Notably, the map function for the function type |
|
1124 |
(@{text \<Rightarrow>}) is simply composition (@{text "op \<circ>"}): |
|
53136 | 1125 |
*} |
52828 | 1126 |
|
53621 | 1127 |
primrec_new ftree_map :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a ftree \<Rightarrow> 'a ftree" where |
1128 |
"ftree_map f (FTLeaf x) = FTLeaf (f x)" | |
|
1129 |
"ftree_map f (FTNode g) = FTNode (ftree_map f \<circ> g)" |
|
52828 | 1130 |
|
52843 | 1131 |
text {* |
53621 | 1132 |
\noindent |
1133 |
(No such function is defined by the package because @{typ 'a} is dead in |
|
1134 |
@{typ "'a ftree"}, but we can easily do it ourselves.) |
|
1135 |
*} |
|
1136 |
||
1137 |
||
1138 |
subsubsection {* Nested-as-Mutual Recursion |
|
53644 | 1139 |
\label{sssec:primrec-nested-as-mutual-recursion} *} |
53621 | 1140 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1141 |
(*<*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1142 |
locale n2m begin |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1143 |
(*>*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1144 |
|
53621 | 1145 |
text {* |
1146 |
For compatibility with the old package, but also because it is sometimes |
|
1147 |
convenient in its own right, it is possible to treat nested recursive datatypes |
|
1148 |
as mutually recursive ones if the recursion takes place though new-style |
|
1149 |
datatypes. For example: |
|
52843 | 1150 |
*} |
1151 |
||
53331
20440c789759
prove theorem in the right context (that knows about local variables)
traytel
parents:
53330
diff
changeset
|
1152 |
primrec_new |
53647 | 1153 |
at\<^sub>f\<^sub>f :: "'a tree\<^sub>f\<^sub>f \<Rightarrow> nat list \<Rightarrow> 'a" and |
1154 |
ats\<^sub>f\<^sub>f :: "'a tree\<^sub>f\<^sub>f list \<Rightarrow> nat \<Rightarrow> nat list \<Rightarrow> 'a" |
|
52843 | 1155 |
where |
53647 | 1156 |
"at\<^sub>f\<^sub>f (Node\<^sub>f\<^sub>f a ts) js = |
52843 | 1157 |
(case js of |
1158 |
[] \<Rightarrow> a |
|
53647 | 1159 |
| j # js' \<Rightarrow> ats\<^sub>f\<^sub>f ts j js')" | |
1160 |
"ats\<^sub>f\<^sub>f (t # ts) j = |
|
52843 | 1161 |
(case j of |
53647 | 1162 |
Zero \<Rightarrow> at\<^sub>f\<^sub>f t |
1163 |
| Suc j' \<Rightarrow> ats\<^sub>f\<^sub>f ts j')" |
|
52843 | 1164 |
|
53647 | 1165 |
text {* |
1166 |
\noindent |
|
1167 |
Appropriate induction principles are generated under the names |
|
1168 |
@{thm [source] "at\<^sub>f\<^sub>f.induct"}, |
|
1169 |
@{thm [source] "ats\<^sub>f\<^sub>f.induct"}, and |
|
1170 |
@{thm [source] "at\<^sub>f\<^sub>f_ats\<^sub>f\<^sub>f.induct"}. |
|
1171 |
||
1172 |
%%% TODO: Add recursors. |
|
1173 |
||
1174 |
Here is a second example: |
|
1175 |
*} |
|
53621 | 1176 |
|
53331
20440c789759
prove theorem in the right context (that knows about local variables)
traytel
parents:
53330
diff
changeset
|
1177 |
primrec_new |
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1178 |
sum_btree :: "('a\<Colon>{zero,plus}) btree \<Rightarrow> 'a" and |
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1179 |
sum_btree_option :: "'a btree option \<Rightarrow> 'a" |
52843 | 1180 |
where |
1181 |
"sum_btree (BNode a lt rt) = |
|
53025 | 1182 |
a + sum_btree_option lt + sum_btree_option rt" | |
53330
77da8d3c46e0
fixed docs w.r.t. availability of "primrec_new" and friends
blanchet
parents:
53262
diff
changeset
|
1183 |
"sum_btree_option None = 0" | |
53025 | 1184 |
"sum_btree_option (Some t) = sum_btree t" |
52843 | 1185 |
|
1186 |
text {* |
|
53621 | 1187 |
% * can pretend a nested type is mutually recursive (if purely inductive) |
1188 |
% * avoids the higher-order map |
|
1189 |
% * e.g. |
|
1190 |
||
53617 | 1191 |
% * this can always be avoided; |
1192 |
% * e.g. in our previous example, we first mapped the recursive |
|
1193 |
% calls, then we used a generic at function to retrieve the result |
|
1194 |
% |
|
1195 |
% * there's no hard-and-fast rule of when to use one or the other, |
|
1196 |
% just like there's no rule when to use fold and when to use |
|
1197 |
% primrec_new |
|
1198 |
% |
|
1199 |
% * higher-order approach, considering nesting as nesting, is more |
|
1200 |
% compositional -- e.g. we saw how we could reuse an existing polymorphic |
|
53647 | 1201 |
% at or the_default, whereas @{const ats\<^sub>f\<^sub>f} is much more specific |
53617 | 1202 |
% |
1203 |
% * but: |
|
1204 |
% * is perhaps less intuitive, because it requires higher-order thinking |
|
1205 |
% * may seem inefficient, and indeed with the code generator the |
|
1206 |
% mutually recursive version might be nicer |
|
1207 |
% * is somewhat indirect -- must apply a map first, then compute a result |
|
1208 |
% (cannot mix) |
|
53647 | 1209 |
% * the auxiliary functions like @{const ats\<^sub>f\<^sub>f} are sometimes useful in own right |
53617 | 1210 |
% |
1211 |
% * impact on automation unclear |
|
1212 |
% |
|
52843 | 1213 |
*} |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1214 |
(*<*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1215 |
end |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1216 |
(*>*) |
52843 | 1217 |
|
52824 | 1218 |
|
53617 | 1219 |
subsection {* Command Syntax |
1220 |
\label{ssec:primrec-command-syntax} *} |
|
1221 |
||
1222 |
||
53621 | 1223 |
subsubsection {* \keyw{primrec\_new} |
1224 |
\label{sssec:primrec-new} *} |
|
52828 | 1225 |
|
1226 |
text {* |
|
53829 | 1227 |
\begin{matharray}{rcl} |
1228 |
@{command_def "primrec_new"} & : & @{text "local_theory \<rightarrow> local_theory"} |
|
1229 |
\end{matharray} |
|
52794 | 1230 |
|
52840 | 1231 |
@{rail " |
53829 | 1232 |
@@{command primrec_new} target? fixes \\ @'where' (@{syntax pr_equation} + '|') |
52840 | 1233 |
; |
53829 | 1234 |
@{syntax_def pr_equation}: thmdecl? prop |
52840 | 1235 |
"} |
52828 | 1236 |
*} |
1237 |
||
52840 | 1238 |
|
53619 | 1239 |
(* |
52840 | 1240 |
subsection {* Generated Theorems |
1241 |
\label{ssec:primrec-generated-theorems} *} |
|
52824 | 1242 |
|
52828 | 1243 |
text {* |
53617 | 1244 |
% * synthesized nonrecursive definition |
1245 |
% * user specification is rederived from it, exactly as entered |
|
1246 |
% |
|
1247 |
% * induct |
|
1248 |
% * mutualized |
|
1249 |
% * without some needless induction hypotheses if not used |
|
1250 |
% * fold, rec |
|
1251 |
% * mutualized |
|
52828 | 1252 |
*} |
53619 | 1253 |
*) |
1254 |
||
52824 | 1255 |
|
52840 | 1256 |
subsection {* Recursive Default Values for Selectors |
53623 | 1257 |
\label{ssec:primrec-recursive-default-values-for-selectors} *} |
52827 | 1258 |
|
1259 |
text {* |
|
1260 |
A datatype selector @{text un_D} can have a default value for each constructor |
|
1261 |
on which it is not otherwise specified. Occasionally, it is useful to have the |
|
1262 |
default value be defined recursively. This produces a chicken-and-egg situation |
|
53621 | 1263 |
that may seem unsolvable, because the datatype is not introduced yet at the |
52827 | 1264 |
moment when the selectors are introduced. Of course, we can always define the |
1265 |
selectors manually afterward, but we then have to state and prove all the |
|
1266 |
characteristic theorems ourselves instead of letting the package do it. |
|
1267 |
||
1268 |
Fortunately, there is a fairly elegant workaround that relies on overloading and |
|
1269 |
that avoids the tedium of manual derivations: |
|
1270 |
||
1271 |
\begin{enumerate} |
|
1272 |
\setlength{\itemsep}{0pt} |
|
1273 |
||
1274 |
\item |
|
1275 |
Introduce a fully unspecified constant @{text "un_D\<^sub>0 \<Colon> 'a"} using |
|
1276 |
@{keyword consts}. |
|
1277 |
||
1278 |
\item |
|
53535 | 1279 |
Define the datatype, specifying @{text "un_D\<^sub>0"} as the selector's default |
1280 |
value. |
|
52827 | 1281 |
|
1282 |
\item |
|
53535 | 1283 |
Define the behavior of @{text "un_D\<^sub>0"} on values of the newly introduced |
1284 |
datatype using the \keyw{overloading} command. |
|
52827 | 1285 |
|
1286 |
\item |
|
1287 |
Derive the desired equation on @{text un_D} from the characteristic equations |
|
1288 |
for @{text "un_D\<^sub>0"}. |
|
1289 |
\end{enumerate} |
|
1290 |
||
53619 | 1291 |
\noindent |
52827 | 1292 |
The following example illustrates this procedure: |
1293 |
*} |
|
1294 |
||
1295 |
consts termi\<^sub>0 :: 'a |
|
1296 |
||
53619 | 1297 |
text {* \blankline *} |
1298 |
||
53491 | 1299 |
datatype_new ('a, 'b) tlist = |
52827 | 1300 |
TNil (termi: 'b) (defaults ttl: TNil) |
53491 | 1301 |
| TCons (thd: 'a) (ttl : "('a, 'b) tlist") (defaults termi: "\<lambda>_ xs. termi\<^sub>0 xs") |
52827 | 1302 |
|
53619 | 1303 |
text {* \blankline *} |
1304 |
||
52827 | 1305 |
overloading |
53491 | 1306 |
termi\<^sub>0 \<equiv> "termi\<^sub>0 \<Colon> ('a, 'b) tlist \<Rightarrow> 'b" |
52827 | 1307 |
begin |
53491 | 1308 |
primrec_new termi\<^sub>0 :: "('a, 'b) tlist \<Rightarrow> 'b" where |
53621 | 1309 |
"termi\<^sub>0 (TNil y) = y" | |
1310 |
"termi\<^sub>0 (TCons x xs) = termi\<^sub>0 xs" |
|
52827 | 1311 |
end |
1312 |
||
53619 | 1313 |
text {* \blankline *} |
1314 |
||
52827 | 1315 |
lemma terminal_TCons[simp]: "termi (TCons x xs) = termi xs" |
1316 |
by (cases xs) auto |
|
1317 |
||
1318 |
||
52828 | 1319 |
subsection {* Compatibility Issues |
53617 | 1320 |
\label{ssec:primrec-compatibility-issues} *} |
52828 | 1321 |
|
1322 |
text {* |
|
53997 | 1323 |
The command @{command primrec_new} has been designed to be highly compatible |
1324 |
with the old \keyw{primrec}, to ease migration. There is nonetheless at least |
|
1325 |
one incompatibility that may arise when porting to the new package: |
|
1326 |
||
1327 |
\begin{itemize} |
|
1328 |
\setlength{\itemsep}{0pt} |
|
1329 |
||
1330 |
\item \emph{Theorems sometimes have different names.} |
|
1331 |
For $m > 1$ mutually recursive functions, |
|
1332 |
@{text "f\<^sub>1_\<dots>_f\<^sub>m.simps(k\<^sub>i,\<dots>,k\<^sub>i+n\<^sub>i-1)"} have |
|
1333 |
been renamed @{text "f\<^sub>i.simps(1,\<dots>,n\<^sub>i-1)"}. |
|
1334 |
\end{itemize} |
|
52828 | 1335 |
*} |
52794 | 1336 |
|
1337 |
||
52827 | 1338 |
section {* Defining Codatatypes |
52805 | 1339 |
\label{sec:defining-codatatypes} *} |
1340 |
||
1341 |
text {* |
|
53829 | 1342 |
Codatatypes can be specified using the @{command codatatype} command. The |
53623 | 1343 |
command is first illustrated through concrete examples featuring different |
1344 |
flavors of corecursion. More examples can be found in the directory |
|
53997 | 1345 |
\verb|~~/src/HOL/|\allowbreak\verb|BNF/Examples|. The |
1346 |
\emph{Archive of Formal Proofs} also includes some useful codatatypes, notably |
|
1347 |
for lazy lists \cite{lochbihler-2010}. |
|
52805 | 1348 |
*} |
52792 | 1349 |
|
52824 | 1350 |
|
53617 | 1351 |
subsection {* Introductory Examples |
1352 |
\label{ssec:codatatype-introductory-examples} *} |
|
52794 | 1353 |
|
53623 | 1354 |
|
1355 |
subsubsection {* Simple Corecursion |
|
1356 |
\label{sssec:codatatype-simple-corecursion} *} |
|
1357 |
||
52805 | 1358 |
text {* |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1359 |
Noncorecursive codatatypes coincide with the corresponding datatypes, so they |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1360 |
are useless in practice. \emph{Corecursive codatatypes} have the same syntax |
53623 | 1361 |
as recursive datatypes, except for the command name. For example, here is the |
1362 |
definition of lazy lists: |
|
1363 |
*} |
|
1364 |
||
1365 |
codatatype (lset: 'a) llist (map: lmap rel: llist_all2) = |
|
1366 |
lnull: LNil (defaults ltl: LNil) |
|
1367 |
| LCons (lhd: 'a) (ltl: "'a llist") |
|
1368 |
||
1369 |
text {* |
|
1370 |
\noindent |
|
1371 |
Lazy lists can be infinite, such as @{text "LCons 0 (LCons 0 (\<dots>))"} and |
|
53647 | 1372 |
@{text "LCons 0 (LCons 1 (LCons 2 (\<dots>)))"}. Here is a related type, that of |
1373 |
infinite streams: |
|
1374 |
*} |
|
1375 |
||
1376 |
codatatype (sset: 'a) stream (map: smap rel: stream_all2) = |
|
1377 |
SCons (shd: 'a) (stl: "'a stream") |
|
1378 |
||
1379 |
text {* |
|
1380 |
\noindent |
|
1381 |
Another interesting type that can |
|
53623 | 1382 |
be defined as a codatatype is that of the extended natural numbers: |
1383 |
*} |
|
1384 |
||
53644 | 1385 |
codatatype enat = EZero | ESuc enat |
53623 | 1386 |
|
1387 |
text {* |
|
1388 |
\noindent |
|
1389 |
This type has exactly one infinite element, @{text "ESuc (ESuc (ESuc (\<dots>)))"}, |
|
1390 |
that represents $\infty$. In addition, it has finite values of the form |
|
1391 |
@{text "ESuc (\<dots> (ESuc EZero)\<dots>)"}. |
|
53675 | 1392 |
|
1393 |
Here is an example with many constructors: |
|
52805 | 1394 |
*} |
53623 | 1395 |
|
53675 | 1396 |
codatatype 'a process = |
1397 |
Fail |
|
1398 |
| Skip (cont: "'a process") |
|
1399 |
| Action (prefix: 'a) (cont: "'a process") |
|
1400 |
| Choice (left: "'a process") (right: "'a process") |
|
1401 |
||
53750 | 1402 |
text {* |
53829 | 1403 |
\noindent |
53750 | 1404 |
Notice that the @{const cont} selector is associated with both @{const Skip} |
1405 |
and @{const Choice}. |
|
1406 |
*} |
|
1407 |
||
53623 | 1408 |
|
1409 |
subsubsection {* Mutual Corecursion |
|
1410 |
\label{sssec:codatatype-mutual-corecursion} *} |
|
1411 |
||
1412 |
text {* |
|
1413 |
\noindent |
|
1414 |
The example below introduces a pair of \emph{mutually corecursive} types: |
|
1415 |
*} |
|
1416 |
||
1417 |
codatatype even_enat = Even_EZero | Even_ESuc odd_enat |
|
1418 |
and odd_enat = Odd_ESuc even_enat |
|
1419 |
||
1420 |
||
1421 |
subsubsection {* Nested Corecursion |
|
1422 |
\label{sssec:codatatype-nested-corecursion} *} |
|
1423 |
||
1424 |
text {* |
|
1425 |
\noindent |
|
53675 | 1426 |
The next examples feature \emph{nested corecursion}: |
53623 | 1427 |
*} |
1428 |
||
53644 | 1429 |
codatatype 'a tree\<^sub>i\<^sub>i = Node\<^sub>i\<^sub>i (lbl\<^sub>i\<^sub>i: 'a) (sub\<^sub>i\<^sub>i: "'a tree\<^sub>i\<^sub>i llist") |
53675 | 1430 |
|
53752 | 1431 |
text {* \blankline *} |
1432 |
||
53644 | 1433 |
codatatype 'a tree\<^sub>i\<^sub>s = Node\<^sub>i\<^sub>s (lbl\<^sub>i\<^sub>s: 'a) (sub\<^sub>i\<^sub>s: "'a tree\<^sub>i\<^sub>s fset") |
52805 | 1434 |
|
53752 | 1435 |
text {* \blankline *} |
1436 |
||
53675 | 1437 |
codatatype 'a state_machine = |
53751 | 1438 |
State_Machine (accept: bool) (trans: "'a \<Rightarrow> 'a state_machine") |
53675 | 1439 |
|
52824 | 1440 |
|
53617 | 1441 |
subsection {* Command Syntax |
1442 |
\label{ssec:codatatype-command-syntax} *} |
|
52805 | 1443 |
|
53619 | 1444 |
|
53621 | 1445 |
subsubsection {* \keyw{codatatype} |
1446 |
\label{sssec:codatatype} *} |
|
53619 | 1447 |
|
52824 | 1448 |
text {* |
53829 | 1449 |
\begin{matharray}{rcl} |
1450 |
@{command_def "codatatype"} & : & @{text "local_theory \<rightarrow> local_theory"} |
|
1451 |
\end{matharray} |
|
1452 |
||
1453 |
@{rail " |
|
1454 |
@@{command codatatype} target? \\ |
|
1455 |
(@{syntax dt_name} '=' (@{syntax ctor} + '|') + @'and') |
|
1456 |
"} |
|
1457 |
||
1458 |
\noindent |
|
52827 | 1459 |
Definitions of codatatypes have almost exactly the same syntax as for datatypes |
53829 | 1460 |
(Section~\ref{ssec:datatype-command-syntax}). The @{text "no_discs_sels"} option |
1461 |
is not available, because destructors are a crucial notion for codatatypes. |
|
53623 | 1462 |
*} |
1463 |
||
1464 |
||
1465 |
subsection {* Generated Constants |
|
1466 |
\label{ssec:codatatype-generated-constants} *} |
|
1467 |
||
1468 |
text {* |
|
1469 |
Given a codatatype @{text "('a\<^sub>1, \<dots>, 'a\<^sub>m) t"} |
|
1470 |
with $m > 0$ live type variables and $n$ constructors @{text "t.C\<^sub>1"}, |
|
1471 |
\ldots, @{text "t.C\<^sub>n"}, the same auxiliary constants are generated as for |
|
1472 |
datatypes (Section~\ref{ssec:datatype-generated-constants}), except that the |
|
1473 |
iterator and the recursor are replaced by dual concepts: |
|
1474 |
||
1475 |
\begin{itemize} |
|
1476 |
\setlength{\itemsep}{0pt} |
|
1477 |
||
1478 |
\item \relax{Coiterator}: @{text t_unfold} |
|
1479 |
||
1480 |
\item \relax{Corecursor}: @{text t_corec} |
|
1481 |
||
1482 |
\end{itemize} |
|
1483 |
*} |
|
1484 |
||
1485 |
||
1486 |
subsection {* Generated Theorems |
|
1487 |
\label{ssec:codatatype-generated-theorems} *} |
|
1488 |
||
1489 |
text {* |
|
53829 | 1490 |
The characteristic theorems generated by @{command codatatype} are grouped in |
53623 | 1491 |
three broad categories: |
1492 |
||
1493 |
\begin{itemize} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1494 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1495 |
|
53623 | 1496 |
\item The \emph{free constructor theorems} are properties about the constructors |
1497 |
and destructors that can be derived for any freely generated type. |
|
1498 |
||
1499 |
\item The \emph{functorial theorems} are properties of datatypes related to |
|
1500 |
their BNF nature. |
|
1501 |
||
1502 |
\item The \emph{coinductive theorems} are properties of datatypes related to |
|
1503 |
their coinductive nature. |
|
1504 |
\end{itemize} |
|
1505 |
||
1506 |
\noindent |
|
1507 |
The first two categories are exactly as for datatypes and are described in |
|
53642 | 1508 |
Sections |
1509 |
\ref{sssec:free-constructor-theorems}~and~\ref{sssec:functorial-theorems}. |
|
52824 | 1510 |
*} |
1511 |
||
53617 | 1512 |
|
53623 | 1513 |
subsubsection {* Coinductive Theorems |
1514 |
\label{sssec:coinductive-theorems} *} |
|
1515 |
||
1516 |
text {* |
|
1517 |
The coinductive theorems are as follows: |
|
1518 |
||
1519 |
\begin{indentblock} |
|
1520 |
\begin{description} |
|
1521 |
||
53643 | 1522 |
\item[\begin{tabular}{@ {}l@ {}} |
1523 |
@{text "t."}\hthm{coinduct} @{text "[coinduct t, consumes m, case_names t\<^sub>1 \<dots> t\<^sub>m,"} \\ |
|
1524 |
\phantom{@{text "t."}\hthm{coinduct} @{text "["}}@{text "case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"}\rm: |
|
1525 |
\end{tabular}] ~ \\ |
|
53623 | 1526 |
@{thm llist.coinduct[no_vars]} |
53617 | 1527 |
|
53643 | 1528 |
\item[\begin{tabular}{@ {}l@ {}} |
1529 |
@{text "t."}\hthm{strong\_coinduct} @{text "[consumes m, case_names t\<^sub>1 \<dots> t\<^sub>m,"} \\ |
|
1530 |
\phantom{@{text "t."}\hthm{strong\_coinduct} @{text "["}}@{text "case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"}\rm: |
|
1531 |
\end{tabular}] ~ \\ |
|
1532 |
@{thm llist.strong_coinduct[no_vars]} |
|
53617 | 1533 |
|
53643 | 1534 |
\item[\begin{tabular}{@ {}l@ {}} |
1535 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{coinduct} @{text "[case_names t\<^sub>1 \<dots> t\<^sub>m, case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"} \\ |
|
1536 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{strong\_coinduct} @{text "[case_names t\<^sub>1 \<dots> t\<^sub>m,"} \\ |
|
1537 |
\phantom{@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{strong\_coinduct} @{text "["}}@{text "case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"}\rm: |
|
1538 |
\end{tabular}] ~ \\ |
|
1539 |
Given $m > 1$ mutually corecursive codatatypes, these coinduction rules can be |
|
1540 |
used to prove $m$ properties simultaneously. |
|
1541 |
||
1542 |
\item[@{text "t."}\hthm{unfold} \rm(@{text "[simp]"})\rm:] ~ \\ |
|
53623 | 1543 |
@{thm llist.unfold(1)[no_vars]} \\ |
1544 |
@{thm llist.unfold(2)[no_vars]} |
|
1545 |
||
53643 | 1546 |
\item[@{text "t."}\hthm{corec} (@{text "[simp]"})\rm:] ~ \\ |
53623 | 1547 |
@{thm llist.corec(1)[no_vars]} \\ |
1548 |
@{thm llist.corec(2)[no_vars]} |
|
1549 |
||
53703 | 1550 |
\item[@{text "t."}\hthm{disc\_unfold}\rm:] ~ \\ |
53643 | 1551 |
@{thm llist.disc_unfold(1)[no_vars]} \\ |
1552 |
@{thm llist.disc_unfold(2)[no_vars]} |
|
1553 |
||
53703 | 1554 |
\item[@{text "t."}\hthm{disc\_corec}\rm:] ~ \\ |
53643 | 1555 |
@{thm llist.disc_corec(1)[no_vars]} \\ |
1556 |
@{thm llist.disc_corec(2)[no_vars]} |
|
1557 |
||
1558 |
\item[@{text "t."}\hthm{disc\_unfold\_iff} @{text "[simp]"}\rm:] ~ \\ |
|
1559 |
@{thm llist.disc_unfold_iff(1)[no_vars]} \\ |
|
1560 |
@{thm llist.disc_unfold_iff(2)[no_vars]} |
|
1561 |
||
1562 |
\item[@{text "t."}\hthm{disc\_corec\_iff} @{text "[simp]"}\rm:] ~ \\ |
|
1563 |
@{thm llist.disc_corec_iff(1)[no_vars]} \\ |
|
1564 |
@{thm llist.disc_corec_iff(2)[no_vars]} |
|
1565 |
||
1566 |
\item[@{text "t."}\hthm{sel\_unfold} @{text "[simp]"}\rm:] ~ \\ |
|
1567 |
@{thm llist.sel_unfold(1)[no_vars]} \\ |
|
1568 |
@{thm llist.sel_unfold(2)[no_vars]} |
|
1569 |
||
1570 |
\item[@{text "t."}\hthm{sel\_corec} @{text "[simp]"}\rm:] ~ \\ |
|
1571 |
@{thm llist.sel_corec(1)[no_vars]} \\ |
|
1572 |
@{thm llist.sel_corec(2)[no_vars]} |
|
1573 |
||
53623 | 1574 |
\end{description} |
1575 |
\end{indentblock} |
|
1576 |
||
1577 |
\noindent |
|
53829 | 1578 |
For convenience, @{command codatatype} also provides the following collection: |
53623 | 1579 |
|
1580 |
\begin{indentblock} |
|
1581 |
\begin{description} |
|
1582 |
||
53643 | 1583 |
\item[@{text "t."}\hthm{simps} = @{text t.inject} @{text t.distinct} @{text t.case} @{text t.corec}$^*$ @{text t.disc_corec}] ~ \\ |
1584 |
@{text t.disc_corec_iff} @{text t.sel_corec} @{text t.unfold}$^*$ @{text t.disc_unfold} @{text t.disc_unfold_iff} ~ \\ |
|
53694 | 1585 |
@{text t.sel_unfold} @{text t.map} @{text t.rel_inject} @{text t.rel_distinct} @{text t.set} |
53623 | 1586 |
|
1587 |
\end{description} |
|
1588 |
\end{indentblock} |
|
1589 |
*} |
|
52805 | 1590 |
|
1591 |
||
52827 | 1592 |
section {* Defining Corecursive Functions |
52805 | 1593 |
\label{sec:defining-corecursive-functions} *} |
1594 |
||
1595 |
text {* |
|
53753
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1596 |
Corecursive functions can be specified using @{command primcorec} and |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1597 |
@{command primcorecursive}, which support primitive corecursion, or using the |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1598 |
more general \keyw{partial\_function} command. Here, the focus is on |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1599 |
the former two. More examples can be found in the directory |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1600 |
\verb|~~/src/HOL/BNF/Examples|. |
53644 | 1601 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1602 |
Whereas recursive functions consume datatypes one constructor at a time, |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1603 |
corecursive functions construct codatatypes one constructor at a time. |
53752 | 1604 |
Partly reflecting a lack of agreement among proponents of coalgebraic methods, |
1605 |
Isabelle supports three competing syntaxes for specifying a function $f$: |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1606 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1607 |
\begin{itemize} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1608 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1609 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1610 |
\abovedisplayskip=.5\abovedisplayskip |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1611 |
\belowdisplayskip=.5\belowdisplayskip |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1612 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1613 |
\item The \emph{destructor view} specifies $f$ by implications of the form |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1614 |
\[@{text "\<dots> \<Longrightarrow> is_C\<^sub>j (f x\<^sub>1 \<dots> x\<^sub>n)"}\] and |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1615 |
equations of the form |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1616 |
\[@{text "un_C\<^sub>ji (f x\<^sub>1 \<dots> x\<^sub>n) = \<dots>"}\] |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1617 |
This style is popular in the coalgebraic literature. |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1618 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1619 |
\item The \emph{constructor view} specifies $f$ by equations of the form |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1620 |
\[@{text "\<dots> \<Longrightarrow> f x\<^sub>1 \<dots> x\<^sub>n = C \<dots>"}\] |
53752 | 1621 |
This style is often more concise than the previous one. |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1622 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1623 |
\item The \emph{code view} specifies $f$ by a single equation of the form |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1624 |
\[@{text "f x\<^sub>1 \<dots> x\<^sub>n = \<dots>"}\] |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1625 |
with restrictions on the format of the right-hand side. Lazy functional |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1626 |
programming languages such as Haskell support a generalized version of this |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1627 |
style. |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1628 |
\end{itemize} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1629 |
|
53753
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1630 |
All three styles are available as input syntax. Whichever syntax is chosen, |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1631 |
characteristic theorems for all three styles are generated. |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1632 |
|
53644 | 1633 |
\begin{framed} |
1634 |
\noindent |
|
53753
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1635 |
\textbf{Warning:}\enskip The @{command primcorec} and @{command primcorecursive} |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1636 |
commands are under development. Some of the functionality described here is |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1637 |
vaporware. An alternative is to define corecursive functions directly using the |
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
1638 |
generated @{text t_unfold} or @{text t_corec} combinators. |
53644 | 1639 |
\end{framed} |
52828 | 1640 |
|
1641 |
%%% TODO: partial_function? E.g. for defining tail recursive function on lazy |
|
1642 |
%%% lists (cf. terminal0 in TLList.thy) |
|
52805 | 1643 |
*} |
1644 |
||
52824 | 1645 |
|
53617 | 1646 |
subsection {* Introductory Examples |
1647 |
\label{ssec:primcorec-introductory-examples} *} |
|
52805 | 1648 |
|
53646 | 1649 |
text {* |
1650 |
Primitive corecursion is illustrated through concrete examples based on the |
|
1651 |
codatatypes defined in Section~\ref{ssec:codatatype-introductory-examples}. More |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1652 |
examples can be found in the directory \verb|~~/src/HOL/BNF/Examples|. The code |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1653 |
view is favored in the examples below. Sections |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1654 |
\ref{ssec:primrec-constructor-view} and \ref{ssec:primrec-destructor-view} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1655 |
present the same examples expressed using the constructor and destructor views. |
53646 | 1656 |
*} |
1657 |
||
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1658 |
(*<*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1659 |
locale code_view |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1660 |
begin |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1661 |
(*>*) |
53644 | 1662 |
|
1663 |
subsubsection {* Simple Corecursion |
|
1664 |
\label{sssec:primcorec-simple-corecursion} *} |
|
1665 |
||
53646 | 1666 |
text {* |
53752 | 1667 |
Following the code view, corecursive calls are allowed on the right-hand side as |
1668 |
long as they occur under a constructor, which itself appears either directly to |
|
1669 |
the right of the equal sign or in a conditional expression: |
|
53646 | 1670 |
*} |
1671 |
||
53826 | 1672 |
primcorec literate :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a llist" where |
53647 | 1673 |
"literate f x = LCons x (literate f (f x))" |
1674 |
||
53677 | 1675 |
text {* \blankline *} |
1676 |
||
53826 | 1677 |
primcorec siterate :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a stream" where |
53647 | 1678 |
"siterate f x = SCons x (siterate f (f x))" |
53644 | 1679 |
|
53646 | 1680 |
text {* |
1681 |
\noindent |
|
1682 |
The constructor ensures that progress is made---i.e., the function is |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1683 |
\emph{productive}. The above functions compute the infinite lazy list or stream |
53646 | 1684 |
@{text "[x, f x, f (f x), \<dots>]"}. Productivity guarantees that prefixes |
1685 |
@{text "[x, f x, f (f x), \<dots>, (f ^^ k) x]"} of arbitrary finite length |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1686 |
@{text k} can be computed by unfolding the code equation a finite number of |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1687 |
times. |
53646 | 1688 |
|
53752 | 1689 |
Corecursive functions construct codatatype values, but nothing prevents them |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1690 |
from also consuming such values. The following function drops every second |
53675 | 1691 |
element in a stream: |
1692 |
*} |
|
1693 |
||
53826 | 1694 |
primcorec every_snd :: "'a stream \<Rightarrow> 'a stream" where |
53675 | 1695 |
"every_snd s = SCons (shd s) (stl (stl s))" |
1696 |
||
1697 |
text {* |
|
53752 | 1698 |
\noindent |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1699 |
Constructs such as @{text "let"}---@{text "in"}, @{text |
53646 | 1700 |
"if"}---@{text "then"}---@{text "else"}, and @{text "case"}---@{text "of"} may |
1701 |
appear around constructors that guard corecursive calls: |
|
1702 |
*} |
|
1703 |
||
53826 | 1704 |
primcorec_notyet lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
53644 | 1705 |
"lappend xs ys = |
1706 |
(case xs of |
|
1707 |
LNil \<Rightarrow> ys |
|
1708 |
| LCons x xs' \<Rightarrow> LCons x (lappend xs' ys))" |
|
1709 |
||
53646 | 1710 |
text {* |
53752 | 1711 |
\noindent |
53646 | 1712 |
Corecursion is useful to specify not only functions but also infinite objects: |
1713 |
*} |
|
1714 |
||
53826 | 1715 |
primcorec infty :: enat where |
53644 | 1716 |
"infty = ESuc infty" |
1717 |
||
53646 | 1718 |
text {* |
53752 | 1719 |
\noindent |
1720 |
The example below constructs a pseudorandom process value. It takes a stream of |
|
53675 | 1721 |
actions (@{text s}), a pseudorandom function generator (@{text f}), and a |
1722 |
pseudorandom seed (@{text n}): |
|
1723 |
*} |
|
1724 |
||
53826 | 1725 |
primcorec_notyet |
53752 | 1726 |
random_process :: "'a stream \<Rightarrow> (int \<Rightarrow> int) \<Rightarrow> int \<Rightarrow> 'a process" |
1727 |
where |
|
53675 | 1728 |
"random_process s f n = |
1729 |
(if n mod 4 = 0 then |
|
1730 |
Fail |
|
1731 |
else if n mod 4 = 1 then |
|
1732 |
Skip (random_process s f (f n)) |
|
1733 |
else if n mod 4 = 2 then |
|
1734 |
Action (shd s) (random_process (stl s) f (f n)) |
|
1735 |
else |
|
1736 |
Choice (random_process (every_snd s) (f \<circ> f) (f n)) |
|
1737 |
(random_process (every_snd (stl s)) (f \<circ> f) (f (f n))))" |
|
1738 |
||
1739 |
text {* |
|
1740 |
\noindent |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1741 |
The main disadvantage of the code view is that the conditions are tested |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1742 |
sequentially. This is visible in the generated theorems. The constructor and |
53752 | 1743 |
destructor views offer nonsequential alternatives. |
53675 | 1744 |
*} |
1745 |
||
53644 | 1746 |
|
1747 |
subsubsection {* Mutual Corecursion |
|
1748 |
\label{sssec:primcorec-mutual-corecursion} *} |
|
1749 |
||
53647 | 1750 |
text {* |
1751 |
The syntax for mutually corecursive functions over mutually corecursive |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1752 |
datatypes is unsurprising: |
53647 | 1753 |
*} |
1754 |
||
53826 | 1755 |
primcorec |
53644 | 1756 |
even_infty :: even_enat and |
1757 |
odd_infty :: odd_enat |
|
1758 |
where |
|
1759 |
"even_infty = Even_ESuc odd_infty" | |
|
1760 |
"odd_infty = Odd_ESuc even_infty" |
|
1761 |
||
1762 |
||
1763 |
subsubsection {* Nested Corecursion |
|
1764 |
\label{sssec:primcorec-nested-corecursion} *} |
|
1765 |
||
53647 | 1766 |
text {* |
1767 |
The next pair of examples generalize the @{const literate} and @{const siterate} |
|
1768 |
functions (Section~\ref{sssec:primcorec-nested-corecursion}) to possibly |
|
1769 |
infinite trees in which subnodes are organized either as a lazy list (@{text |
|
1770 |
tree\<^sub>i\<^sub>i}) or as a finite set (@{text tree\<^sub>i\<^sub>s}): |
|
1771 |
*} |
|
1772 |
||
53826 | 1773 |
primcorec iterate\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>i" where |
53644 | 1774 |
"iterate\<^sub>i\<^sub>i f x = Node\<^sub>i\<^sub>i x (lmap (iterate\<^sub>i\<^sub>i f) (f x))" |
1775 |
||
53677 | 1776 |
text {* \blankline *} |
1777 |
||
53826 | 1778 |
primcorec iterate\<^sub>i\<^sub>s :: "('a \<Rightarrow> 'a fset) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>s" where |
54014 | 1779 |
"iterate\<^sub>i\<^sub>s f x = Node\<^sub>i\<^sub>s x (fimage (iterate\<^sub>i\<^sub>s f) (f x))" |
53644 | 1780 |
|
52805 | 1781 |
text {* |
53752 | 1782 |
\noindent |
53675 | 1783 |
Deterministic finite automata (DFAs) are usually defined as 5-tuples |
1784 |
@{text "(Q, \<Sigma>, \<delta>, q\<^sub>0, F)"}, where @{text Q} is a finite set of states, |
|
1785 |
@{text \<Sigma>} is a finite alphabet, @{text \<delta>} is a transition function, @{text q\<^sub>0} |
|
1786 |
is an initial state, and @{text F} is a set of final states. The following |
|
1787 |
function translates a DFA into a @{type state_machine}: |
|
1788 |
*} |
|
1789 |
||
53826 | 1790 |
primcorec (*<*)(in early) (*>*) |
53752 | 1791 |
sm_of_dfa :: "('q \<Rightarrow> 'a \<Rightarrow> 'q) \<Rightarrow> 'q set \<Rightarrow> 'q \<Rightarrow> 'a state_machine" |
1792 |
where |
|
1793 |
"sm_of_dfa \<delta> F q = State_Machine (q \<in> F) (sm_of_dfa \<delta> F o \<delta> q)" |
|
53675 | 1794 |
|
53751 | 1795 |
text {* |
1796 |
\noindent |
|
1797 |
The map function for the function type (@{text \<Rightarrow>}) is composition |
|
53752 | 1798 |
(@{text "op \<circ>"}). For convenience, corecursion through functions can be |
1799 |
expressed using @{text \<lambda>}-expressions and function application rather |
|
1800 |
than composition. For example: |
|
53751 | 1801 |
*} |
1802 |
||
53826 | 1803 |
primcorec |
53752 | 1804 |
sm_of_dfa :: "('q \<Rightarrow> 'a \<Rightarrow> 'q) \<Rightarrow> 'q set \<Rightarrow> 'q \<Rightarrow> 'a state_machine" |
1805 |
where |
|
1806 |
"sm_of_dfa \<delta> F q = State_Machine (q \<in> F) (sm_of_dfa \<delta> F o \<delta> q)" |
|
1807 |
||
1808 |
text {* \blankline *} |
|
1809 |
||
53826 | 1810 |
primcorec empty_sm :: "'a state_machine" where |
53752 | 1811 |
"empty_sm = State_Machine False (\<lambda>_. empty_sm)" |
53751 | 1812 |
|
53752 | 1813 |
text {* \blankline *} |
1814 |
||
53826 | 1815 |
primcorec not_sm :: "'a state_machine \<Rightarrow> 'a state_machine" where |
53752 | 1816 |
"not_sm M = State_Machine (\<not> accept M) (\<lambda>a. not_sm (trans M a))" |
53751 | 1817 |
|
53752 | 1818 |
text {* \blankline *} |
1819 |
||
53826 | 1820 |
primcorec |
53752 | 1821 |
or_sm :: "'a state_machine \<Rightarrow> 'a state_machine \<Rightarrow> 'a state_machine" |
1822 |
where |
|
1823 |
"or_sm M N = |
|
53751 | 1824 |
State_Machine (accept M \<or> accept N) |
53752 | 1825 |
(\<lambda>a. or_sm (trans M a) (trans N a))" |
53751 | 1826 |
|
53644 | 1827 |
|
1828 |
subsubsection {* Nested-as-Mutual Corecursion |
|
1829 |
\label{sssec:primcorec-nested-as-mutual-corecursion} *} |
|
1830 |
||
53647 | 1831 |
text {* |
1832 |
Just as it is possible to recurse over nested recursive datatypes as if they |
|
1833 |
were mutually recursive |
|
1834 |
(Section~\ref{sssec:primrec-nested-as-mutual-recursion}), it is possible to |
|
53752 | 1835 |
pretend that nested codatatypes are mutually corecursive. For example: |
53647 | 1836 |
*} |
1837 |
||
53826 | 1838 |
primcorec_notyet |
53644 | 1839 |
iterate\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>i" and |
1840 |
iterates\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a llist \<Rightarrow> 'a tree\<^sub>i\<^sub>i llist" |
|
1841 |
where |
|
1842 |
"iterate\<^sub>i\<^sub>i f x = Node\<^sub>i\<^sub>i x (iterates\<^sub>i\<^sub>i f (f x))" | |
|
1843 |
"iterates\<^sub>i\<^sub>i f xs = |
|
1844 |
(case xs of |
|
1845 |
LNil \<Rightarrow> LNil |
|
1846 |
| LCons x xs' \<Rightarrow> LCons (iterate\<^sub>i\<^sub>i f x) (iterates\<^sub>i\<^sub>i f xs'))" |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1847 |
(*<*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1848 |
end |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1849 |
(*>*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1850 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1851 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1852 |
subsubsection {* Constructor View |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1853 |
\label{ssec:primrec-constructor-view} *} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1854 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1855 |
(*<*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1856 |
locale ctr_view = code_view |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1857 |
begin |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1858 |
(*>*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1859 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1860 |
text {* |
53750 | 1861 |
The constructor view is similar to the code view, but there is one separate |
1862 |
conditional equation per constructor rather than a single unconditional |
|
1863 |
equation. Examples that rely on a single constructor, such as @{const literate} |
|
1864 |
and @{const siterate}, are identical in both styles. |
|
1865 |
||
1866 |
Here is an example where there is a difference: |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1867 |
*} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1868 |
|
53826 | 1869 |
primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1870 |
"lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lappend xs ys = LNil" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1871 |
"_ \<Longrightarrow> lappend xs ys = LCons (lhd (if lnull xs then ys else xs)) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1872 |
(if xs = LNil then ltl ys else lappend (ltl xs) ys)" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1873 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1874 |
text {* |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1875 |
\noindent |
53752 | 1876 |
With the constructor view, we must distinguish between the @{const LNil} and |
1877 |
the @{const LCons} case. The condition for @{const LCons} is |
|
1878 |
left implicit, as the negation of that for @{const LNil}. |
|
53750 | 1879 |
|
1880 |
For this example, the constructor view is slighlty more involved than the |
|
1881 |
code equation. Recall the code view version presented in |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1882 |
Section~\ref{sssec:primcorec-simple-corecursion}. |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1883 |
% TODO: \[{thm code_view.lappend.code}\] |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1884 |
The constructor view requires us to analyze the second argument (@{term ys}). |
53752 | 1885 |
The code equation generated from the constructor view also suffers from this. |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1886 |
% TODO: \[{thm lappend.code}\] |
53750 | 1887 |
|
53752 | 1888 |
In contrast, the next example is arguably more naturally expressed in the |
1889 |
constructor view: |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1890 |
*} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1891 |
|
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
1892 |
primcorec |
53752 | 1893 |
random_process :: "'a stream \<Rightarrow> (int \<Rightarrow> int) \<Rightarrow> int \<Rightarrow> 'a process" |
1894 |
where |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1895 |
"n mod 4 = 0 \<Longrightarrow> random_process s f n = Fail" | |
53752 | 1896 |
"n mod 4 = 1 \<Longrightarrow> |
1897 |
random_process s f n = Skip (random_process s f (f n))" | |
|
1898 |
"n mod 4 = 2 \<Longrightarrow> |
|
1899 |
random_process s f n = Action (shd s) (random_process (stl s) f (f n))" | |
|
1900 |
"n mod 4 = 3 \<Longrightarrow> |
|
1901 |
random_process s f n = Choice (random_process (every_snd s) f (f n)) |
|
53826 | 1902 |
(random_process (every_snd (stl s)) f (f n))" |
1903 |
(*<*) |
|
53644 | 1904 |
end |
1905 |
(*>*) |
|
52805 | 1906 |
|
53750 | 1907 |
text {* |
53752 | 1908 |
\noindent |
53750 | 1909 |
Since there is no sequentiality, we can apply the equation for @{const Choice} |
53752 | 1910 |
without having first to discharge @{term "n mod (4\<Colon>int) \<noteq> 0"}, |
1911 |
@{term "n mod (4\<Colon>int) \<noteq> 1"}, and |
|
1912 |
@{term "n mod (4\<Colon>int) \<noteq> 2"}. |
|
53750 | 1913 |
The price to pay for this elegance is that we must discharge exclusivity proof |
1914 |
obligations, one for each pair of conditions |
|
53752 | 1915 |
@{term "(n mod (4\<Colon>int) = i, n mod (4\<Colon>int) = j)"} |
1916 |
with @{term "i < j"}. If we prefer not to discharge any obligations, we can |
|
1917 |
enable the @{text "sequential"} option. This pushes the problem to the users of |
|
1918 |
the generated properties. |
|
53750 | 1919 |
%Here are more examples to conclude: |
1920 |
*} |
|
1921 |
||
52824 | 1922 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1923 |
subsubsection {* Destructor View |
53752 | 1924 |
\label{ssec:primrec-destructor-view} *} |
1925 |
||
1926 |
(*<*) |
|
1927 |
locale dest_view |
|
1928 |
begin |
|
1929 |
(*>*) |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1930 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1931 |
text {* |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1932 |
The destructor view is in many respects dual to the constructor view. Conditions |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1933 |
determine which constructor to choose, and these conditions are interpreted |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1934 |
sequentially or not depending on the @{text "sequential"} option. |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1935 |
Consider the following examples: |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1936 |
*} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1937 |
|
53826 | 1938 |
primcorec literate :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a llist" where |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1939 |
"\<not> lnull (literate _ x)" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1940 |
"lhd (literate _ x) = x" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1941 |
"ltl (literate f x) = literate f (f x)" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1942 |
|
53752 | 1943 |
text {* \blankline *} |
1944 |
||
53826 | 1945 |
primcorec siterate :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a stream" where |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1946 |
"shd (siterate _ x) = x" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1947 |
"stl (siterate f x) = siterate f (f x)" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1948 |
|
53752 | 1949 |
text {* \blankline *} |
1950 |
||
53826 | 1951 |
primcorec every_snd :: "'a stream \<Rightarrow> 'a stream" where |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1952 |
"shd (every_snd s) = shd s" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1953 |
"stl (every_snd s) = stl (stl s)" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1954 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1955 |
text {* |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1956 |
\noindent |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1957 |
The first formula in the @{const literate} specification indicates which |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1958 |
constructor to choose. For @{const siterate} and @{const every_snd}, no such |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1959 |
formula is necessary, since the type has only one constructor. The last two |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1960 |
formulas are equations specifying the value of the result for the relevant |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1961 |
selectors. Corecursive calls appear directly to the right of the equal sign. |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1962 |
Their arguments are unrestricted. |
53750 | 1963 |
|
1964 |
The next example shows how to specify functions that rely on more than one |
|
1965 |
constructor: |
|
1966 |
*} |
|
1967 |
||
53826 | 1968 |
primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
53750 | 1969 |
"lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lnull (lappend xs ys)" | |
1970 |
"lhd (lappend xs ys) = lhd (if lnull xs then ys else xs)" | |
|
1971 |
"ltl (lappend xs ys) = (if xs = LNil then ltl ys else lappend (ltl xs) ys)" |
|
1972 |
||
1973 |
text {* |
|
1974 |
\noindent |
|
1975 |
For a codatatype with $n$ constructors, it is sufficient to specify $n - 1$ |
|
1976 |
discriminator formulas. The command will then assume that the remaining |
|
1977 |
constructor should be taken otherwise. This can be made explicit by adding |
|
1978 |
*} |
|
1979 |
||
1980 |
(*<*) |
|
1981 |
end |
|
1982 |
||
53826 | 1983 |
primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
53750 | 1984 |
"lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lnull (lappend xs ys)" | |
1985 |
(*>*) |
|
53752 | 1986 |
"_ \<Longrightarrow> \<not> lnull (lappend xs ys)" |
1987 |
(*<*) | |
|
53750 | 1988 |
"lhd (lappend xs ys) = lhd (if lnull xs then ys else xs)" | |
1989 |
"ltl (lappend xs ys) = (if xs = LNil then ltl ys else lappend (ltl xs) ys)" |
|
1990 |
||
1991 |
context dest_view begin |
|
1992 |
(*>*) |
|
1993 |
||
1994 |
text {* |
|
1995 |
\noindent |
|
53752 | 1996 |
to the specification. The generated selector theorems are conditional. |
1997 |
||
1998 |
The next example illustrates how to cope with selectors defined for several |
|
53750 | 1999 |
constructors: |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2000 |
*} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2001 |
|
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
2002 |
primcorec |
53752 | 2003 |
random_process :: "'a stream \<Rightarrow> (int \<Rightarrow> int) \<Rightarrow> int \<Rightarrow> 'a process" |
2004 |
where |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2005 |
"n mod 4 = 0 \<Longrightarrow> is_Fail (random_process s f n)" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2006 |
"n mod 4 = 1 \<Longrightarrow> is_Skip (random_process s f n)" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2007 |
"n mod 4 = 2 \<Longrightarrow> is_Action (random_process s f n)" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2008 |
"n mod 4 = 3 \<Longrightarrow> is_Choice (random_process s f n)" | |
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
2009 |
"cont (random_process s f n) = random_process s f (f n)" of Skip | |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2010 |
"prefix (random_process s f n) = shd s" | |
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
2011 |
"cont (random_process s f n) = random_process (stl s) f (f n)" of Action | |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2012 |
"left (random_process s f n) = random_process (every_snd s) f (f n)" | |
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
2013 |
"right (random_process s f n) = random_process (every_snd (stl s)) f (f n)" |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2014 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2015 |
text {* |
53750 | 2016 |
\noindent |
2017 |
Using the @{text "of"} keyword, different equations are specified for @{const |
|
2018 |
cont} depending on which constructor is selected. |
|
2019 |
||
2020 |
Here are more examples to conclude: |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2021 |
*} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2022 |
|
53826 | 2023 |
primcorec |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2024 |
even_infty :: even_enat and |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2025 |
odd_infty :: odd_enat |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2026 |
where |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2027 |
"\<not> is_Even_EZero even_infty" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2028 |
"un_Even_ESuc even_infty = odd_infty" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2029 |
"un_Odd_ESuc odd_infty = even_infty" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2030 |
|
53752 | 2031 |
text {* \blankline *} |
2032 |
||
53826 | 2033 |
primcorec iterate\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>i" where |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2034 |
"lbl\<^sub>i\<^sub>i (iterate\<^sub>i\<^sub>i f x) = x" | |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2035 |
"sub\<^sub>i\<^sub>i (iterate\<^sub>i\<^sub>i f x) = lmap (iterate\<^sub>i\<^sub>i f) (f x)" |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2036 |
(*<*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2037 |
end |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2038 |
(*>*) |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2039 |
|
53750 | 2040 |
|
53617 | 2041 |
subsection {* Command Syntax |
2042 |
\label{ssec:primcorec-command-syntax} *} |
|
2043 |
||
2044 |
||
53826 | 2045 |
subsubsection {* \keyw{primcorec} and \keyw{primcorecursive} |
53753
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
2046 |
\label{sssec:primcorecursive-and-primcorec} *} |
52840 | 2047 |
|
2048 |
text {* |
|
53829 | 2049 |
\begin{matharray}{rcl} |
2050 |
@{command_def "primcorec"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
2051 |
@{command_def "primcorecursive"} & : & @{text "local_theory \<rightarrow> proof(prove)"} |
|
2052 |
\end{matharray} |
|
52840 | 2053 |
|
2054 |
@{rail " |
|
53829 | 2055 |
(@@{command primcorec} | @@{command primcorecursive}) target? \\ @{syntax pcr_option}? fixes @'where' |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2056 |
(@{syntax pcr_formula} + '|') |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2057 |
; |
53828 | 2058 |
@{syntax_def pcr_option}: '(' ('sequential' | 'exhaustive') ')' |
52840 | 2059 |
; |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2060 |
@{syntax_def pcr_formula}: thmdecl? prop (@'of' (term * ))? |
52840 | 2061 |
"} |
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2062 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2063 |
The optional target is optionally followed by a corecursion-specific option: |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2064 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2065 |
\begin{itemize} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2066 |
\setlength{\itemsep}{0pt} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2067 |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2068 |
\item |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2069 |
The @{text "sequential"} option indicates that the conditions in specifications |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2070 |
expressed using the constructor or destructor view are to be interpreted |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2071 |
sequentially. |
53826 | 2072 |
|
2073 |
\item |
|
2074 |
The @{text "exhaustive"} option indicates that the conditions in specifications |
|
2075 |
expressed using the constructor or destructor view cover all possible cases. |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2076 |
\end{itemize} |
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2077 |
|
53826 | 2078 |
\noindent |
2079 |
The @{command primcorec} command is an abbreviation for @{command primcorecursive} with |
|
2080 |
@{text "by auto?"} to discharge any emerging proof obligations. |
|
52840 | 2081 |
*} |
52794 | 2082 |
|
52824 | 2083 |
|
53619 | 2084 |
(* |
52840 | 2085 |
subsection {* Generated Theorems |
2086 |
\label{ssec:primcorec-generated-theorems} *} |
|
53619 | 2087 |
*) |
52794 | 2088 |
|
2089 |
||
53623 | 2090 |
(* |
2091 |
subsection {* Recursive Default Values for Selectors |
|
2092 |
\label{ssec:primcorec-recursive-default-values-for-selectors} *} |
|
2093 |
||
2094 |
text {* |
|
2095 |
partial_function to the rescue |
|
2096 |
*} |
|
2097 |
*) |
|
2098 |
||
2099 |
||
52827 | 2100 |
section {* Registering Bounded Natural Functors |
52805 | 2101 |
\label{sec:registering-bounded-natural-functors} *} |
52792 | 2102 |
|
52805 | 2103 |
text {* |
53647 | 2104 |
The (co)datatype package can be set up to allow nested recursion through |
2105 |
arbitrary type constructors, as long as they adhere to the BNF requirements and |
|
2106 |
are registered as BNFs. |
|
52805 | 2107 |
*} |
2108 |
||
52824 | 2109 |
|
53619 | 2110 |
(* |
53617 | 2111 |
subsection {* Introductory Example |
2112 |
\label{ssec:bnf-introductory-example} *} |
|
52805 | 2113 |
|
2114 |
text {* |
|
2115 |
More examples in \verb|~~/src/HOL/BNF/Basic_BNFs.thy| and |
|
2116 |
\verb|~~/src/HOL/BNF/More_BNFs.thy|. |
|
52806 | 2117 |
|
53617 | 2118 |
%Mention distinction between live and dead type arguments; |
2119 |
% * and existence of map, set for those |
|
2120 |
%mention =>. |
|
52805 | 2121 |
*} |
53619 | 2122 |
*) |
52794 | 2123 |
|
52824 | 2124 |
|
53617 | 2125 |
subsection {* Command Syntax |
2126 |
\label{ssec:bnf-command-syntax} *} |
|
2127 |
||
2128 |
||
53621 | 2129 |
subsubsection {* \keyw{bnf} |
2130 |
\label{sssec:bnf} *} |
|
52794 | 2131 |
|
53028 | 2132 |
text {* |
53829 | 2133 |
\begin{matharray}{rcl} |
2134 |
@{command_def "bnf"} & : & @{text "local_theory \<rightarrow> proof(prove)"} |
|
2135 |
\end{matharray} |
|
2136 |
||
53028 | 2137 |
@{rail " |
53829 | 2138 |
@@{command bnf} target? (name ':')? term \\ |
53534 | 2139 |
term_list term term_list term? |
53028 | 2140 |
; |
53534 | 2141 |
X_list: '[' (X + ',') ']' |
53028 | 2142 |
"} |
2143 |
*} |
|
52805 | 2144 |
|
53617 | 2145 |
|
53621 | 2146 |
subsubsection {* \keyw{print\_bnfs} |
2147 |
\label{sssec:print-bnfs} *} |
|
53617 | 2148 |
|
2149 |
text {* |
|
53829 | 2150 |
\begin{matharray}{rcl} |
2151 |
@{command_def "print_bnfs"} & : & @{text "local_theory \<rightarrow>"} |
|
2152 |
\end{matharray} |
|
2153 |
||
53647 | 2154 |
@{rail " |
53829 | 2155 |
@@{command print_bnfs} |
53647 | 2156 |
"} |
53617 | 2157 |
*} |
2158 |
||
2159 |
||
2160 |
section {* Deriving Destructors and Theorems for Free Constructors |
|
2161 |
\label{sec:deriving-destructors-and-theorems-for-free-constructors} *} |
|
52794 | 2162 |
|
52805 | 2163 |
text {* |
53623 | 2164 |
The derivation of convenience theorems for types equipped with free constructors, |
53829 | 2165 |
as performed internally by @{command datatype_new} and @{command codatatype}, |
53623 | 2166 |
is available as a stand-alone command called @{command wrap_free_constructors}. |
52794 | 2167 |
|
53617 | 2168 |
% * need for this is rare but may arise if you want e.g. to add destructors to |
2169 |
% a type not introduced by ... |
|
2170 |
% |
|
2171 |
% * also useful for compatibility with old package, e.g. add destructors to |
|
2172 |
% old \keyw{datatype} |
|
2173 |
% |
|
2174 |
% * @{command wrap_free_constructors} |
|
53623 | 2175 |
% * @{text "no_discs_sels"}, @{text "rep_compat"} |
53617 | 2176 |
% * hack to have both co and nonco view via locale (cf. ext nats) |
52805 | 2177 |
*} |
52792 | 2178 |
|
52824 | 2179 |
|
53619 | 2180 |
(* |
53617 | 2181 |
subsection {* Introductory Example |
2182 |
\label{ssec:ctors-introductory-example} *} |
|
53619 | 2183 |
*) |
52794 | 2184 |
|
52824 | 2185 |
|
53617 | 2186 |
subsection {* Command Syntax |
2187 |
\label{ssec:ctors-command-syntax} *} |
|
2188 |
||
2189 |
||
53621 | 2190 |
subsubsection {* \keyw{wrap\_free\_constructors} |
53675 | 2191 |
\label{sssec:wrap-free-constructors} *} |
52828 | 2192 |
|
53018 | 2193 |
text {* |
53829 | 2194 |
\begin{matharray}{rcl} |
2195 |
@{command_def "wrap_free_constructors"} & : & @{text "local_theory \<rightarrow> proof(prove)"} |
|
2196 |
\end{matharray} |
|
53018 | 2197 |
|
2198 |
@{rail " |
|
53829 | 2199 |
@@{command wrap_free_constructors} target? @{syntax dt_options} \\ |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2200 |
term_list name @{syntax wfc_discs_sels}? |
53018 | 2201 |
; |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2202 |
@{syntax_def wfc_discs_sels}: name_list (name_list_list name_term_list_list? )? |
53018 | 2203 |
; |
53534 | 2204 |
@{syntax_def name_term}: (name ':' term) |
53018 | 2205 |
"} |
2206 |
||
53617 | 2207 |
% options: no_discs_sels rep_compat |
53028 | 2208 |
|
53617 | 2209 |
% X_list is as for BNF |
53028 | 2210 |
|
53829 | 2211 |
\noindent |
53542 | 2212 |
Section~\ref{ssec:datatype-generated-theorems} lists the generated theorems. |
53018 | 2213 |
*} |
52828 | 2214 |
|
52794 | 2215 |
|
53617 | 2216 |
(* |
52827 | 2217 |
section {* Standard ML Interface |
52805 | 2218 |
\label{sec:standard-ml-interface} *} |
52792 | 2219 |
|
52805 | 2220 |
text {* |
53623 | 2221 |
The package's programmatic interface. |
52805 | 2222 |
*} |
53617 | 2223 |
*) |
52794 | 2224 |
|
2225 |
||
53617 | 2226 |
(* |
52827 | 2227 |
section {* Interoperability |
52805 | 2228 |
\label{sec:interoperability} *} |
52794 | 2229 |
|
52805 | 2230 |
text {* |
53623 | 2231 |
The package's interaction with other Isabelle packages and tools, such as the |
2232 |
code generator and the counterexample generators. |
|
52805 | 2233 |
*} |
52794 | 2234 |
|
52824 | 2235 |
|
52828 | 2236 |
subsection {* Transfer and Lifting |
2237 |
\label{ssec:transfer-and-lifting} *} |
|
52794 | 2238 |
|
52824 | 2239 |
|
52828 | 2240 |
subsection {* Code Generator |
2241 |
\label{ssec:code-generator} *} |
|
52794 | 2242 |
|
52824 | 2243 |
|
52828 | 2244 |
subsection {* Quickcheck |
2245 |
\label{ssec:quickcheck} *} |
|
52794 | 2246 |
|
52824 | 2247 |
|
52828 | 2248 |
subsection {* Nitpick |
2249 |
\label{ssec:nitpick} *} |
|
52794 | 2250 |
|
52824 | 2251 |
|
52828 | 2252 |
subsection {* Nominal Isabelle |
2253 |
\label{ssec:nominal-isabelle} *} |
|
53617 | 2254 |
*) |
52794 | 2255 |
|
52805 | 2256 |
|
53617 | 2257 |
(* |
52827 | 2258 |
section {* Known Bugs and Limitations |
52805 | 2259 |
\label{sec:known-bugs-and-limitations} *} |
2260 |
||
2261 |
text {* |
|
53623 | 2262 |
Known open issues of the package. |
52805 | 2263 |
*} |
52794 | 2264 |
|
2265 |
text {* |
|
53753
ae7f50e70c09
renamed "primcorec" to "primcorecursive", to open the door to a 'theory -> theory' command called "primcorec" (cf. "fun" vs. "function")
blanchet
parents:
53752
diff
changeset
|
2266 |
%* primcorecursive and primcorec is unfinished |
53617 | 2267 |
% |
2268 |
%* slow n-ary mutual (co)datatype, avoid as much as possible (e.g. using nesting) |
|
2269 |
% |
|
2270 |
%* issues with HOL-Proofs? |
|
2271 |
% |
|
2272 |
%* partial documentation |
|
2273 |
% |
|
2274 |
%* no way to register "sum" and "prod" as (co)datatypes to enable N2M reduction for them |
|
2275 |
% (for @{command datatype_new_compat} and prim(co)rec) |
|
2276 |
% |
|
53619 | 2277 |
% * a fortiori, no way to register same type as both data- and codatatype |
53617 | 2278 |
% |
2279 |
%* no recursion through unused arguments (unlike with the old package) |
|
2280 |
% |
|
2281 |
%* in a locale, cannot use locally fixed types (because of limitation in typedef)? |
|
53619 | 2282 |
% |
2283 |
% *names of variables suboptimal |
|
52822 | 2284 |
*} |
53675 | 2285 |
*) |
52822 | 2286 |
|
2287 |
||
2288 |
text {* |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2289 |
\section*{Acknowledgment} |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2290 |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2291 |
Tobias Nipkow and Makarius Wenzel encouraged us to implement the new |
53617 | 2292 |
(co)datatype package. Andreas Lochbihler provided lots of comments on earlier |
2293 |
versions of the package, especially for the coinductive part. Brian Huffman |
|
2294 |
suggested major simplifications to the internal constructions, much of which has |
|
2295 |
yet to be implemented. Florian Haftmann and Christian Urban provided general |
|
53675 | 2296 |
advice on Isabelle and package writing. Stefan Milius and Lutz Schr\"oder |
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2297 |
found an elegant proof to eliminate one of the BNF assumptions. Christian |
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2298 |
Sternagel suggested many textual improvements to this tutorial. |
52794 | 2299 |
*} |
53617 | 2300 |
|
52792 | 2301 |
end |