| author | Andreas Lochbihler |
| Thu, 26 Sep 2013 16:50:40 +0200 | |
| changeset 53928 | 2e75da4fe4b6 |
| parent 53917 | bf74357f91f8 |
| child 53997 | 8ff43f638da2 |
| 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 {*
|
| 53647 | 879 |
The command @{command datatype_new} was designed to be highly compatible with
|
| 53752 | 880 |
\keyw{datatype}, to ease migration. There are nonetheless a number of
|
| 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.}
|
|
912 |
The properties @{text t.cases} and @{text t.recs} have been renamed to
|
|
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, |
|
916 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m.inducts(i)"} has been renamed to
|
|
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 |
||
| 53617 | 1319 |
(* |
| 52828 | 1320 |
subsection {* Compatibility Issues
|
| 53617 | 1321 |
\label{ssec:primrec-compatibility-issues} *}
|
| 52828 | 1322 |
|
1323 |
text {*
|
|
| 53617 | 1324 |
% * different induction in nested case |
1325 |
% * solution: define nested-as-mutual functions with primrec, |
|
1326 |
% and look at .induct |
|
1327 |
% |
|
1328 |
% * different induction and recursor in nested case |
|
1329 |
% * only matters to low-level users; they can define a dummy function to force |
|
1330 |
% generation of mutualized recursor |
|
| 52828 | 1331 |
*} |
| 53617 | 1332 |
*) |
| 52794 | 1333 |
|
1334 |
||
| 52827 | 1335 |
section {* Defining Codatatypes
|
| 52805 | 1336 |
\label{sec:defining-codatatypes} *}
|
1337 |
||
1338 |
text {*
|
|
| 53829 | 1339 |
Codatatypes can be specified using the @{command codatatype} command. The
|
| 53623 | 1340 |
command is first illustrated through concrete examples featuring different |
1341 |
flavors of corecursion. More examples can be found in the directory |
|
1342 |
\verb|~~/src/HOL/BNF/Examples|. The \emph{Archive of Formal Proofs} also
|
|
1343 |
includes some useful codatatypes, notably for lazy lists \cite{lochbihler-2010}.
|
|
| 52805 | 1344 |
*} |
| 52792 | 1345 |
|
| 52824 | 1346 |
|
| 53617 | 1347 |
subsection {* Introductory Examples
|
1348 |
\label{ssec:codatatype-introductory-examples} *}
|
|
| 52794 | 1349 |
|
| 53623 | 1350 |
|
1351 |
subsubsection {* Simple Corecursion
|
|
1352 |
\label{sssec:codatatype-simple-corecursion} *}
|
|
1353 |
||
| 52805 | 1354 |
text {*
|
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1355 |
Noncorecursive codatatypes coincide with the corresponding datatypes, so they |
|
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1356 |
are useless in practice. \emph{Corecursive codatatypes} have the same syntax
|
| 53623 | 1357 |
as recursive datatypes, except for the command name. For example, here is the |
1358 |
definition of lazy lists: |
|
1359 |
*} |
|
1360 |
||
1361 |
codatatype (lset: 'a) llist (map: lmap rel: llist_all2) = |
|
1362 |
lnull: LNil (defaults ltl: LNil) |
|
1363 |
| LCons (lhd: 'a) (ltl: "'a llist") |
|
1364 |
||
1365 |
text {*
|
|
1366 |
\noindent |
|
1367 |
Lazy lists can be infinite, such as @{text "LCons 0 (LCons 0 (\<dots>))"} and
|
|
| 53647 | 1368 |
@{text "LCons 0 (LCons 1 (LCons 2 (\<dots>)))"}. Here is a related type, that of
|
1369 |
infinite streams: |
|
1370 |
*} |
|
1371 |
||
1372 |
codatatype (sset: 'a) stream (map: smap rel: stream_all2) = |
|
1373 |
SCons (shd: 'a) (stl: "'a stream") |
|
1374 |
||
1375 |
text {*
|
|
1376 |
\noindent |
|
1377 |
Another interesting type that can |
|
| 53623 | 1378 |
be defined as a codatatype is that of the extended natural numbers: |
1379 |
*} |
|
1380 |
||
| 53644 | 1381 |
codatatype enat = EZero | ESuc enat |
| 53623 | 1382 |
|
1383 |
text {*
|
|
1384 |
\noindent |
|
1385 |
This type has exactly one infinite element, @{text "ESuc (ESuc (ESuc (\<dots>)))"},
|
|
1386 |
that represents $\infty$. In addition, it has finite values of the form |
|
1387 |
@{text "ESuc (\<dots> (ESuc EZero)\<dots>)"}.
|
|
| 53675 | 1388 |
|
1389 |
Here is an example with many constructors: |
|
| 52805 | 1390 |
*} |
| 53623 | 1391 |
|
| 53675 | 1392 |
codatatype 'a process = |
1393 |
Fail |
|
1394 |
| Skip (cont: "'a process") |
|
1395 |
| Action (prefix: 'a) (cont: "'a process") |
|
1396 |
| Choice (left: "'a process") (right: "'a process") |
|
1397 |
||
| 53750 | 1398 |
text {*
|
| 53829 | 1399 |
\noindent |
| 53750 | 1400 |
Notice that the @{const cont} selector is associated with both @{const Skip}
|
1401 |
and @{const Choice}.
|
|
1402 |
*} |
|
1403 |
||
| 53623 | 1404 |
|
1405 |
subsubsection {* Mutual Corecursion
|
|
1406 |
\label{sssec:codatatype-mutual-corecursion} *}
|
|
1407 |
||
1408 |
text {*
|
|
1409 |
\noindent |
|
1410 |
The example below introduces a pair of \emph{mutually corecursive} types:
|
|
1411 |
*} |
|
1412 |
||
1413 |
codatatype even_enat = Even_EZero | Even_ESuc odd_enat |
|
1414 |
and odd_enat = Odd_ESuc even_enat |
|
1415 |
||
1416 |
||
1417 |
subsubsection {* Nested Corecursion
|
|
1418 |
\label{sssec:codatatype-nested-corecursion} *}
|
|
1419 |
||
1420 |
text {*
|
|
1421 |
\noindent |
|
| 53675 | 1422 |
The next examples feature \emph{nested corecursion}:
|
| 53623 | 1423 |
*} |
1424 |
||
| 53644 | 1425 |
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 | 1426 |
|
| 53752 | 1427 |
text {* \blankline *}
|
1428 |
||
| 53644 | 1429 |
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 | 1430 |
|
| 53752 | 1431 |
text {* \blankline *}
|
1432 |
||
| 53675 | 1433 |
codatatype 'a state_machine = |
| 53751 | 1434 |
State_Machine (accept: bool) (trans: "'a \<Rightarrow> 'a state_machine") |
| 53675 | 1435 |
|
| 52824 | 1436 |
|
| 53617 | 1437 |
subsection {* Command Syntax
|
1438 |
\label{ssec:codatatype-command-syntax} *}
|
|
| 52805 | 1439 |
|
| 53619 | 1440 |
|
| 53621 | 1441 |
subsubsection {* \keyw{codatatype}
|
1442 |
\label{sssec:codatatype} *}
|
|
| 53619 | 1443 |
|
| 52824 | 1444 |
text {*
|
| 53829 | 1445 |
\begin{matharray}{rcl}
|
1446 |
@{command_def "codatatype"} & : & @{text "local_theory \<rightarrow> local_theory"}
|
|
1447 |
\end{matharray}
|
|
1448 |
||
1449 |
@{rail "
|
|
1450 |
@@{command codatatype} target? \\
|
|
1451 |
(@{syntax dt_name} '=' (@{syntax ctor} + '|') + @'and')
|
|
1452 |
"} |
|
1453 |
||
1454 |
\noindent |
|
| 52827 | 1455 |
Definitions of codatatypes have almost exactly the same syntax as for datatypes |
| 53829 | 1456 |
(Section~\ref{ssec:datatype-command-syntax}). The @{text "no_discs_sels"} option
|
1457 |
is not available, because destructors are a crucial notion for codatatypes. |
|
| 53623 | 1458 |
*} |
1459 |
||
1460 |
||
1461 |
subsection {* Generated Constants
|
|
1462 |
\label{ssec:codatatype-generated-constants} *}
|
|
1463 |
||
1464 |
text {*
|
|
1465 |
Given a codatatype @{text "('a\<^sub>1, \<dots>, 'a\<^sub>m) t"}
|
|
1466 |
with $m > 0$ live type variables and $n$ constructors @{text "t.C\<^sub>1"},
|
|
1467 |
\ldots, @{text "t.C\<^sub>n"}, the same auxiliary constants are generated as for
|
|
1468 |
datatypes (Section~\ref{ssec:datatype-generated-constants}), except that the
|
|
1469 |
iterator and the recursor are replaced by dual concepts: |
|
1470 |
||
1471 |
\begin{itemize}
|
|
1472 |
\setlength{\itemsep}{0pt}
|
|
1473 |
||
1474 |
\item \relax{Coiterator}: @{text t_unfold}
|
|
1475 |
||
1476 |
\item \relax{Corecursor}: @{text t_corec}
|
|
1477 |
||
1478 |
\end{itemize}
|
|
1479 |
*} |
|
1480 |
||
1481 |
||
1482 |
subsection {* Generated Theorems
|
|
1483 |
\label{ssec:codatatype-generated-theorems} *}
|
|
1484 |
||
1485 |
text {*
|
|
| 53829 | 1486 |
The characteristic theorems generated by @{command codatatype} are grouped in
|
| 53623 | 1487 |
three broad categories: |
1488 |
||
1489 |
\begin{itemize}
|
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1490 |
\setlength{\itemsep}{0pt}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1491 |
|
| 53623 | 1492 |
\item The \emph{free constructor theorems} are properties about the constructors
|
1493 |
and destructors that can be derived for any freely generated type. |
|
1494 |
||
1495 |
\item The \emph{functorial theorems} are properties of datatypes related to
|
|
1496 |
their BNF nature. |
|
1497 |
||
1498 |
\item The \emph{coinductive theorems} are properties of datatypes related to
|
|
1499 |
their coinductive nature. |
|
1500 |
\end{itemize}
|
|
1501 |
||
1502 |
\noindent |
|
1503 |
The first two categories are exactly as for datatypes and are described in |
|
| 53642 | 1504 |
Sections |
1505 |
\ref{sssec:free-constructor-theorems}~and~\ref{sssec:functorial-theorems}.
|
|
| 52824 | 1506 |
*} |
1507 |
||
| 53617 | 1508 |
|
| 53623 | 1509 |
subsubsection {* Coinductive Theorems
|
1510 |
\label{sssec:coinductive-theorems} *}
|
|
1511 |
||
1512 |
text {*
|
|
1513 |
The coinductive theorems are as follows: |
|
1514 |
||
1515 |
\begin{indentblock}
|
|
1516 |
\begin{description}
|
|
1517 |
||
| 53643 | 1518 |
\item[\begin{tabular}{@ {}l@ {}}
|
1519 |
@{text "t."}\hthm{coinduct} @{text "[coinduct t, consumes m, case_names t\<^sub>1 \<dots> t\<^sub>m,"} \\
|
|
1520 |
\phantom{@{text "t."}\hthm{coinduct} @{text "["}}@{text "case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"}\rm:
|
|
1521 |
\end{tabular}] ~ \\
|
|
| 53623 | 1522 |
@{thm llist.coinduct[no_vars]}
|
| 53617 | 1523 |
|
| 53643 | 1524 |
\item[\begin{tabular}{@ {}l@ {}}
|
1525 |
@{text "t."}\hthm{strong\_coinduct} @{text "[consumes m, case_names t\<^sub>1 \<dots> t\<^sub>m,"} \\
|
|
1526 |
\phantom{@{text "t."}\hthm{strong\_coinduct} @{text "["}}@{text "case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"}\rm:
|
|
1527 |
\end{tabular}] ~ \\
|
|
1528 |
@{thm llist.strong_coinduct[no_vars]}
|
|
| 53617 | 1529 |
|
| 53643 | 1530 |
\item[\begin{tabular}{@ {}l@ {}}
|
1531 |
@{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]"} \\
|
|
1532 |
@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{strong\_coinduct} @{text "[case_names t\<^sub>1 \<dots> t\<^sub>m,"} \\
|
|
1533 |
\phantom{@{text "t\<^sub>1_\<dots>_t\<^sub>m."}\hthm{strong\_coinduct} @{text "["}}@{text "case_conclusion D\<^sub>1 \<dots> D\<^sub>n]"}\rm:
|
|
1534 |
\end{tabular}] ~ \\
|
|
1535 |
Given $m > 1$ mutually corecursive codatatypes, these coinduction rules can be |
|
1536 |
used to prove $m$ properties simultaneously. |
|
1537 |
||
1538 |
\item[@{text "t."}\hthm{unfold} \rm(@{text "[simp]"})\rm:] ~ \\
|
|
| 53623 | 1539 |
@{thm llist.unfold(1)[no_vars]} \\
|
1540 |
@{thm llist.unfold(2)[no_vars]}
|
|
1541 |
||
| 53643 | 1542 |
\item[@{text "t."}\hthm{corec} (@{text "[simp]"})\rm:] ~ \\
|
| 53623 | 1543 |
@{thm llist.corec(1)[no_vars]} \\
|
1544 |
@{thm llist.corec(2)[no_vars]}
|
|
1545 |
||
| 53703 | 1546 |
\item[@{text "t."}\hthm{disc\_unfold}\rm:] ~ \\
|
| 53643 | 1547 |
@{thm llist.disc_unfold(1)[no_vars]} \\
|
1548 |
@{thm llist.disc_unfold(2)[no_vars]}
|
|
1549 |
||
| 53703 | 1550 |
\item[@{text "t."}\hthm{disc\_corec}\rm:] ~ \\
|
| 53643 | 1551 |
@{thm llist.disc_corec(1)[no_vars]} \\
|
1552 |
@{thm llist.disc_corec(2)[no_vars]}
|
|
1553 |
||
1554 |
\item[@{text "t."}\hthm{disc\_unfold\_iff} @{text "[simp]"}\rm:] ~ \\
|
|
1555 |
@{thm llist.disc_unfold_iff(1)[no_vars]} \\
|
|
1556 |
@{thm llist.disc_unfold_iff(2)[no_vars]}
|
|
1557 |
||
1558 |
\item[@{text "t."}\hthm{disc\_corec\_iff} @{text "[simp]"}\rm:] ~ \\
|
|
1559 |
@{thm llist.disc_corec_iff(1)[no_vars]} \\
|
|
1560 |
@{thm llist.disc_corec_iff(2)[no_vars]}
|
|
1561 |
||
1562 |
\item[@{text "t."}\hthm{sel\_unfold} @{text "[simp]"}\rm:] ~ \\
|
|
1563 |
@{thm llist.sel_unfold(1)[no_vars]} \\
|
|
1564 |
@{thm llist.sel_unfold(2)[no_vars]}
|
|
1565 |
||
1566 |
\item[@{text "t."}\hthm{sel\_corec} @{text "[simp]"}\rm:] ~ \\
|
|
1567 |
@{thm llist.sel_corec(1)[no_vars]} \\
|
|
1568 |
@{thm llist.sel_corec(2)[no_vars]}
|
|
1569 |
||
| 53623 | 1570 |
\end{description}
|
1571 |
\end{indentblock}
|
|
1572 |
||
1573 |
\noindent |
|
| 53829 | 1574 |
For convenience, @{command codatatype} also provides the following collection:
|
| 53623 | 1575 |
|
1576 |
\begin{indentblock}
|
|
1577 |
\begin{description}
|
|
1578 |
||
| 53643 | 1579 |
\item[@{text "t."}\hthm{simps} = @{text t.inject} @{text t.distinct} @{text t.case} @{text t.corec}$^*$ @{text t.disc_corec}] ~ \\
|
1580 |
@{text t.disc_corec_iff} @{text t.sel_corec} @{text t.unfold}$^*$ @{text t.disc_unfold} @{text t.disc_unfold_iff} ~ \\
|
|
| 53694 | 1581 |
@{text t.sel_unfold} @{text t.map} @{text t.rel_inject} @{text t.rel_distinct} @{text t.set}
|
| 53623 | 1582 |
|
1583 |
\end{description}
|
|
1584 |
\end{indentblock}
|
|
1585 |
*} |
|
| 52805 | 1586 |
|
1587 |
||
| 52827 | 1588 |
section {* Defining Corecursive Functions
|
| 52805 | 1589 |
\label{sec:defining-corecursive-functions} *}
|
1590 |
||
1591 |
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
|
1592 |
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
|
1593 |
@{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
|
1594 |
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
|
1595 |
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
|
1596 |
\verb|~~/src/HOL/BNF/Examples|. |
| 53644 | 1597 |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1598 |
Whereas recursive functions consume datatypes one constructor at a time, |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1599 |
corecursive functions construct codatatypes one constructor at a time. |
| 53752 | 1600 |
Partly reflecting a lack of agreement among proponents of coalgebraic methods, |
1601 |
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
|
1602 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1603 |
\begin{itemize}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1604 |
\setlength{\itemsep}{0pt}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1605 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1606 |
\abovedisplayskip=.5\abovedisplayskip |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1607 |
\belowdisplayskip=.5\belowdisplayskip |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1608 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1609 |
\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
|
1610 |
\[@{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
|
1611 |
equations of the form |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1612 |
\[@{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
|
1613 |
This style is popular in the coalgebraic literature. |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1614 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1615 |
\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
|
1616 |
\[@{text "\<dots> \<Longrightarrow> f x\<^sub>1 \<dots> x\<^sub>n = C \<dots>"}\]
|
| 53752 | 1617 |
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
|
1618 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1619 |
\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
|
1620 |
\[@{text "f x\<^sub>1 \<dots> x\<^sub>n = \<dots>"}\]
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1621 |
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
|
1622 |
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
|
1623 |
style. |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1624 |
\end{itemize}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1625 |
|
|
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
|
1626 |
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
|
1627 |
characteristic theorems for all three styles are generated. |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1628 |
|
| 53644 | 1629 |
\begin{framed}
|
1630 |
\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
|
1631 |
\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
|
1632 |
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
|
1633 |
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
|
1634 |
generated @{text t_unfold} or @{text t_corec} combinators.
|
| 53644 | 1635 |
\end{framed}
|
| 52828 | 1636 |
|
1637 |
%%% TODO: partial_function? E.g. for defining tail recursive function on lazy |
|
1638 |
%%% lists (cf. terminal0 in TLList.thy) |
|
| 52805 | 1639 |
*} |
1640 |
||
| 52824 | 1641 |
|
| 53617 | 1642 |
subsection {* Introductory Examples
|
1643 |
\label{ssec:primcorec-introductory-examples} *}
|
|
| 52805 | 1644 |
|
| 53646 | 1645 |
text {*
|
1646 |
Primitive corecursion is illustrated through concrete examples based on the |
|
1647 |
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
|
1648 |
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
|
1649 |
view is favored in the examples below. Sections |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1650 |
\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
|
1651 |
present the same examples expressed using the constructor and destructor views. |
| 53646 | 1652 |
*} |
1653 |
||
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1654 |
(*<*) |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1655 |
locale code_view |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1656 |
begin |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1657 |
(*>*) |
| 53644 | 1658 |
|
1659 |
subsubsection {* Simple Corecursion
|
|
1660 |
\label{sssec:primcorec-simple-corecursion} *}
|
|
1661 |
||
| 53646 | 1662 |
text {*
|
| 53752 | 1663 |
Following the code view, corecursive calls are allowed on the right-hand side as |
1664 |
long as they occur under a constructor, which itself appears either directly to |
|
1665 |
the right of the equal sign or in a conditional expression: |
|
| 53646 | 1666 |
*} |
1667 |
||
| 53826 | 1668 |
primcorec literate :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a llist" where
|
| 53647 | 1669 |
"literate f x = LCons x (literate f (f x))" |
1670 |
||
| 53677 | 1671 |
text {* \blankline *}
|
1672 |
||
| 53826 | 1673 |
primcorec siterate :: "('a \<Rightarrow> 'a) \<Rightarrow> 'a \<Rightarrow> 'a stream" where
|
| 53647 | 1674 |
"siterate f x = SCons x (siterate f (f x))" |
| 53644 | 1675 |
|
| 53646 | 1676 |
text {*
|
1677 |
\noindent |
|
1678 |
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
|
1679 |
\emph{productive}. The above functions compute the infinite lazy list or stream
|
| 53646 | 1680 |
@{text "[x, f x, f (f x), \<dots>]"}. Productivity guarantees that prefixes
|
1681 |
@{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
|
1682 |
@{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
|
1683 |
times. |
| 53646 | 1684 |
|
| 53752 | 1685 |
Corecursive functions construct codatatype values, but nothing prevents them |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
1686 |
from also consuming such values. The following function drops every second |
| 53675 | 1687 |
element in a stream: |
1688 |
*} |
|
1689 |
||
| 53826 | 1690 |
primcorec every_snd :: "'a stream \<Rightarrow> 'a stream" where |
| 53675 | 1691 |
"every_snd s = SCons (shd s) (stl (stl s))" |
1692 |
||
1693 |
text {*
|
|
| 53752 | 1694 |
\noindent |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1695 |
Constructs such as @{text "let"}---@{text "in"}, @{text
|
| 53646 | 1696 |
"if"}---@{text "then"}---@{text "else"}, and @{text "case"}---@{text "of"} may
|
1697 |
appear around constructors that guard corecursive calls: |
|
1698 |
*} |
|
1699 |
||
| 53826 | 1700 |
primcorec_notyet lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
| 53644 | 1701 |
"lappend xs ys = |
1702 |
(case xs of |
|
1703 |
LNil \<Rightarrow> ys |
|
1704 |
| LCons x xs' \<Rightarrow> LCons x (lappend xs' ys))" |
|
1705 |
||
| 53646 | 1706 |
text {*
|
| 53752 | 1707 |
\noindent |
| 53646 | 1708 |
Corecursion is useful to specify not only functions but also infinite objects: |
1709 |
*} |
|
1710 |
||
| 53826 | 1711 |
primcorec infty :: enat where |
| 53644 | 1712 |
"infty = ESuc infty" |
1713 |
||
| 53646 | 1714 |
text {*
|
| 53752 | 1715 |
\noindent |
1716 |
The example below constructs a pseudorandom process value. It takes a stream of |
|
| 53675 | 1717 |
actions (@{text s}), a pseudorandom function generator (@{text f}), and a
|
1718 |
pseudorandom seed (@{text n}):
|
|
1719 |
*} |
|
1720 |
||
| 53826 | 1721 |
primcorec_notyet |
| 53752 | 1722 |
random_process :: "'a stream \<Rightarrow> (int \<Rightarrow> int) \<Rightarrow> int \<Rightarrow> 'a process" |
1723 |
where |
|
| 53675 | 1724 |
"random_process s f n = |
1725 |
(if n mod 4 = 0 then |
|
1726 |
Fail |
|
1727 |
else if n mod 4 = 1 then |
|
1728 |
Skip (random_process s f (f n)) |
|
1729 |
else if n mod 4 = 2 then |
|
1730 |
Action (shd s) (random_process (stl s) f (f n)) |
|
1731 |
else |
|
1732 |
Choice (random_process (every_snd s) (f \<circ> f) (f n)) |
|
1733 |
(random_process (every_snd (stl s)) (f \<circ> f) (f (f n))))" |
|
1734 |
||
1735 |
text {*
|
|
1736 |
\noindent |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1737 |
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
|
1738 |
sequentially. This is visible in the generated theorems. The constructor and |
| 53752 | 1739 |
destructor views offer nonsequential alternatives. |
| 53675 | 1740 |
*} |
1741 |
||
| 53644 | 1742 |
|
1743 |
subsubsection {* Mutual Corecursion
|
|
1744 |
\label{sssec:primcorec-mutual-corecursion} *}
|
|
1745 |
||
| 53647 | 1746 |
text {*
|
1747 |
The syntax for mutually corecursive functions over mutually corecursive |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1748 |
datatypes is unsurprising: |
| 53647 | 1749 |
*} |
1750 |
||
| 53826 | 1751 |
primcorec |
| 53644 | 1752 |
even_infty :: even_enat and |
1753 |
odd_infty :: odd_enat |
|
1754 |
where |
|
1755 |
"even_infty = Even_ESuc odd_infty" | |
|
1756 |
"odd_infty = Odd_ESuc even_infty" |
|
1757 |
||
1758 |
||
1759 |
subsubsection {* Nested Corecursion
|
|
1760 |
\label{sssec:primcorec-nested-corecursion} *}
|
|
1761 |
||
| 53647 | 1762 |
text {*
|
1763 |
The next pair of examples generalize the @{const literate} and @{const siterate}
|
|
1764 |
functions (Section~\ref{sssec:primcorec-nested-corecursion}) to possibly
|
|
1765 |
infinite trees in which subnodes are organized either as a lazy list (@{text
|
|
1766 |
tree\<^sub>i\<^sub>i}) or as a finite set (@{text tree\<^sub>i\<^sub>s}):
|
|
1767 |
*} |
|
1768 |
||
| 53826 | 1769 |
primcorec iterate\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>i" where
|
| 53644 | 1770 |
"iterate\<^sub>i\<^sub>i f x = Node\<^sub>i\<^sub>i x (lmap (iterate\<^sub>i\<^sub>i f) (f x))" |
1771 |
||
| 53677 | 1772 |
text {* \blankline *}
|
1773 |
||
| 53826 | 1774 |
primcorec iterate\<^sub>i\<^sub>s :: "('a \<Rightarrow> 'a fset) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>s" where
|
| 53644 | 1775 |
"iterate\<^sub>i\<^sub>s f x = Node\<^sub>i\<^sub>s x (fmap (iterate\<^sub>i\<^sub>s f) (f x))" |
1776 |
||
| 52805 | 1777 |
text {*
|
| 53752 | 1778 |
\noindent |
| 53675 | 1779 |
Deterministic finite automata (DFAs) are usually defined as 5-tuples |
1780 |
@{text "(Q, \<Sigma>, \<delta>, q\<^sub>0, F)"}, where @{text Q} is a finite set of states,
|
|
1781 |
@{text \<Sigma>} is a finite alphabet, @{text \<delta>} is a transition function, @{text q\<^sub>0}
|
|
1782 |
is an initial state, and @{text F} is a set of final states. The following
|
|
1783 |
function translates a DFA into a @{type state_machine}:
|
|
1784 |
*} |
|
1785 |
||
| 53826 | 1786 |
primcorec (*<*)(in early) (*>*) |
| 53752 | 1787 |
sm_of_dfa :: "('q \<Rightarrow> 'a \<Rightarrow> 'q) \<Rightarrow> 'q set \<Rightarrow> 'q \<Rightarrow> 'a state_machine"
|
1788 |
where |
|
1789 |
"sm_of_dfa \<delta> F q = State_Machine (q \<in> F) (sm_of_dfa \<delta> F o \<delta> q)" |
|
| 53675 | 1790 |
|
| 53751 | 1791 |
text {*
|
1792 |
\noindent |
|
1793 |
The map function for the function type (@{text \<Rightarrow>}) is composition
|
|
| 53752 | 1794 |
(@{text "op \<circ>"}). For convenience, corecursion through functions can be
|
1795 |
expressed using @{text \<lambda>}-expressions and function application rather
|
|
1796 |
than composition. For example: |
|
| 53751 | 1797 |
*} |
1798 |
||
| 53826 | 1799 |
primcorec |
| 53752 | 1800 |
sm_of_dfa :: "('q \<Rightarrow> 'a \<Rightarrow> 'q) \<Rightarrow> 'q set \<Rightarrow> 'q \<Rightarrow> 'a state_machine"
|
1801 |
where |
|
1802 |
"sm_of_dfa \<delta> F q = State_Machine (q \<in> F) (sm_of_dfa \<delta> F o \<delta> q)" |
|
1803 |
||
1804 |
text {* \blankline *}
|
|
1805 |
||
| 53826 | 1806 |
primcorec empty_sm :: "'a state_machine" where |
| 53752 | 1807 |
"empty_sm = State_Machine False (\<lambda>_. empty_sm)" |
| 53751 | 1808 |
|
| 53752 | 1809 |
text {* \blankline *}
|
1810 |
||
| 53826 | 1811 |
primcorec not_sm :: "'a state_machine \<Rightarrow> 'a state_machine" where |
| 53752 | 1812 |
"not_sm M = State_Machine (\<not> accept M) (\<lambda>a. not_sm (trans M a))" |
| 53751 | 1813 |
|
| 53752 | 1814 |
text {* \blankline *}
|
1815 |
||
| 53826 | 1816 |
primcorec |
| 53752 | 1817 |
or_sm :: "'a state_machine \<Rightarrow> 'a state_machine \<Rightarrow> 'a state_machine" |
1818 |
where |
|
1819 |
"or_sm M N = |
|
| 53751 | 1820 |
State_Machine (accept M \<or> accept N) |
| 53752 | 1821 |
(\<lambda>a. or_sm (trans M a) (trans N a))" |
| 53751 | 1822 |
|
| 53644 | 1823 |
|
1824 |
subsubsection {* Nested-as-Mutual Corecursion
|
|
1825 |
\label{sssec:primcorec-nested-as-mutual-corecursion} *}
|
|
1826 |
||
| 53647 | 1827 |
text {*
|
1828 |
Just as it is possible to recurse over nested recursive datatypes as if they |
|
1829 |
were mutually recursive |
|
1830 |
(Section~\ref{sssec:primrec-nested-as-mutual-recursion}), it is possible to
|
|
| 53752 | 1831 |
pretend that nested codatatypes are mutually corecursive. For example: |
| 53647 | 1832 |
*} |
1833 |
||
| 53826 | 1834 |
primcorec_notyet |
| 53644 | 1835 |
iterate\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a \<Rightarrow> 'a tree\<^sub>i\<^sub>i" and
|
1836 |
iterates\<^sub>i\<^sub>i :: "('a \<Rightarrow> 'a llist) \<Rightarrow> 'a llist \<Rightarrow> 'a tree\<^sub>i\<^sub>i llist"
|
|
1837 |
where |
|
1838 |
"iterate\<^sub>i\<^sub>i f x = Node\<^sub>i\<^sub>i x (iterates\<^sub>i\<^sub>i f (f x))" | |
|
1839 |
"iterates\<^sub>i\<^sub>i f xs = |
|
1840 |
(case xs of |
|
1841 |
LNil \<Rightarrow> LNil |
|
1842 |
| 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
|
1843 |
(*<*) |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1844 |
end |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1845 |
(*>*) |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1846 |
|
|
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 |
subsubsection {* Constructor View
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1849 |
\label{ssec:primrec-constructor-view} *}
|
|
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 |
locale ctr_view = code_view |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1853 |
begin |
|
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 |
text {*
|
| 53750 | 1857 |
The constructor view is similar to the code view, but there is one separate |
1858 |
conditional equation per constructor rather than a single unconditional |
|
1859 |
equation. Examples that rely on a single constructor, such as @{const literate}
|
|
1860 |
and @{const siterate}, are identical in both styles.
|
|
1861 |
||
1862 |
Here is an example where there is a difference: |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1863 |
*} |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1864 |
|
| 53826 | 1865 |
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
|
1866 |
"lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lappend xs ys = LNil" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1867 |
"_ \<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
|
1868 |
(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
|
1869 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1870 |
text {*
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1871 |
\noindent |
| 53752 | 1872 |
With the constructor view, we must distinguish between the @{const LNil} and
|
1873 |
the @{const LCons} case. The condition for @{const LCons} is
|
|
1874 |
left implicit, as the negation of that for @{const LNil}.
|
|
| 53750 | 1875 |
|
1876 |
For this example, the constructor view is slighlty more involved than the |
|
1877 |
code equation. Recall the code view version presented in |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1878 |
Section~\ref{sssec:primcorec-simple-corecursion}.
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1879 |
% TODO: \[{thm code_view.lappend.code}\]
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1880 |
The constructor view requires us to analyze the second argument (@{term ys}).
|
| 53752 | 1881 |
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
|
1882 |
% TODO: \[{thm lappend.code}\]
|
| 53750 | 1883 |
|
| 53752 | 1884 |
In contrast, the next example is arguably more naturally expressed in the |
1885 |
constructor view: |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1886 |
*} |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1887 |
|
|
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
1888 |
primcorec |
| 53752 | 1889 |
random_process :: "'a stream \<Rightarrow> (int \<Rightarrow> int) \<Rightarrow> int \<Rightarrow> 'a process" |
1890 |
where |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1891 |
"n mod 4 = 0 \<Longrightarrow> random_process s f n = Fail" | |
| 53752 | 1892 |
"n mod 4 = 1 \<Longrightarrow> |
1893 |
random_process s f n = Skip (random_process s f (f n))" | |
|
1894 |
"n mod 4 = 2 \<Longrightarrow> |
|
1895 |
random_process s f n = Action (shd s) (random_process (stl s) f (f n))" | |
|
1896 |
"n mod 4 = 3 \<Longrightarrow> |
|
1897 |
random_process s f n = Choice (random_process (every_snd s) f (f n)) |
|
| 53826 | 1898 |
(random_process (every_snd (stl s)) f (f n))" |
1899 |
(*<*) |
|
| 53644 | 1900 |
end |
1901 |
(*>*) |
|
| 52805 | 1902 |
|
| 53750 | 1903 |
text {*
|
| 53752 | 1904 |
\noindent |
| 53750 | 1905 |
Since there is no sequentiality, we can apply the equation for @{const Choice}
|
| 53752 | 1906 |
without having first to discharge @{term "n mod (4\<Colon>int) \<noteq> 0"},
|
1907 |
@{term "n mod (4\<Colon>int) \<noteq> 1"}, and
|
|
1908 |
@{term "n mod (4\<Colon>int) \<noteq> 2"}.
|
|
| 53750 | 1909 |
The price to pay for this elegance is that we must discharge exclusivity proof |
1910 |
obligations, one for each pair of conditions |
|
| 53752 | 1911 |
@{term "(n mod (4\<Colon>int) = i, n mod (4\<Colon>int) = j)"}
|
1912 |
with @{term "i < j"}. If we prefer not to discharge any obligations, we can
|
|
1913 |
enable the @{text "sequential"} option. This pushes the problem to the users of
|
|
1914 |
the generated properties. |
|
| 53750 | 1915 |
%Here are more examples to conclude: |
1916 |
*} |
|
1917 |
||
| 52824 | 1918 |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1919 |
subsubsection {* Destructor View
|
| 53752 | 1920 |
\label{ssec:primrec-destructor-view} *}
|
1921 |
||
1922 |
(*<*) |
|
1923 |
locale dest_view |
|
1924 |
begin |
|
1925 |
(*>*) |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1926 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1927 |
text {*
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1928 |
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
|
1929 |
determine which constructor to choose, and these conditions are interpreted |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1930 |
sequentially or not depending on the @{text "sequential"} option.
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1931 |
Consider the following examples: |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1932 |
*} |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1933 |
|
| 53826 | 1934 |
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
|
1935 |
"\<not> lnull (literate _ x)" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1936 |
"lhd (literate _ x) = x" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1937 |
"ltl (literate f x) = literate f (f x)" |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1938 |
|
| 53752 | 1939 |
text {* \blankline *}
|
1940 |
||
| 53826 | 1941 |
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
|
1942 |
"shd (siterate _ x) = x" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1943 |
"stl (siterate f x) = siterate f (f x)" |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1944 |
|
| 53752 | 1945 |
text {* \blankline *}
|
1946 |
||
| 53826 | 1947 |
primcorec every_snd :: "'a stream \<Rightarrow> 'a stream" where |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1948 |
"shd (every_snd s) = shd s" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1949 |
"stl (every_snd s) = stl (stl s)" |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1950 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1951 |
text {*
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1952 |
\noindent |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1953 |
The first formula in the @{const literate} specification indicates which
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1954 |
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
|
1955 |
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
|
1956 |
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
|
1957 |
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
|
1958 |
Their arguments are unrestricted. |
| 53750 | 1959 |
|
1960 |
The next example shows how to specify functions that rely on more than one |
|
1961 |
constructor: |
|
1962 |
*} |
|
1963 |
||
| 53826 | 1964 |
primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
| 53750 | 1965 |
"lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lnull (lappend xs ys)" | |
1966 |
"lhd (lappend xs ys) = lhd (if lnull xs then ys else xs)" | |
|
1967 |
"ltl (lappend xs ys) = (if xs = LNil then ltl ys else lappend (ltl xs) ys)" |
|
1968 |
||
1969 |
text {*
|
|
1970 |
\noindent |
|
1971 |
For a codatatype with $n$ constructors, it is sufficient to specify $n - 1$ |
|
1972 |
discriminator formulas. The command will then assume that the remaining |
|
1973 |
constructor should be taken otherwise. This can be made explicit by adding |
|
1974 |
*} |
|
1975 |
||
1976 |
(*<*) |
|
1977 |
end |
|
1978 |
||
| 53826 | 1979 |
primcorec lappend :: "'a llist \<Rightarrow> 'a llist \<Rightarrow> 'a llist" where |
| 53750 | 1980 |
"lnull xs \<Longrightarrow> lnull ys \<Longrightarrow> lnull (lappend xs ys)" | |
1981 |
(*>*) |
|
| 53752 | 1982 |
"_ \<Longrightarrow> \<not> lnull (lappend xs ys)" |
1983 |
(*<*) | |
|
| 53750 | 1984 |
"lhd (lappend xs ys) = lhd (if lnull xs then ys else xs)" | |
1985 |
"ltl (lappend xs ys) = (if xs = LNil then ltl ys else lappend (ltl xs) ys)" |
|
1986 |
||
1987 |
context dest_view begin |
|
1988 |
(*>*) |
|
1989 |
||
1990 |
text {*
|
|
1991 |
\noindent |
|
| 53752 | 1992 |
to the specification. The generated selector theorems are conditional. |
1993 |
||
1994 |
The next example illustrates how to cope with selectors defined for several |
|
| 53750 | 1995 |
constructors: |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1996 |
*} |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
1997 |
|
|
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
1998 |
primcorec |
| 53752 | 1999 |
random_process :: "'a stream \<Rightarrow> (int \<Rightarrow> int) \<Rightarrow> int \<Rightarrow> 'a process" |
2000 |
where |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2001 |
"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
|
2002 |
"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
|
2003 |
"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
|
2004 |
"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
|
2005 |
"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
|
2006 |
"prefix (random_process s f n) = shd s" | |
|
53831
80423b9080cf
support "of" syntax to disambiguate selector equations
panny
parents:
53829
diff
changeset
|
2007 |
"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
|
2008 |
"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
|
2009 |
"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
|
2010 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2011 |
text {*
|
| 53750 | 2012 |
\noindent |
2013 |
Using the @{text "of"} keyword, different equations are specified for @{const
|
|
2014 |
cont} depending on which constructor is selected. |
|
2015 |
||
2016 |
Here are more examples to conclude: |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2017 |
*} |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2018 |
|
| 53826 | 2019 |
primcorec |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2020 |
even_infty :: even_enat and |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2021 |
odd_infty :: odd_enat |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2022 |
where |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2023 |
"\<not> is_Even_EZero even_infty" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2024 |
"un_Even_ESuc even_infty = odd_infty" | |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2025 |
"un_Odd_ESuc odd_infty = even_infty" |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2026 |
|
| 53752 | 2027 |
text {* \blankline *}
|
2028 |
||
| 53826 | 2029 |
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
|
2030 |
"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
|
2031 |
"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
|
2032 |
(*<*) |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2033 |
end |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2034 |
(*>*) |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2035 |
|
| 53750 | 2036 |
|
| 53617 | 2037 |
subsection {* Command Syntax
|
2038 |
\label{ssec:primcorec-command-syntax} *}
|
|
2039 |
||
2040 |
||
| 53826 | 2041 |
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
|
2042 |
\label{sssec:primcorecursive-and-primcorec} *}
|
| 52840 | 2043 |
|
2044 |
text {*
|
|
| 53829 | 2045 |
\begin{matharray}{rcl}
|
2046 |
@{command_def "primcorec"} & : & @{text "local_theory \<rightarrow> local_theory"} \\
|
|
2047 |
@{command_def "primcorecursive"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
|
|
2048 |
\end{matharray}
|
|
| 52840 | 2049 |
|
2050 |
@{rail "
|
|
| 53829 | 2051 |
(@@{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
|
2052 |
(@{syntax pcr_formula} + '|')
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2053 |
; |
| 53828 | 2054 |
@{syntax_def pcr_option}: '(' ('sequential' | 'exhaustive') ')'
|
| 52840 | 2055 |
; |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2056 |
@{syntax_def pcr_formula}: thmdecl? prop (@'of' (term * ))?
|
| 52840 | 2057 |
"} |
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2058 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2059 |
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
|
2060 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2061 |
\begin{itemize}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2062 |
\setlength{\itemsep}{0pt}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2063 |
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2064 |
\item |
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2065 |
The @{text "sequential"} option indicates that the conditions in specifications
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2066 |
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
|
2067 |
sequentially. |
| 53826 | 2068 |
|
2069 |
\item |
|
2070 |
The @{text "exhaustive"} option indicates that the conditions in specifications
|
|
2071 |
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
|
2072 |
\end{itemize}
|
|
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2073 |
|
| 53826 | 2074 |
\noindent |
2075 |
The @{command primcorec} command is an abbreviation for @{command primcorecursive} with
|
|
2076 |
@{text "by auto?"} to discharge any emerging proof obligations.
|
|
| 52840 | 2077 |
*} |
| 52794 | 2078 |
|
| 52824 | 2079 |
|
| 53619 | 2080 |
(* |
| 52840 | 2081 |
subsection {* Generated Theorems
|
2082 |
\label{ssec:primcorec-generated-theorems} *}
|
|
| 53619 | 2083 |
*) |
| 52794 | 2084 |
|
2085 |
||
| 53623 | 2086 |
(* |
2087 |
subsection {* Recursive Default Values for Selectors
|
|
2088 |
\label{ssec:primcorec-recursive-default-values-for-selectors} *}
|
|
2089 |
||
2090 |
text {*
|
|
2091 |
partial_function to the rescue |
|
2092 |
*} |
|
2093 |
*) |
|
2094 |
||
2095 |
||
| 52827 | 2096 |
section {* Registering Bounded Natural Functors
|
| 52805 | 2097 |
\label{sec:registering-bounded-natural-functors} *}
|
| 52792 | 2098 |
|
| 52805 | 2099 |
text {*
|
| 53647 | 2100 |
The (co)datatype package can be set up to allow nested recursion through |
2101 |
arbitrary type constructors, as long as they adhere to the BNF requirements and |
|
2102 |
are registered as BNFs. |
|
| 52805 | 2103 |
*} |
2104 |
||
| 52824 | 2105 |
|
| 53619 | 2106 |
(* |
| 53617 | 2107 |
subsection {* Introductory Example
|
2108 |
\label{ssec:bnf-introductory-example} *}
|
|
| 52805 | 2109 |
|
2110 |
text {*
|
|
2111 |
More examples in \verb|~~/src/HOL/BNF/Basic_BNFs.thy| and |
|
2112 |
\verb|~~/src/HOL/BNF/More_BNFs.thy|. |
|
| 52806 | 2113 |
|
| 53617 | 2114 |
%Mention distinction between live and dead type arguments; |
2115 |
% * and existence of map, set for those |
|
2116 |
%mention =>. |
|
| 52805 | 2117 |
*} |
| 53619 | 2118 |
*) |
| 52794 | 2119 |
|
| 52824 | 2120 |
|
| 53617 | 2121 |
subsection {* Command Syntax
|
2122 |
\label{ssec:bnf-command-syntax} *}
|
|
2123 |
||
2124 |
||
| 53621 | 2125 |
subsubsection {* \keyw{bnf}
|
2126 |
\label{sssec:bnf} *}
|
|
| 52794 | 2127 |
|
| 53028 | 2128 |
text {*
|
| 53829 | 2129 |
\begin{matharray}{rcl}
|
2130 |
@{command_def "bnf"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
|
|
2131 |
\end{matharray}
|
|
2132 |
||
| 53028 | 2133 |
@{rail "
|
| 53829 | 2134 |
@@{command bnf} target? (name ':')? term \\
|
| 53534 | 2135 |
term_list term term_list term? |
| 53028 | 2136 |
; |
| 53534 | 2137 |
X_list: '[' (X + ',') ']' |
| 53028 | 2138 |
"} |
2139 |
*} |
|
| 52805 | 2140 |
|
| 53617 | 2141 |
|
| 53621 | 2142 |
subsubsection {* \keyw{print\_bnfs}
|
2143 |
\label{sssec:print-bnfs} *}
|
|
| 53617 | 2144 |
|
2145 |
text {*
|
|
| 53829 | 2146 |
\begin{matharray}{rcl}
|
2147 |
@{command_def "print_bnfs"} & : & @{text "local_theory \<rightarrow>"}
|
|
2148 |
\end{matharray}
|
|
2149 |
||
| 53647 | 2150 |
@{rail "
|
| 53829 | 2151 |
@@{command print_bnfs}
|
| 53647 | 2152 |
"} |
| 53617 | 2153 |
*} |
2154 |
||
2155 |
||
2156 |
section {* Deriving Destructors and Theorems for Free Constructors
|
|
2157 |
\label{sec:deriving-destructors-and-theorems-for-free-constructors} *}
|
|
| 52794 | 2158 |
|
| 52805 | 2159 |
text {*
|
| 53623 | 2160 |
The derivation of convenience theorems for types equipped with free constructors, |
| 53829 | 2161 |
as performed internally by @{command datatype_new} and @{command codatatype},
|
| 53623 | 2162 |
is available as a stand-alone command called @{command wrap_free_constructors}.
|
| 52794 | 2163 |
|
| 53617 | 2164 |
% * need for this is rare but may arise if you want e.g. to add destructors to |
2165 |
% a type not introduced by ... |
|
2166 |
% |
|
2167 |
% * also useful for compatibility with old package, e.g. add destructors to |
|
2168 |
% old \keyw{datatype}
|
|
2169 |
% |
|
2170 |
% * @{command wrap_free_constructors}
|
|
| 53623 | 2171 |
% * @{text "no_discs_sels"}, @{text "rep_compat"}
|
| 53617 | 2172 |
% * hack to have both co and nonco view via locale (cf. ext nats) |
| 52805 | 2173 |
*} |
| 52792 | 2174 |
|
| 52824 | 2175 |
|
| 53619 | 2176 |
(* |
| 53617 | 2177 |
subsection {* Introductory Example
|
2178 |
\label{ssec:ctors-introductory-example} *}
|
|
| 53619 | 2179 |
*) |
| 52794 | 2180 |
|
| 52824 | 2181 |
|
| 53617 | 2182 |
subsection {* Command Syntax
|
2183 |
\label{ssec:ctors-command-syntax} *}
|
|
2184 |
||
2185 |
||
| 53621 | 2186 |
subsubsection {* \keyw{wrap\_free\_constructors}
|
| 53675 | 2187 |
\label{sssec:wrap-free-constructors} *}
|
| 52828 | 2188 |
|
| 53018 | 2189 |
text {*
|
| 53829 | 2190 |
\begin{matharray}{rcl}
|
2191 |
@{command_def "wrap_free_constructors"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
|
|
2192 |
\end{matharray}
|
|
| 53018 | 2193 |
|
2194 |
@{rail "
|
|
| 53829 | 2195 |
@@{command wrap_free_constructors} target? @{syntax dt_options} \\
|
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2196 |
term_list name @{syntax wfc_discs_sels}?
|
| 53018 | 2197 |
; |
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2198 |
@{syntax_def wfc_discs_sels}: name_list (name_list_list name_term_list_list? )?
|
| 53018 | 2199 |
; |
| 53534 | 2200 |
@{syntax_def name_term}: (name ':' term)
|
| 53018 | 2201 |
"} |
2202 |
||
| 53617 | 2203 |
% options: no_discs_sels rep_compat |
| 53028 | 2204 |
|
| 53617 | 2205 |
% X_list is as for BNF |
| 53028 | 2206 |
|
| 53829 | 2207 |
\noindent |
| 53542 | 2208 |
Section~\ref{ssec:datatype-generated-theorems} lists the generated theorems.
|
| 53018 | 2209 |
*} |
| 52828 | 2210 |
|
| 52794 | 2211 |
|
| 53617 | 2212 |
(* |
| 52827 | 2213 |
section {* Standard ML Interface
|
| 52805 | 2214 |
\label{sec:standard-ml-interface} *}
|
| 52792 | 2215 |
|
| 52805 | 2216 |
text {*
|
| 53623 | 2217 |
The package's programmatic interface. |
| 52805 | 2218 |
*} |
| 53617 | 2219 |
*) |
| 52794 | 2220 |
|
2221 |
||
| 53617 | 2222 |
(* |
| 52827 | 2223 |
section {* Interoperability
|
| 52805 | 2224 |
\label{sec:interoperability} *}
|
| 52794 | 2225 |
|
| 52805 | 2226 |
text {*
|
| 53623 | 2227 |
The package's interaction with other Isabelle packages and tools, such as the |
2228 |
code generator and the counterexample generators. |
|
| 52805 | 2229 |
*} |
| 52794 | 2230 |
|
| 52824 | 2231 |
|
| 52828 | 2232 |
subsection {* Transfer and Lifting
|
2233 |
\label{ssec:transfer-and-lifting} *}
|
|
| 52794 | 2234 |
|
| 52824 | 2235 |
|
| 52828 | 2236 |
subsection {* Code Generator
|
2237 |
\label{ssec:code-generator} *}
|
|
| 52794 | 2238 |
|
| 52824 | 2239 |
|
| 52828 | 2240 |
subsection {* Quickcheck
|
2241 |
\label{ssec:quickcheck} *}
|
|
| 52794 | 2242 |
|
| 52824 | 2243 |
|
| 52828 | 2244 |
subsection {* Nitpick
|
2245 |
\label{ssec:nitpick} *}
|
|
| 52794 | 2246 |
|
| 52824 | 2247 |
|
| 52828 | 2248 |
subsection {* Nominal Isabelle
|
2249 |
\label{ssec:nominal-isabelle} *}
|
|
| 53617 | 2250 |
*) |
| 52794 | 2251 |
|
| 52805 | 2252 |
|
| 53617 | 2253 |
(* |
| 52827 | 2254 |
section {* Known Bugs and Limitations
|
| 52805 | 2255 |
\label{sec:known-bugs-and-limitations} *}
|
2256 |
||
2257 |
text {*
|
|
| 53623 | 2258 |
Known open issues of the package. |
| 52805 | 2259 |
*} |
| 52794 | 2260 |
|
2261 |
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
|
2262 |
%* primcorecursive and primcorec is unfinished |
| 53617 | 2263 |
% |
2264 |
%* slow n-ary mutual (co)datatype, avoid as much as possible (e.g. using nesting) |
|
2265 |
% |
|
2266 |
%* issues with HOL-Proofs? |
|
2267 |
% |
|
2268 |
%* partial documentation |
|
2269 |
% |
|
2270 |
%* no way to register "sum" and "prod" as (co)datatypes to enable N2M reduction for them |
|
2271 |
% (for @{command datatype_new_compat} and prim(co)rec)
|
|
2272 |
% |
|
| 53619 | 2273 |
% * a fortiori, no way to register same type as both data- and codatatype |
| 53617 | 2274 |
% |
2275 |
%* no recursion through unused arguments (unlike with the old package) |
|
2276 |
% |
|
2277 |
%* in a locale, cannot use locally fixed types (because of limitation in typedef)? |
|
| 53619 | 2278 |
% |
2279 |
% *names of variables suboptimal |
|
| 52822 | 2280 |
*} |
| 53675 | 2281 |
*) |
| 52822 | 2282 |
|
2283 |
||
2284 |
text {*
|
|
|
53863
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2285 |
\section*{Acknowledgment}
|
|
c7364dca96f2
textual improvements following Christian Sternagel's feedback
blanchet
parents:
53857
diff
changeset
|
2286 |
|
|
53749
b37db925b663
adapted primcorec documentation to reflect the three views
blanchet
parents:
53748
diff
changeset
|
2287 |
Tobias Nipkow and Makarius Wenzel encouraged us to implement the new |
| 53617 | 2288 |
(co)datatype package. Andreas Lochbihler provided lots of comments on earlier |
2289 |
versions of the package, especially for the coinductive part. Brian Huffman |
|
2290 |
suggested major simplifications to the internal constructions, much of which has |
|
2291 |
yet to be implemented. Florian Haftmann and Christian Urban provided general |
|
| 53675 | 2292 |
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
|
2293 |
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
|
2294 |
Sternagel suggested many textual improvements to this tutorial. |
| 52794 | 2295 |
*} |
| 53617 | 2296 |
|
| 52792 | 2297 |
end |