author | haftmann |
Fri, 06 Feb 2015 17:57:03 +0100 | |
changeset 59487 | adaa430fc0f7 |
parent 58618 | 782f0b662cae |
child 59783 | 00b62aa9f430 |
permissions | -rw-r--r-- |
26840 | 1 |
theory HOL_Specific |
58372
bfd497f2f4c2
moved 'old_datatype' out of 'Main' (but put it in 'HOL-Proofs' because of the inductive realizer)
blanchet
parents:
58310
diff
changeset
|
2 |
imports Base "~~/src/HOL/Library/Old_Datatype" "~~/src/HOL/Library/Old_Recdef" |
bfd497f2f4c2
moved 'old_datatype' out of 'Main' (but put it in 'HOL-Proofs' because of the inductive realizer)
blanchet
parents:
58310
diff
changeset
|
3 |
"~~/src/Tools/Adhoc_Overloading" |
26840 | 4 |
begin |
5 |
||
58618 | 6 |
chapter \<open>Higher-Order Logic\<close> |
7 |
||
8 |
text \<open>Isabelle/HOL is based on Higher-Order Logic, a polymorphic |
|
42914 | 9 |
version of Church's Simple Theory of Types. HOL can be best |
10 |
understood as a simply-typed version of classical set theory. The |
|
11 |
logic was first implemented in Gordon's HOL system |
|
58552 | 12 |
@{cite "mgordon-hol"}. It extends Church's original logic |
13 |
@{cite "church40"} by explicit type variables (naive polymorphism) and |
|
42914 | 14 |
a sound axiomatization scheme for new types based on subsets of |
15 |
existing types. |
|
16 |
||
58552 | 17 |
Andrews's book @{cite andrews86} is a full description of the |
42914 | 18 |
original Church-style higher-order logic, with proofs of correctness |
19 |
and completeness wrt.\ certain set-theoretic interpretations. The |
|
20 |
particular extensions of Gordon-style HOL are explained semantically |
|
58552 | 21 |
in two chapters of the 1993 HOL book @{cite pitts93}. |
42914 | 22 |
|
23 |
Experience with HOL over decades has demonstrated that higher-order |
|
24 |
logic is widely applicable in many areas of mathematics and computer |
|
25 |
science. In a sense, Higher-Order Logic is simpler than First-Order |
|
26 |
Logic, because there are fewer restrictions and special cases. Note |
|
27 |
that HOL is \emph{weaker} than FOL with axioms for ZF set theory, |
|
28 |
which is traditionally considered the standard foundation of regular |
|
29 |
mathematics, but for most applications this does not matter. If you |
|
30 |
prefer ML to Lisp, you will probably prefer HOL to ZF. |
|
31 |
||
32 |
\medskip The syntax of HOL follows @{text "\<lambda>"}-calculus and |
|
33 |
functional programming. Function application is curried. To apply |
|
34 |
the function @{text f} of type @{text "\<tau>\<^sub>1 \<Rightarrow> \<tau>\<^sub>2 \<Rightarrow> \<tau>\<^sub>3"} to the |
|
35 |
arguments @{text a} and @{text b} in HOL, you simply write @{text "f |
|
36 |
a b"} (as in ML or Haskell). There is no ``apply'' operator; the |
|
37 |
existing application of the Pure @{text "\<lambda>"}-calculus is re-used. |
|
38 |
Note that in HOL @{text "f (a, b)"} means ``@{text "f"} applied to |
|
39 |
the pair @{text "(a, b)"} (which is notation for @{text "Pair a |
|
40 |
b"}). The latter typically introduces extra formal efforts that can |
|
41 |
be avoided by currying functions by default. Explicit tuples are as |
|
42 |
infrequent in HOL formalizations as in good ML or Haskell programs. |
|
43 |
||
44 |
\medskip Isabelle/HOL has a distinct feel, compared to other |
|
45 |
object-logics like Isabelle/ZF. It identifies object-level types |
|
46 |
with meta-level types, taking advantage of the default |
|
47 |
type-inference mechanism of Isabelle/Pure. HOL fully identifies |
|
48 |
object-level functions with meta-level functions, with native |
|
49 |
abstraction and application. |
|
50 |
||
51 |
These identifications allow Isabelle to support HOL particularly |
|
52 |
nicely, but they also mean that HOL requires some sophistication |
|
53 |
from the user. In particular, an understanding of Hindley-Milner |
|
54 |
type-inference with type-classes, which are both used extensively in |
|
55 |
the standard libraries and applications. Beginners can set |
|
56 |
@{attribute show_types} or even @{attribute show_sorts} to get more |
|
58618 | 57 |
explicit information about the result of type-inference.\<close> |
58 |
||
59 |
||
60 |
chapter \<open>Derived specification elements\<close> |
|
61 |
||
62 |
section \<open>Inductive and coinductive definitions \label{sec:hol-inductive}\<close> |
|
63 |
||
64 |
text \<open> |
|
46280 | 65 |
\begin{matharray}{rcl} |
66 |
@{command_def (HOL) "inductive"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
67 |
@{command_def (HOL) "inductive_set"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
68 |
@{command_def (HOL) "coinductive"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
69 |
@{command_def (HOL) "coinductive_set"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
50302 | 70 |
@{command_def "print_inductives"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
46280 | 71 |
@{attribute_def (HOL) mono} & : & @{text attribute} \\ |
72 |
\end{matharray} |
|
73 |
||
74 |
An \emph{inductive definition} specifies the least predicate or set |
|
75 |
@{text R} closed under given rules: applying a rule to elements of |
|
76 |
@{text R} yields a result within @{text R}. For example, a |
|
77 |
structural operational semantics is an inductive definition of an |
|
78 |
evaluation relation. |
|
42908 | 79 |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
80 |
Dually, a \emph{coinductive definition} specifies the greatest |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
81 |
predicate or set @{text R} that is consistent with given rules: |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
82 |
every element of @{text R} can be seen as arising by applying a rule |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
83 |
to elements of @{text R}. An important example is using |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
84 |
bisimulation relations to formalise equivalence of processes and |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
85 |
infinite data structures. |
47859 | 86 |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
87 |
Both inductive and coinductive definitions are based on the |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
88 |
Knaster-Tarski fixed-point theorem for complete lattices. The |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
89 |
collection of introduction rules given by the user determines a |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
90 |
functor on subsets of set-theoretic relations. The required |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
91 |
monotonicity of the recursion scheme is proven as a prerequisite to |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
92 |
the fixed-point definition and the resulting consequences. This |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
93 |
works by pushing inclusion through logical connectives and any other |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
94 |
operator that might be wrapped around recursive occurrences of the |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
95 |
defined relation: there must be a monotonicity theorem of the form |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
96 |
@{text "A \<le> B \<Longrightarrow> \<M> A \<le> \<M> B"}, for each premise @{text "\<M> R t"} in an |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
97 |
introduction rule. The default rule declarations of Isabelle/HOL |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
98 |
already take care of most common situations. |
42907
dfd4ef8e73f6
updated and re-unified HOL typedef, with some live examples;
wenzelm
parents:
42705
diff
changeset
|
99 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
100 |
@{rail \<open> |
42908 | 101 |
(@@{command (HOL) inductive} | @@{command (HOL) inductive_set} | |
102 |
@@{command (HOL) coinductive} | @@{command (HOL) coinductive_set}) |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
103 |
@{syntax target}? \<newline> |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
104 |
@{syntax "fixes"} (@'for' @{syntax "fixes"})? (@'where' clauses)? \<newline> |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
105 |
(@'monos' @{syntax thmrefs})? |
42908 | 106 |
; |
107 |
clauses: (@{syntax thmdecl}? @{syntax prop} + '|') |
|
108 |
; |
|
109 |
@@{attribute (HOL) mono} (() | 'add' | 'del') |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
110 |
\<close>} |
42908 | 111 |
|
112 |
\begin{description} |
|
113 |
||
114 |
\item @{command (HOL) "inductive"} and @{command (HOL) |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
115 |
"coinductive"} define (co)inductive predicates from the introduction |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
116 |
rules. |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
117 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
118 |
The propositions given as @{text "clauses"} in the @{keyword |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
119 |
"where"} part are either rules of the usual @{text "\<And>/\<Longrightarrow>"} format |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
120 |
(with arbitrary nesting), or equalities using @{text "\<equiv>"}. The |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
121 |
latter specifies extra-logical abbreviations in the sense of |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
122 |
@{command_ref abbreviation}. Introducing abstract syntax |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
123 |
simultaneously with the actual introduction rules is occasionally |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
124 |
useful for complex specifications. |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
125 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
126 |
The optional @{keyword "for"} part contains a list of parameters of |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
127 |
the (co)inductive predicates that remain fixed throughout the |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
128 |
definition, in contrast to arguments of the relation that may vary |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
129 |
in each occurrence within the given @{text "clauses"}. |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
130 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
131 |
The optional @{keyword "monos"} declaration contains additional |
42908 | 132 |
\emph{monotonicity theorems}, which are required for each operator |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
133 |
applied to a recursive set in the introduction rules. |
42908 | 134 |
|
135 |
\item @{command (HOL) "inductive_set"} and @{command (HOL) |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
136 |
"coinductive_set"} are wrappers for to the previous commands for |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
137 |
native HOL predicates. This allows to define (co)inductive sets, |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
138 |
where multiple arguments are simulated via tuples. |
42908 | 139 |
|
50302 | 140 |
\item @{command "print_inductives"} prints (co)inductive definitions and |
141 |
monotonicity rules. |
|
142 |
||
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
143 |
\item @{attribute (HOL) mono} declares monotonicity rules in the |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
144 |
context. These rule are involved in the automated monotonicity |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
145 |
proof of the above inductive and coinductive definitions. |
42908 | 146 |
|
147 |
\end{description} |
|
58618 | 148 |
\<close> |
149 |
||
150 |
||
151 |
subsection \<open>Derived rules\<close> |
|
152 |
||
153 |
text \<open>A (co)inductive definition of @{text R} provides the following |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
154 |
main theorems: |
42908 | 155 |
|
156 |
\begin{description} |
|
157 |
||
158 |
\item @{text R.intros} is the list of introduction rules as proven |
|
159 |
theorems, for the recursive predicates (or sets). The rules are |
|
160 |
also available individually, using the names given them in the |
|
161 |
theory file; |
|
162 |
||
163 |
\item @{text R.cases} is the case analysis (or elimination) rule; |
|
164 |
||
165 |
\item @{text R.induct} or @{text R.coinduct} is the (co)induction |
|
44273
336752fb25df
adding documentation about simps equation in the inductive package
bulwahn
parents:
44055
diff
changeset
|
166 |
rule; |
336752fb25df
adding documentation about simps equation in the inductive package
bulwahn
parents:
44055
diff
changeset
|
167 |
|
336752fb25df
adding documentation about simps equation in the inductive package
bulwahn
parents:
44055
diff
changeset
|
168 |
\item @{text R.simps} is the equation unrolling the fixpoint of the |
336752fb25df
adding documentation about simps equation in the inductive package
bulwahn
parents:
44055
diff
changeset
|
169 |
predicate one step. |
47859 | 170 |
|
42908 | 171 |
\end{description} |
172 |
||
173 |
When several predicates @{text "R\<^sub>1, \<dots>, R\<^sub>n"} are |
|
174 |
defined simultaneously, the list of introduction rules is called |
|
175 |
@{text "R\<^sub>1_\<dots>_R\<^sub>n.intros"}, the case analysis rules are |
|
176 |
called @{text "R\<^sub>1.cases, \<dots>, R\<^sub>n.cases"}, and the list |
|
177 |
of mutual induction rules is called @{text |
|
178 |
"R\<^sub>1_\<dots>_R\<^sub>n.inducts"}. |
|
58618 | 179 |
\<close> |
180 |
||
181 |
||
182 |
subsection \<open>Monotonicity theorems\<close> |
|
183 |
||
184 |
text \<open>The context maintains a default set of theorems that are used |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
185 |
in monotonicity proofs. New rules can be declared via the |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
186 |
@{attribute (HOL) mono} attribute. See the main Isabelle/HOL |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
187 |
sources for some examples. The general format of such monotonicity |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
188 |
theorems is as follows: |
42908 | 189 |
|
190 |
\begin{itemize} |
|
191 |
||
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
192 |
\item Theorems of the form @{text "A \<le> B \<Longrightarrow> \<M> A \<le> \<M> B"}, for proving |
42908 | 193 |
monotonicity of inductive definitions whose introduction rules have |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
194 |
premises involving terms such as @{text "\<M> R t"}. |
42908 | 195 |
|
196 |
\item Monotonicity theorems for logical operators, which are of the |
|
197 |
general form @{text "(\<dots> \<longrightarrow> \<dots>) \<Longrightarrow> \<dots> (\<dots> \<longrightarrow> \<dots>) \<Longrightarrow> \<dots> \<longrightarrow> \<dots>"}. For example, in |
|
198 |
the case of the operator @{text "\<or>"}, the corresponding theorem is |
|
199 |
\[ |
|
200 |
\infer{@{text "P\<^sub>1 \<or> P\<^sub>2 \<longrightarrow> Q\<^sub>1 \<or> Q\<^sub>2"}}{@{text "P\<^sub>1 \<longrightarrow> Q\<^sub>1"} & @{text "P\<^sub>2 \<longrightarrow> Q\<^sub>2"}} |
|
201 |
\] |
|
202 |
||
203 |
\item De Morgan style equations for reasoning about the ``polarity'' |
|
204 |
of expressions, e.g. |
|
205 |
\[ |
|
206 |
@{prop "\<not> \<not> P \<longleftrightarrow> P"} \qquad\qquad |
|
207 |
@{prop "\<not> (P \<and> Q) \<longleftrightarrow> \<not> P \<or> \<not> Q"} |
|
208 |
\] |
|
209 |
||
210 |
\item Equations for reducing complex operators to more primitive |
|
211 |
ones whose monotonicity can easily be proved, e.g. |
|
212 |
\[ |
|
213 |
@{prop "(P \<longrightarrow> Q) \<longleftrightarrow> \<not> P \<or> Q"} \qquad\qquad |
|
214 |
@{prop "Ball A P \<equiv> \<forall>x. x \<in> A \<longrightarrow> P x"} |
|
215 |
\] |
|
216 |
||
217 |
\end{itemize} |
|
58618 | 218 |
\<close> |
219 |
||
220 |
subsubsection \<open>Examples\<close> |
|
221 |
||
222 |
text \<open>The finite powerset operator can be defined inductively like this:\<close> |
|
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
223 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
224 |
inductive_set Fin :: "'a set \<Rightarrow> 'a set set" for A :: "'a set" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
225 |
where |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
226 |
empty: "{} \<in> Fin A" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
227 |
| insert: "a \<in> A \<Longrightarrow> B \<in> Fin A \<Longrightarrow> insert a B \<in> Fin A" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
228 |
|
58618 | 229 |
text \<open>The accessible part of a relation is defined as follows:\<close> |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
230 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
231 |
inductive acc :: "('a \<Rightarrow> 'a \<Rightarrow> bool) \<Rightarrow> 'a \<Rightarrow> bool" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
232 |
for r :: "'a \<Rightarrow> 'a \<Rightarrow> bool" (infix "\<prec>" 50) |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
233 |
where acc: "(\<And>y. y \<prec> x \<Longrightarrow> acc r y) \<Longrightarrow> acc r x" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
234 |
|
58618 | 235 |
text \<open>Common logical connectives can be easily characterized as |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
236 |
non-recursive inductive definitions with parameters, but without |
58618 | 237 |
arguments.\<close> |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
238 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
239 |
inductive AND for A B :: bool |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
240 |
where "A \<Longrightarrow> B \<Longrightarrow> AND A B" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
241 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
242 |
inductive OR for A B :: bool |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
243 |
where "A \<Longrightarrow> OR A B" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
244 |
| "B \<Longrightarrow> OR A B" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
245 |
|
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
246 |
inductive EXISTS for B :: "'a \<Rightarrow> bool" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
247 |
where "B a \<Longrightarrow> EXISTS B" |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
248 |
|
58618 | 249 |
text \<open>Here the @{text "cases"} or @{text "induct"} rules produced by |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
250 |
the @{command inductive} package coincide with the expected |
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
251 |
elimination rules for Natural Deduction. Already in the original |
58552 | 252 |
article by Gerhard Gentzen @{cite "Gentzen:1935"} there is a hint that |
42913
68bc69bdce88
updated and re-unified (co)inductive definitions in HOL;
wenzelm
parents:
42912
diff
changeset
|
253 |
each connective can be characterized by its introductions, and the |
58618 | 254 |
elimination can be constructed systematically.\<close> |
255 |
||
256 |
||
257 |
section \<open>Recursive functions \label{sec:recursion}\<close> |
|
258 |
||
259 |
text \<open> |
|
42908 | 260 |
\begin{matharray}{rcl} |
261 |
@{command_def (HOL) "primrec"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
262 |
@{command_def (HOL) "fun"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
263 |
@{command_def (HOL) "function"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\ |
|
264 |
@{command_def (HOL) "termination"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\ |
|
54017
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
265 |
@{command_def (HOL) "fun_cases"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
42908 | 266 |
\end{matharray} |
267 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
268 |
@{rail \<open> |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
269 |
@@{command (HOL) primrec} @{syntax target}? @{syntax "fixes"} @'where' equations |
42908 | 270 |
; |
271 |
(@@{command (HOL) fun} | @@{command (HOL) function}) @{syntax target}? functionopts? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
272 |
@{syntax "fixes"} \<newline> @'where' equations |
26849 | 273 |
; |
274 |
||
42908 | 275 |
equations: (@{syntax thmdecl}? @{syntax prop} + '|') |
26849 | 276 |
; |
42908 | 277 |
functionopts: '(' (('sequential' | 'domintros') + ',') ')' |
26849 | 278 |
; |
42908 | 279 |
@@{command (HOL) termination} @{syntax term}? |
54017
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
280 |
; |
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
281 |
@@{command (HOL) fun_cases} (@{syntax thmdecl}? @{syntax prop} + @'and') |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
282 |
\<close>} |
26849 | 283 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
284 |
\begin{description} |
42123 | 285 |
|
42908 | 286 |
\item @{command (HOL) "primrec"} defines primitive recursive |
58310 | 287 |
functions over datatypes (see also @{command_ref (HOL) datatype}). |
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
288 |
The given @{text equations} specify reduction rules that are produced |
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
289 |
by instantiating the generic combinator for primitive recursion that |
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
290 |
is available for each datatype. |
42912 | 291 |
|
292 |
Each equation needs to be of the form: |
|
293 |
||
294 |
@{text [display] "f x\<^sub>1 \<dots> x\<^sub>m (C y\<^sub>1 \<dots> y\<^sub>k) z\<^sub>1 \<dots> z\<^sub>n = rhs"} |
|
295 |
||
296 |
such that @{text C} is a datatype constructor, @{text rhs} contains |
|
297 |
only the free variables on the left-hand side (or from the context), |
|
298 |
and all recursive occurrences of @{text "f"} in @{text "rhs"} are of |
|
299 |
the form @{text "f \<dots> y\<^sub>i \<dots>"} for some @{text i}. At most one |
|
300 |
reduction rule for each constructor can be given. The order does |
|
301 |
not matter. For missing constructors, the function is defined to |
|
302 |
return a default value, but this equation is made difficult to |
|
303 |
access for users. |
|
304 |
||
305 |
The reduction rules are declared as @{attribute simp} by default, |
|
306 |
which enables standard proof methods like @{method simp} and |
|
307 |
@{method auto} to normalize expressions of @{text "f"} applied to |
|
308 |
datatype constructions, by simulating symbolic computation via |
|
309 |
rewriting. |
|
35744 | 310 |
|
42908 | 311 |
\item @{command (HOL) "function"} defines functions by general |
312 |
wellfounded recursion. A detailed description with examples can be |
|
58552 | 313 |
found in @{cite "isabelle-function"}. The function is specified by a |
42908 | 314 |
set of (possibly conditional) recursive equations with arbitrary |
315 |
pattern matching. The command generates proof obligations for the |
|
316 |
completeness and the compatibility of patterns. |
|
42907
dfd4ef8e73f6
updated and re-unified HOL typedef, with some live examples;
wenzelm
parents:
42705
diff
changeset
|
317 |
|
42908 | 318 |
The defined function is considered partial, and the resulting |
319 |
simplification rules (named @{text "f.psimps"}) and induction rule |
|
320 |
(named @{text "f.pinduct"}) are guarded by a generated domain |
|
321 |
predicate @{text "f_dom"}. The @{command (HOL) "termination"} |
|
322 |
command can then be used to establish that the function is total. |
|
42123 | 323 |
|
42908 | 324 |
\item @{command (HOL) "fun"} is a shorthand notation for ``@{command |
325 |
(HOL) "function"}~@{text "(sequential)"}, followed by automated |
|
326 |
proof attempts regarding pattern matching and termination. See |
|
58552 | 327 |
@{cite "isabelle-function"} for further details. |
42123 | 328 |
|
42908 | 329 |
\item @{command (HOL) "termination"}~@{text f} commences a |
330 |
termination proof for the previously defined function @{text f}. If |
|
331 |
this is omitted, the command refers to the most recent function |
|
332 |
definition. After the proof is closed, the recursive equations and |
|
333 |
the induction principle is established. |
|
26849 | 334 |
|
54017
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
335 |
\item @{command (HOL) "fun_cases"} generates specialized elimination |
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
336 |
rules for function equations. It expects one or more function equations |
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
337 |
and produces rules that eliminate the given equalities, following the cases |
2a3c07f49615
basic documentation for function elimination rules and fun_cases
krauss
parents:
53982
diff
changeset
|
338 |
given in the function definition. |
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
339 |
\end{description} |
42907
dfd4ef8e73f6
updated and re-unified HOL typedef, with some live examples;
wenzelm
parents:
42705
diff
changeset
|
340 |
|
42908 | 341 |
Recursive definitions introduced by the @{command (HOL) "function"} |
42912 | 342 |
command accommodate reasoning by induction (cf.\ @{method induct}): |
343 |
rule @{text "f.induct"} refers to a specific induction rule, with |
|
344 |
parameters named according to the user-specified equations. Cases |
|
345 |
are numbered starting from 1. For @{command (HOL) "primrec"}, the |
|
346 |
induction principle coincides with structural recursion on the |
|
347 |
datatype where the recursion is carried out. |
|
42908 | 348 |
|
349 |
The equations provided by these packages may be referred later as |
|
350 |
theorem list @{text "f.simps"}, where @{text f} is the (collective) |
|
351 |
name of the functions defined. Individual equations may be named |
|
352 |
explicitly as well. |
|
353 |
||
354 |
The @{command (HOL) "function"} command accepts the following |
|
355 |
options. |
|
356 |
||
357 |
\begin{description} |
|
358 |
||
359 |
\item @{text sequential} enables a preprocessor which disambiguates |
|
360 |
overlapping patterns by making them mutually disjoint. Earlier |
|
361 |
equations take precedence over later ones. This allows to give the |
|
362 |
specification in a format very similar to functional programming. |
|
363 |
Note that the resulting simplification and induction rules |
|
364 |
correspond to the transformed specification, not the one given |
|
365 |
originally. This usually means that each equation given by the user |
|
366 |
may result in several theorems. Also note that this automatic |
|
367 |
transformation only works for ML-style datatype patterns. |
|
368 |
||
369 |
\item @{text domintros} enables the automated generation of |
|
370 |
introduction rules for the domain predicate. While mostly not |
|
371 |
needed, they can be helpful in some proofs about partial functions. |
|
372 |
||
373 |
\end{description} |
|
58618 | 374 |
\<close> |
375 |
||
376 |
subsubsection \<open>Example: evaluation of expressions\<close> |
|
377 |
||
378 |
text \<open>Subsequently, we define mutual datatypes for arithmetic and |
|
42912 | 379 |
boolean expressions, and use @{command primrec} for evaluation |
58618 | 380 |
functions that follow the same recursive structure.\<close> |
42912 | 381 |
|
58310 | 382 |
datatype 'a aexp = |
42912 | 383 |
IF "'a bexp" "'a aexp" "'a aexp" |
384 |
| Sum "'a aexp" "'a aexp" |
|
385 |
| Diff "'a aexp" "'a aexp" |
|
386 |
| Var 'a |
|
387 |
| Num nat |
|
388 |
and 'a bexp = |
|
389 |
Less "'a aexp" "'a aexp" |
|
390 |
| And "'a bexp" "'a bexp" |
|
391 |
| Neg "'a bexp" |
|
392 |
||
393 |
||
58618 | 394 |
text \<open>\medskip Evaluation of arithmetic and boolean expressions\<close> |
42912 | 395 |
|
396 |
primrec evala :: "('a \<Rightarrow> nat) \<Rightarrow> 'a aexp \<Rightarrow> nat" |
|
397 |
and evalb :: "('a \<Rightarrow> nat) \<Rightarrow> 'a bexp \<Rightarrow> bool" |
|
398 |
where |
|
399 |
"evala env (IF b a1 a2) = (if evalb env b then evala env a1 else evala env a2)" |
|
400 |
| "evala env (Sum a1 a2) = evala env a1 + evala env a2" |
|
401 |
| "evala env (Diff a1 a2) = evala env a1 - evala env a2" |
|
402 |
| "evala env (Var v) = env v" |
|
403 |
| "evala env (Num n) = n" |
|
404 |
| "evalb env (Less a1 a2) = (evala env a1 < evala env a2)" |
|
405 |
| "evalb env (And b1 b2) = (evalb env b1 \<and> evalb env b2)" |
|
406 |
| "evalb env (Neg b) = (\<not> evalb env b)" |
|
407 |
||
58618 | 408 |
text \<open>Since the value of an expression depends on the value of its |
42912 | 409 |
variables, the functions @{const evala} and @{const evalb} take an |
410 |
additional parameter, an \emph{environment} that maps variables to |
|
411 |
their values. |
|
412 |
||
413 |
\medskip Substitution on expressions can be defined similarly. The |
|
414 |
mapping @{text f} of type @{typ "'a \<Rightarrow> 'a aexp"} given as a |
|
415 |
parameter is lifted canonically on the types @{typ "'a aexp"} and |
|
416 |
@{typ "'a bexp"}, respectively. |
|
58618 | 417 |
\<close> |
42912 | 418 |
|
419 |
primrec substa :: "('a \<Rightarrow> 'b aexp) \<Rightarrow> 'a aexp \<Rightarrow> 'b aexp" |
|
420 |
and substb :: "('a \<Rightarrow> 'b aexp) \<Rightarrow> 'a bexp \<Rightarrow> 'b bexp" |
|
421 |
where |
|
422 |
"substa f (IF b a1 a2) = IF (substb f b) (substa f a1) (substa f a2)" |
|
423 |
| "substa f (Sum a1 a2) = Sum (substa f a1) (substa f a2)" |
|
424 |
| "substa f (Diff a1 a2) = Diff (substa f a1) (substa f a2)" |
|
425 |
| "substa f (Var v) = f v" |
|
426 |
| "substa f (Num n) = Num n" |
|
427 |
| "substb f (Less a1 a2) = Less (substa f a1) (substa f a2)" |
|
428 |
| "substb f (And b1 b2) = And (substb f b1) (substb f b2)" |
|
429 |
| "substb f (Neg b) = Neg (substb f b)" |
|
430 |
||
58618 | 431 |
text \<open>In textbooks about semantics one often finds substitution |
42912 | 432 |
theorems, which express the relationship between substitution and |
433 |
evaluation. For @{typ "'a aexp"} and @{typ "'a bexp"}, we can prove |
|
434 |
such a theorem by mutual induction, followed by simplification. |
|
58618 | 435 |
\<close> |
42912 | 436 |
|
437 |
lemma subst_one: |
|
438 |
"evala env (substa (Var (v := a')) a) = evala (env (v := evala env a')) a" |
|
439 |
"evalb env (substb (Var (v := a')) b) = evalb (env (v := evala env a')) b" |
|
440 |
by (induct a and b) simp_all |
|
441 |
||
442 |
lemma subst_all: |
|
443 |
"evala env (substa s a) = evala (\<lambda>x. evala env (s x)) a" |
|
444 |
"evalb env (substb s b) = evalb (\<lambda>x. evala env (s x)) b" |
|
445 |
by (induct a and b) simp_all |
|
446 |
||
447 |
||
58618 | 448 |
subsubsection \<open>Example: a substitution function for terms\<close> |
449 |
||
450 |
text \<open>Functions on datatypes with nested recursion are also defined |
|
451 |
by mutual primitive recursion.\<close> |
|
42912 | 452 |
|
58310 | 453 |
datatype ('a, 'b) "term" = Var 'a | App 'b "('a, 'b) term list" |
42912 | 454 |
|
58618 | 455 |
text \<open>A substitution function on type @{typ "('a, 'b) term"} can be |
42912 | 456 |
defined as follows, by working simultaneously on @{typ "('a, 'b) |
58618 | 457 |
term list"}:\<close> |
42912 | 458 |
|
459 |
primrec subst_term :: "('a \<Rightarrow> ('a, 'b) term) \<Rightarrow> ('a, 'b) term \<Rightarrow> ('a, 'b) term" and |
|
460 |
subst_term_list :: "('a \<Rightarrow> ('a, 'b) term) \<Rightarrow> ('a, 'b) term list \<Rightarrow> ('a, 'b) term list" |
|
461 |
where |
|
462 |
"subst_term f (Var a) = f a" |
|
463 |
| "subst_term f (App b ts) = App b (subst_term_list f ts)" |
|
464 |
| "subst_term_list f [] = []" |
|
465 |
| "subst_term_list f (t # ts) = subst_term f t # subst_term_list f ts" |
|
466 |
||
58618 | 467 |
text \<open>The recursion scheme follows the structure of the unfolded |
42912 | 468 |
definition of type @{typ "('a, 'b) term"}. To prove properties of this |
469 |
substitution function, mutual induction is needed: |
|
58618 | 470 |
\<close> |
42912 | 471 |
|
472 |
lemma "subst_term (subst_term f1 \<circ> f2) t = subst_term f1 (subst_term f2 t)" and |
|
473 |
"subst_term_list (subst_term f1 \<circ> f2) ts = subst_term_list f1 (subst_term_list f2 ts)" |
|
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
474 |
by (induct t and ts rule: subst_term.induct subst_term_list.induct) simp_all |
42912 | 475 |
|
476 |
||
58618 | 477 |
subsubsection \<open>Example: a map function for infinitely branching trees\<close> |
478 |
||
479 |
text \<open>Defining functions on infinitely branching datatypes by |
|
42912 | 480 |
primitive recursion is just as easy. |
58618 | 481 |
\<close> |
42912 | 482 |
|
58310 | 483 |
datatype 'a tree = Atom 'a | Branch "nat \<Rightarrow> 'a tree" |
42912 | 484 |
|
485 |
primrec map_tree :: "('a \<Rightarrow> 'b) \<Rightarrow> 'a tree \<Rightarrow> 'b tree" |
|
486 |
where |
|
487 |
"map_tree f (Atom a) = Atom (f a)" |
|
488 |
| "map_tree f (Branch ts) = Branch (\<lambda>x. map_tree f (ts x))" |
|
489 |
||
58618 | 490 |
text \<open>Note that all occurrences of functions such as @{text ts} |
42912 | 491 |
above must be applied to an argument. In particular, @{term |
58618 | 492 |
"map_tree f \<circ> ts"} is not allowed here.\<close> |
493 |
||
494 |
text \<open>Here is a simple composition lemma for @{term map_tree}:\<close> |
|
42912 | 495 |
|
496 |
lemma "map_tree g (map_tree f t) = map_tree (g \<circ> f) t" |
|
497 |
by (induct t) simp_all |
|
498 |
||
42907
dfd4ef8e73f6
updated and re-unified HOL typedef, with some live examples;
wenzelm
parents:
42705
diff
changeset
|
499 |
|
58618 | 500 |
subsection \<open>Proof methods related to recursive definitions\<close> |
501 |
||
502 |
text \<open> |
|
26849 | 503 |
\begin{matharray}{rcl} |
42908 | 504 |
@{method_def (HOL) pat_completeness} & : & @{text method} \\ |
505 |
@{method_def (HOL) relation} & : & @{text method} \\ |
|
506 |
@{method_def (HOL) lexicographic_order} & : & @{text method} \\ |
|
507 |
@{method_def (HOL) size_change} & : & @{text method} \\ |
|
45944
e586f6d136b7
added some basic documentation about method induction_schema extracted from old NEWS
bulwahn
parents:
45943
diff
changeset
|
508 |
@{method_def (HOL) induction_schema} & : & @{text method} \\ |
26849 | 509 |
\end{matharray} |
510 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
511 |
@{rail \<open> |
42908 | 512 |
@@{method (HOL) relation} @{syntax term} |
513 |
; |
|
514 |
@@{method (HOL) lexicographic_order} (@{syntax clasimpmod} * ) |
|
515 |
; |
|
516 |
@@{method (HOL) size_change} ( orders (@{syntax clasimpmod} * ) ) |
|
517 |
; |
|
45944
e586f6d136b7
added some basic documentation about method induction_schema extracted from old NEWS
bulwahn
parents:
45943
diff
changeset
|
518 |
@@{method (HOL) induction_schema} |
e586f6d136b7
added some basic documentation about method induction_schema extracted from old NEWS
bulwahn
parents:
45943
diff
changeset
|
519 |
; |
42908 | 520 |
orders: ( 'max' | 'min' | 'ms' ) * |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
521 |
\<close>} |
42908 | 522 |
|
523 |
\begin{description} |
|
524 |
||
525 |
\item @{method (HOL) pat_completeness} is a specialized method to |
|
526 |
solve goals regarding the completeness of pattern matching, as |
|
527 |
required by the @{command (HOL) "function"} package (cf.\ |
|
58552 | 528 |
@{cite "isabelle-function"}). |
42908 | 529 |
|
530 |
\item @{method (HOL) relation}~@{text R} introduces a termination |
|
531 |
proof using the relation @{text R}. The resulting proof state will |
|
532 |
contain goals expressing that @{text R} is wellfounded, and that the |
|
533 |
arguments of recursive calls decrease with respect to @{text R}. |
|
534 |
Usually, this method is used as the initial proof step of manual |
|
535 |
termination proofs. |
|
536 |
||
537 |
\item @{method (HOL) "lexicographic_order"} attempts a fully |
|
538 |
automated termination proof by searching for a lexicographic |
|
539 |
combination of size measures on the arguments of the function. The |
|
540 |
method accepts the same arguments as the @{method auto} method, |
|
42930 | 541 |
which it uses internally to prove local descents. The @{syntax |
542 |
clasimpmod} modifiers are accepted (as for @{method auto}). |
|
42908 | 543 |
|
544 |
In case of failure, extensive information is printed, which can help |
|
58552 | 545 |
to analyse the situation (cf.\ @{cite "isabelle-function"}). |
42908 | 546 |
|
547 |
\item @{method (HOL) "size_change"} also works on termination goals, |
|
548 |
using a variation of the size-change principle, together with a |
|
58552 | 549 |
graph decomposition technique (see @{cite krauss_phd} for details). |
42908 | 550 |
Three kinds of orders are used internally: @{text max}, @{text min}, |
551 |
and @{text ms} (multiset), which is only available when the theory |
|
552 |
@{text Multiset} is loaded. When no order kinds are given, they are |
|
553 |
tried in order. The search for a termination proof uses SAT solving |
|
554 |
internally. |
|
555 |
||
42930 | 556 |
For local descent proofs, the @{syntax clasimpmod} modifiers are |
557 |
accepted (as for @{method auto}). |
|
42908 | 558 |
|
45944
e586f6d136b7
added some basic documentation about method induction_schema extracted from old NEWS
bulwahn
parents:
45943
diff
changeset
|
559 |
\item @{method (HOL) induction_schema} derives user-specified |
46283 | 560 |
induction rules from well-founded induction and completeness of |
561 |
patterns. This factors out some operations that are done internally |
|
562 |
by the function package and makes them available separately. See |
|
563 |
@{file "~~/src/HOL/ex/Induction_Schema.thy"} for examples. |
|
45944
e586f6d136b7
added some basic documentation about method induction_schema extracted from old NEWS
bulwahn
parents:
45943
diff
changeset
|
564 |
|
42908 | 565 |
\end{description} |
58618 | 566 |
\<close> |
567 |
||
568 |
||
569 |
subsection \<open>Functions with explicit partiality\<close> |
|
570 |
||
571 |
text \<open> |
|
42908 | 572 |
\begin{matharray}{rcl} |
573 |
@{command_def (HOL) "partial_function"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
|
574 |
@{attribute_def (HOL) "partial_function_mono"} & : & @{text attribute} \\ |
|
575 |
\end{matharray} |
|
576 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
577 |
@{rail \<open> |
42908 | 578 |
@@{command (HOL) partial_function} @{syntax target}? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
579 |
'(' @{syntax nameref} ')' @{syntax "fixes"} \<newline> |
42908 | 580 |
@'where' @{syntax thmdecl}? @{syntax prop} |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
581 |
\<close>} |
26849 | 582 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
583 |
\begin{description} |
42123 | 584 |
|
42908 | 585 |
\item @{command (HOL) "partial_function"}~@{text "(mode)"} defines |
586 |
recursive functions based on fixpoints in complete partial |
|
587 |
orders. No termination proof is required from the user or |
|
588 |
constructed internally. Instead, the possibility of non-termination |
|
589 |
is modelled explicitly in the result type, which contains an |
|
590 |
explicit bottom element. |
|
591 |
||
592 |
Pattern matching and mutual recursion are currently not supported. |
|
593 |
Thus, the specification consists of a single function described by a |
|
594 |
single recursive equation. |
|
595 |
||
596 |
There are no fixed syntactic restrictions on the body of the |
|
597 |
function, but the induced functional must be provably monotonic |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
598 |
wrt.\ the underlying order. The monotonicity proof is performed |
42908 | 599 |
internally, and the definition is rejected when it fails. The proof |
600 |
can be influenced by declaring hints using the |
|
601 |
@{attribute (HOL) partial_function_mono} attribute. |
|
602 |
||
603 |
The mandatory @{text mode} argument specifies the mode of operation |
|
604 |
of the command, which directly corresponds to a complete partial |
|
605 |
order on the result type. By default, the following modes are |
|
606 |
defined: |
|
26849 | 607 |
|
42908 | 608 |
\begin{description} |
46283 | 609 |
|
42908 | 610 |
\item @{text option} defines functions that map into the @{type |
611 |
option} type. Here, the value @{term None} is used to model a |
|
612 |
non-terminating computation. Monotonicity requires that if @{term |
|
46283 | 613 |
None} is returned by a recursive call, then the overall result must |
614 |
also be @{term None}. This is best achieved through the use of the |
|
615 |
monadic operator @{const "Option.bind"}. |
|
42908 | 616 |
|
617 |
\item @{text tailrec} defines functions with an arbitrary result |
|
618 |
type and uses the slightly degenerated partial order where @{term |
|
619 |
"undefined"} is the bottom element. Now, monotonicity requires that |
|
620 |
if @{term undefined} is returned by a recursive call, then the |
|
621 |
overall result must also be @{term undefined}. In practice, this is |
|
622 |
only satisfied when each recursive call is a tail call, whose result |
|
623 |
is directly returned. Thus, this mode of operation allows the |
|
624 |
definition of arbitrary tail-recursive functions. |
|
46283 | 625 |
|
42908 | 626 |
\end{description} |
627 |
||
628 |
Experienced users may define new modes by instantiating the locale |
|
629 |
@{const "partial_function_definitions"} appropriately. |
|
630 |
||
631 |
\item @{attribute (HOL) partial_function_mono} declares rules for |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
632 |
use in the internal monotonicity proofs of partial function |
42908 | 633 |
definitions. |
26849 | 634 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
635 |
\end{description} |
42908 | 636 |
|
58618 | 637 |
\<close> |
638 |
||
639 |
||
640 |
subsection \<open>Old-style recursive function definitions (TFL)\<close> |
|
641 |
||
642 |
text \<open> |
|
42908 | 643 |
\begin{matharray}{rcl} |
644 |
@{command_def (HOL) "recdef"} & : & @{text "theory \<rightarrow> theory)"} \\ |
|
645 |
@{command_def (HOL) "recdef_tc"}@{text "\<^sup>*"} & : & @{text "theory \<rightarrow> proof(prove)"} \\ |
|
646 |
\end{matharray} |
|
647 |
||
46280 | 648 |
The old TFL commands @{command (HOL) "recdef"} and @{command (HOL) |
649 |
"recdef_tc"} for defining recursive are mostly obsolete; @{command |
|
650 |
(HOL) "function"} or @{command (HOL) "fun"} should be used instead. |
|
651 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
652 |
@{rail \<open> |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
653 |
@@{command (HOL) recdef} ('(' @'permissive' ')')? \<newline> |
42908 | 654 |
@{syntax name} @{syntax term} (@{syntax prop} +) hints? |
655 |
; |
|
656 |
recdeftc @{syntax thmdecl}? tc |
|
657 |
; |
|
658 |
hints: '(' @'hints' ( recdefmod * ) ')' |
|
659 |
; |
|
660 |
recdefmod: (('recdef_simp' | 'recdef_cong' | 'recdef_wf') |
|
661 |
(() | 'add' | 'del') ':' @{syntax thmrefs}) | @{syntax clasimpmod} |
|
662 |
; |
|
663 |
tc: @{syntax nameref} ('(' @{syntax nat} ')')? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
664 |
\<close>} |
42908 | 665 |
|
666 |
\begin{description} |
|
667 |
||
668 |
\item @{command (HOL) "recdef"} defines general well-founded |
|
669 |
recursive functions (using the TFL package), see also |
|
58552 | 670 |
@{cite "isabelle-HOL"}. The ``@{text "(permissive)"}'' option tells |
42908 | 671 |
TFL to recover from failed proof attempts, returning unfinished |
672 |
results. The @{text recdef_simp}, @{text recdef_cong}, and @{text |
|
673 |
recdef_wf} hints refer to auxiliary rules to be used in the internal |
|
674 |
automated proof process of TFL. Additional @{syntax clasimpmod} |
|
42930 | 675 |
declarations may be given to tune the context of the Simplifier |
676 |
(cf.\ \secref{sec:simplifier}) and Classical reasoner (cf.\ |
|
677 |
\secref{sec:classical}). |
|
42908 | 678 |
|
679 |
\item @{command (HOL) "recdef_tc"}~@{text "c (i)"} recommences the |
|
680 |
proof for leftover termination condition number @{text i} (default |
|
681 |
1) as generated by a @{command (HOL) "recdef"} definition of |
|
682 |
constant @{text c}. |
|
683 |
||
684 |
Note that in most cases, @{command (HOL) "recdef"} is able to finish |
|
685 |
its internal proofs without manual intervention. |
|
686 |
||
687 |
\end{description} |
|
688 |
||
689 |
\medskip Hints for @{command (HOL) "recdef"} may be also declared |
|
690 |
globally, using the following attributes. |
|
691 |
||
692 |
\begin{matharray}{rcl} |
|
693 |
@{attribute_def (HOL) recdef_simp} & : & @{text attribute} \\ |
|
694 |
@{attribute_def (HOL) recdef_cong} & : & @{text attribute} \\ |
|
695 |
@{attribute_def (HOL) recdef_wf} & : & @{text attribute} \\ |
|
696 |
\end{matharray} |
|
697 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
698 |
@{rail \<open> |
42908 | 699 |
(@@{attribute (HOL) recdef_simp} | @@{attribute (HOL) recdef_cong} | |
700 |
@@{attribute (HOL) recdef_wf}) (() | 'add' | 'del') |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
701 |
\<close>} |
58618 | 702 |
\<close> |
703 |
||
704 |
||
705 |
section \<open>Old-style datatypes \label{sec:hol-datatype}\<close> |
|
706 |
||
707 |
text \<open> |
|
42908 | 708 |
\begin{matharray}{rcl} |
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
709 |
@{command_def (HOL) "old_datatype"} & : & @{text "theory \<rightarrow> theory"} \\ |
58306
117ba6cbe414
renamed 'rep_datatype' to 'old_rep_datatype' (HOL)
blanchet
parents:
58305
diff
changeset
|
710 |
@{command_def (HOL) "old_rep_datatype"} & : & @{text "theory \<rightarrow> proof(prove)"} \\ |
42908 | 711 |
\end{matharray} |
712 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
713 |
@{rail \<open> |
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
714 |
@@{command (HOL) old_datatype} (spec + @'and') |
42908 | 715 |
; |
58306
117ba6cbe414
renamed 'rep_datatype' to 'old_rep_datatype' (HOL)
blanchet
parents:
58305
diff
changeset
|
716 |
@@{command (HOL) old_rep_datatype} ('(' (@{syntax name} +) ')')? (@{syntax term} +) |
42908 | 717 |
; |
718 |
||
45839
43a5b86bc102
'datatype' specifications allow explicit sort constraints;
wenzelm
parents:
45768
diff
changeset
|
719 |
spec: @{syntax typespec_sorts} @{syntax mixfix}? '=' (cons + '|') |
42908 | 720 |
; |
721 |
cons: @{syntax name} (@{syntax type} * ) @{syntax mixfix}? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
722 |
\<close>} |
42908 | 723 |
|
724 |
\begin{description} |
|
725 |
||
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
726 |
\item @{command (HOL) "old_datatype"} defines old-style inductive |
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
727 |
datatypes in HOL. |
42908 | 728 |
|
58306
117ba6cbe414
renamed 'rep_datatype' to 'old_rep_datatype' (HOL)
blanchet
parents:
58305
diff
changeset
|
729 |
\item @{command (HOL) "old_rep_datatype"} represents existing types as |
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
730 |
old-style datatypes. |
42908 | 731 |
|
732 |
\end{description} |
|
733 |
||
58305
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
734 |
These commands are mostly obsolete; @{command (HOL) "datatype"} |
57752a91eec4
renamed 'datatype' to 'old_datatype'; 'datatype' is now alias for 'datatype_new'
blanchet
parents:
58100
diff
changeset
|
735 |
should be used instead. |
42908 | 736 |
|
58552 | 737 |
See @{cite "isabelle-HOL"} for more details on datatypes, but beware of |
42908 | 738 |
the old-style theory syntax being used there! Apart from proper |
739 |
proof methods for case-analysis and induction, there are also |
|
740 |
emulations of ML tactics @{method (HOL) case_tac} and @{method (HOL) |
|
741 |
induct_tac} available, see \secref{sec:hol-induct-tac}; these admit |
|
742 |
to refer directly to the internal structure of subgoals (including |
|
743 |
internally bound parameters). |
|
58618 | 744 |
\<close> |
745 |
||
746 |
||
747 |
subsubsection \<open>Examples\<close> |
|
748 |
||
749 |
text \<open>We define a type of finite sequences, with slightly different |
|
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
750 |
names than the existing @{typ "'a list"} that is already in @{theory |
58618 | 751 |
Main}:\<close> |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
752 |
|
58310 | 753 |
datatype 'a seq = Empty | Seq 'a "'a seq" |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
754 |
|
58618 | 755 |
text \<open>We can now prove some simple lemma by structural induction:\<close> |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
756 |
|
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
757 |
lemma "Seq x xs \<noteq> xs" |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
758 |
proof (induct xs arbitrary: x) |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
759 |
case Empty |
58618 | 760 |
txt \<open>This case can be proved using the simplifier: the freeness |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
761 |
properties of the datatype are already declared as @{attribute |
58618 | 762 |
simp} rules.\<close> |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
763 |
show "Seq x Empty \<noteq> Empty" |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
764 |
by simp |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
765 |
next |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
766 |
case (Seq y ys) |
58618 | 767 |
txt \<open>The step case is proved similarly.\<close> |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
768 |
show "Seq x (Seq y ys) \<noteq> Seq y ys" |
58618 | 769 |
using \<open>Seq y ys \<noteq> ys\<close> by simp |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
770 |
qed |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
771 |
|
58618 | 772 |
text \<open>Here is a more succinct version of the same proof:\<close> |
42910
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
773 |
|
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
774 |
lemma "Seq x xs \<noteq> xs" |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
775 |
by (induct xs arbitrary: x) simp_all |
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
776 |
|
6834af822a8b
updated and simplified HOL datatype examples (NB: special treatment of distinctness has been discontinued in the vicinity of 542b34b178ec);
wenzelm
parents:
42909
diff
changeset
|
777 |
|
58618 | 778 |
section \<open>Records \label{sec:hol-record}\<close> |
779 |
||
780 |
text \<open> |
|
26849 | 781 |
In principle, records merely generalize the concept of tuples, where |
782 |
components may be addressed by labels instead of just position. The |
|
783 |
logical infrastructure of records in Isabelle/HOL is slightly more |
|
784 |
advanced, though, supporting truly extensible record schemes. This |
|
785 |
admits operations that are polymorphic with respect to record |
|
786 |
extension, yielding ``object-oriented'' effects like (single) |
|
58552 | 787 |
inheritance. See also @{cite "NaraschewskiW-TPHOLs98"} for more |
26849 | 788 |
details on object-oriented verification and record subtyping in HOL. |
58618 | 789 |
\<close> |
790 |
||
791 |
||
792 |
subsection \<open>Basic concepts\<close> |
|
793 |
||
794 |
text \<open> |
|
26849 | 795 |
Isabelle/HOL supports both \emph{fixed} and \emph{schematic} records |
796 |
at the level of terms and types. The notation is as follows: |
|
797 |
||
798 |
\begin{center} |
|
799 |
\begin{tabular}{l|l|l} |
|
800 |
& record terms & record types \\ \hline |
|
801 |
fixed & @{text "\<lparr>x = a, y = b\<rparr>"} & @{text "\<lparr>x :: A, y :: B\<rparr>"} \\ |
|
802 |
schematic & @{text "\<lparr>x = a, y = b, \<dots> = m\<rparr>"} & |
|
803 |
@{text "\<lparr>x :: A, y :: B, \<dots> :: M\<rparr>"} \\ |
|
804 |
\end{tabular} |
|
805 |
\end{center} |
|
806 |
||
807 |
\noindent The ASCII representation of @{text "\<lparr>x = a\<rparr>"} is @{text |
|
808 |
"(| x = a |)"}. |
|
809 |
||
810 |
A fixed record @{text "\<lparr>x = a, y = b\<rparr>"} has field @{text x} of value |
|
811 |
@{text a} and field @{text y} of value @{text b}. The corresponding |
|
812 |
type is @{text "\<lparr>x :: A, y :: B\<rparr>"}, assuming that @{text "a :: A"} |
|
813 |
and @{text "b :: B"}. |
|
814 |
||
815 |
A record scheme like @{text "\<lparr>x = a, y = b, \<dots> = m\<rparr>"} contains fields |
|
816 |
@{text x} and @{text y} as before, but also possibly further fields |
|
817 |
as indicated by the ``@{text "\<dots>"}'' notation (which is actually part |
|
818 |
of the syntax). The improper field ``@{text "\<dots>"}'' of a record |
|
819 |
scheme is called the \emph{more part}. Logically it is just a free |
|
820 |
variable, which is occasionally referred to as ``row variable'' in |
|
821 |
the literature. The more part of a record scheme may be |
|
822 |
instantiated by zero or more further components. For example, the |
|
823 |
previous scheme may get instantiated to @{text "\<lparr>x = a, y = b, z = |
|
26852 | 824 |
c, \<dots> = m'\<rparr>"}, where @{text m'} refers to a different more part. |
26849 | 825 |
Fixed records are special instances of record schemes, where |
826 |
``@{text "\<dots>"}'' is properly terminated by the @{text "() :: unit"} |
|
827 |
element. In fact, @{text "\<lparr>x = a, y = b\<rparr>"} is just an abbreviation |
|
828 |
for @{text "\<lparr>x = a, y = b, \<dots> = ()\<rparr>"}. |
|
42123 | 829 |
|
26849 | 830 |
\medskip Two key observations make extensible records in a simply |
831 |
typed language like HOL work out: |
|
832 |
||
833 |
\begin{enumerate} |
|
834 |
||
835 |
\item the more part is internalized, as a free term or type |
|
836 |
variable, |
|
837 |
||
26852 | 838 |
\item field names are externalized, they cannot be accessed within |
839 |
the logic as first-class values. |
|
26849 | 840 |
|
841 |
\end{enumerate} |
|
842 |
||
843 |
\medskip In Isabelle/HOL record types have to be defined explicitly, |
|
844 |
fixing their field names and types, and their (optional) parent |
|
845 |
record. Afterwards, records may be formed using above syntax, while |
|
846 |
obeying the canonical order of fields as given by their declaration. |
|
847 |
The record package provides several standard operations like |
|
848 |
selectors and updates. The common setup for various generic proof |
|
849 |
tools enable succinct reasoning patterns. See also the Isabelle/HOL |
|
58552 | 850 |
tutorial @{cite "isabelle-hol-book"} for further instructions on using |
26849 | 851 |
records in practice. |
58618 | 852 |
\<close> |
853 |
||
854 |
||
855 |
subsection \<open>Record specifications\<close> |
|
856 |
||
857 |
text \<open> |
|
26849 | 858 |
\begin{matharray}{rcl} |
28761
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
859 |
@{command_def (HOL) "record"} & : & @{text "theory \<rightarrow> theory"} \\ |
26849 | 860 |
\end{matharray} |
861 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
862 |
@{rail \<open> |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
863 |
@@{command (HOL) record} @{syntax typespec_sorts} '=' \<newline> |
46494
ea2ae63336f3
clarified outer syntax "constdecl", which is only local to some rail diagrams;
wenzelm
parents:
46457
diff
changeset
|
864 |
(@{syntax type} '+')? (constdecl +) |
ea2ae63336f3
clarified outer syntax "constdecl", which is only local to some rail diagrams;
wenzelm
parents:
46457
diff
changeset
|
865 |
; |
ea2ae63336f3
clarified outer syntax "constdecl", which is only local to some rail diagrams;
wenzelm
parents:
46457
diff
changeset
|
866 |
constdecl: @{syntax name} '::' @{syntax type} @{syntax mixfix}? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
867 |
\<close>} |
26849 | 868 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
869 |
\begin{description} |
26849 | 870 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
871 |
\item @{command (HOL) "record"}~@{text "(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>m) t = \<tau> + c\<^sub>1 :: \<sigma>\<^sub>1 |
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
872 |
\<dots> c\<^sub>n :: \<sigma>\<^sub>n"} defines extensible record type @{text "(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>m) t"}, |
26849 | 873 |
derived from the optional parent record @{text "\<tau>"} by adding new |
874 |
field components @{text "c\<^sub>i :: \<sigma>\<^sub>i"} etc. |
|
875 |
||
876 |
The type variables of @{text "\<tau>"} and @{text "\<sigma>\<^sub>i"} need to be |
|
877 |
covered by the (distinct) parameters @{text "\<alpha>\<^sub>1, \<dots>, |
|
878 |
\<alpha>\<^sub>m"}. Type constructor @{text t} has to be new, while @{text |
|
879 |
\<tau>} needs to specify an instance of an existing record type. At |
|
880 |
least one new field @{text "c\<^sub>i"} has to be specified. |
|
881 |
Basically, field names need to belong to a unique record. This is |
|
882 |
not a real restriction in practice, since fields are qualified by |
|
883 |
the record name internally. |
|
884 |
||
885 |
The parent record specification @{text \<tau>} is optional; if omitted |
|
886 |
@{text t} becomes a root record. The hierarchy of all records |
|
887 |
declared within a theory context forms a forest structure, i.e.\ a |
|
888 |
set of trees starting with a root record each. There is no way to |
|
889 |
merge multiple parent records! |
|
890 |
||
891 |
For convenience, @{text "(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>m) t"} is made a |
|
892 |
type abbreviation for the fixed record type @{text "\<lparr>c\<^sub>1 :: |
|
893 |
\<sigma>\<^sub>1, \<dots>, c\<^sub>n :: \<sigma>\<^sub>n\<rparr>"}, likewise is @{text |
|
894 |
"(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>m, \<zeta>) t_scheme"} made an abbreviation for |
|
895 |
@{text "\<lparr>c\<^sub>1 :: \<sigma>\<^sub>1, \<dots>, c\<^sub>n :: \<sigma>\<^sub>n, \<dots> :: |
|
896 |
\<zeta>\<rparr>"}. |
|
897 |
||
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
898 |
\end{description} |
58618 | 899 |
\<close> |
900 |
||
901 |
||
902 |
subsection \<open>Record operations\<close> |
|
903 |
||
904 |
text \<open> |
|
26849 | 905 |
Any record definition of the form presented above produces certain |
906 |
standard operations. Selectors and updates are provided for any |
|
907 |
field, including the improper one ``@{text more}''. There are also |
|
908 |
cumulative record constructor functions. To simplify the |
|
909 |
presentation below, we assume for now that @{text "(\<alpha>\<^sub>1, \<dots>, |
|
910 |
\<alpha>\<^sub>m) t"} is a root record with fields @{text "c\<^sub>1 :: |
|
911 |
\<sigma>\<^sub>1, \<dots>, c\<^sub>n :: \<sigma>\<^sub>n"}. |
|
912 |
||
913 |
\medskip \textbf{Selectors} and \textbf{updates} are available for |
|
914 |
any field (including ``@{text more}''): |
|
915 |
||
916 |
\begin{matharray}{lll} |
|
26852 | 917 |
@{text "c\<^sub>i"} & @{text "::"} & @{text "\<lparr>\<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr> \<Rightarrow> \<sigma>\<^sub>i"} \\ |
918 |
@{text "c\<^sub>i_update"} & @{text "::"} & @{text "\<sigma>\<^sub>i \<Rightarrow> \<lparr>\<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr> \<Rightarrow> \<lparr>\<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr>"} \\ |
|
26849 | 919 |
\end{matharray} |
920 |
||
921 |
There is special syntax for application of updates: @{text "r\<lparr>x := |
|
922 |
a\<rparr>"} abbreviates term @{text "x_update a r"}. Further notation for |
|
923 |
repeated updates is also available: @{text "r\<lparr>x := a\<rparr>\<lparr>y := b\<rparr>\<lparr>z := |
|
924 |
c\<rparr>"} may be written @{text "r\<lparr>x := a, y := b, z := c\<rparr>"}. Note that |
|
925 |
because of postfix notation the order of fields shown here is |
|
926 |
reverse than in the actual term. Since repeated updates are just |
|
927 |
function applications, fields may be freely permuted in @{text "\<lparr>x |
|
928 |
:= a, y := b, z := c\<rparr>"}, as far as logical equality is concerned. |
|
929 |
Thus commutativity of independent updates can be proven within the |
|
930 |
logic for any two fields, but not as a general theorem. |
|
931 |
||
932 |
\medskip The \textbf{make} operation provides a cumulative record |
|
933 |
constructor function: |
|
934 |
||
935 |
\begin{matharray}{lll} |
|
26852 | 936 |
@{text "t.make"} & @{text "::"} & @{text "\<sigma>\<^sub>1 \<Rightarrow> \<dots> \<sigma>\<^sub>n \<Rightarrow> \<lparr>\<^vec>c :: \<^vec>\<sigma>\<rparr>"} \\ |
26849 | 937 |
\end{matharray} |
938 |
||
939 |
\medskip We now reconsider the case of non-root records, which are |
|
940 |
derived of some parent. In general, the latter may depend on |
|
941 |
another parent as well, resulting in a list of \emph{ancestor |
|
942 |
records}. Appending the lists of fields of all ancestors results in |
|
943 |
a certain field prefix. The record package automatically takes care |
|
944 |
of this by lifting operations over this context of ancestor fields. |
|
945 |
Assuming that @{text "(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>m) t"} has ancestor |
|
946 |
fields @{text "b\<^sub>1 :: \<rho>\<^sub>1, \<dots>, b\<^sub>k :: \<rho>\<^sub>k"}, |
|
947 |
the above record operations will get the following types: |
|
948 |
||
26852 | 949 |
\medskip |
950 |
\begin{tabular}{lll} |
|
951 |
@{text "c\<^sub>i"} & @{text "::"} & @{text "\<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr> \<Rightarrow> \<sigma>\<^sub>i"} \\ |
|
42123 | 952 |
@{text "c\<^sub>i_update"} & @{text "::"} & @{text "\<sigma>\<^sub>i \<Rightarrow> |
26852 | 953 |
\<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr> \<Rightarrow> |
954 |
\<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr>"} \\ |
|
955 |
@{text "t.make"} & @{text "::"} & @{text "\<rho>\<^sub>1 \<Rightarrow> \<dots> \<rho>\<^sub>k \<Rightarrow> \<sigma>\<^sub>1 \<Rightarrow> \<dots> \<sigma>\<^sub>n \<Rightarrow> |
|
956 |
\<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>\<rparr>"} \\ |
|
957 |
\end{tabular} |
|
958 |
\medskip |
|
26849 | 959 |
|
26852 | 960 |
\noindent Some further operations address the extension aspect of a |
26849 | 961 |
derived record scheme specifically: @{text "t.fields"} produces a |
962 |
record fragment consisting of exactly the new fields introduced here |
|
963 |
(the result may serve as a more part elsewhere); @{text "t.extend"} |
|
964 |
takes a fixed record and adds a given more part; @{text |
|
965 |
"t.truncate"} restricts a record scheme to a fixed record. |
|
966 |
||
26852 | 967 |
\medskip |
968 |
\begin{tabular}{lll} |
|
969 |
@{text "t.fields"} & @{text "::"} & @{text "\<sigma>\<^sub>1 \<Rightarrow> \<dots> \<sigma>\<^sub>n \<Rightarrow> \<lparr>\<^vec>c :: \<^vec>\<sigma>\<rparr>"} \\ |
|
970 |
@{text "t.extend"} & @{text "::"} & @{text "\<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>\<rparr> \<Rightarrow> |
|
971 |
\<zeta> \<Rightarrow> \<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr>"} \\ |
|
972 |
@{text "t.truncate"} & @{text "::"} & @{text "\<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>, \<dots> :: \<zeta>\<rparr> \<Rightarrow> \<lparr>\<^vec>b :: \<^vec>\<rho>, \<^vec>c :: \<^vec>\<sigma>\<rparr>"} \\ |
|
973 |
\end{tabular} |
|
974 |
\medskip |
|
26849 | 975 |
|
976 |
\noindent Note that @{text "t.make"} and @{text "t.fields"} coincide |
|
977 |
for root records. |
|
58618 | 978 |
\<close> |
979 |
||
980 |
||
981 |
subsection \<open>Derived rules and proof tools\<close> |
|
982 |
||
983 |
text \<open> |
|
26849 | 984 |
The record package proves several results internally, declaring |
985 |
these facts to appropriate proof tools. This enables users to |
|
986 |
reason about record structures quite conveniently. Assume that |
|
987 |
@{text t} is a record type as specified above. |
|
988 |
||
989 |
\begin{enumerate} |
|
42123 | 990 |
|
26849 | 991 |
\item Standard conversions for selectors or updates applied to |
992 |
record constructor terms are made part of the default Simplifier |
|
993 |
context; thus proofs by reduction of basic operations merely require |
|
994 |
the @{method simp} method without further arguments. These rules |
|
995 |
are available as @{text "t.simps"}, too. |
|
42123 | 996 |
|
26849 | 997 |
\item Selectors applied to updated records are automatically reduced |
998 |
by an internal simplification procedure, which is also part of the |
|
999 |
standard Simplifier setup. |
|
1000 |
||
1001 |
\item Inject equations of a form analogous to @{prop "(x, y) = (x', |
|
1002 |
y') \<equiv> x = x' \<and> y = y'"} are declared to the Simplifier and Classical |
|
1003 |
Reasoner as @{attribute iff} rules. These rules are available as |
|
1004 |
@{text "t.iffs"}. |
|
1005 |
||
1006 |
\item The introduction rule for record equality analogous to @{text |
|
1007 |
"x r = x r' \<Longrightarrow> y r = y r' \<dots> \<Longrightarrow> r = r'"} is declared to the Simplifier, |
|
1008 |
and as the basic rule context as ``@{attribute intro}@{text "?"}''. |
|
1009 |
The rule is called @{text "t.equality"}. |
|
1010 |
||
1011 |
\item Representations of arbitrary record expressions as canonical |
|
1012 |
constructor terms are provided both in @{method cases} and @{method |
|
1013 |
induct} format (cf.\ the generic proof methods of the same name, |
|
1014 |
\secref{sec:cases-induct}). Several variations are available, for |
|
1015 |
fixed records, record schemes, more parts etc. |
|
42123 | 1016 |
|
26849 | 1017 |
The generic proof methods are sufficiently smart to pick the most |
1018 |
sensible rule according to the type of the indicated record |
|
1019 |
expression: users just need to apply something like ``@{text "(cases |
|
1020 |
r)"}'' to a certain proof problem. |
|
1021 |
||
1022 |
\item The derived record operations @{text "t.make"}, @{text |
|
1023 |
"t.fields"}, @{text "t.extend"}, @{text "t.truncate"} are \emph{not} |
|
1024 |
treated automatically, but usually need to be expanded by hand, |
|
1025 |
using the collective fact @{text "t.defs"}. |
|
1026 |
||
1027 |
\end{enumerate} |
|
58618 | 1028 |
\<close> |
1029 |
||
1030 |
||
1031 |
subsubsection \<open>Examples\<close> |
|
1032 |
||
1033 |
text \<open>See @{file "~~/src/HOL/ex/Records.thy"}, for example.\<close> |
|
1034 |
||
1035 |
section \<open>Typedef axiomatization \label{sec:hol-typedef}\<close> |
|
1036 |
||
1037 |
text \<open> |
|
46280 | 1038 |
\begin{matharray}{rcl} |
1039 |
@{command_def (HOL) "typedef"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\ |
|
1040 |
\end{matharray} |
|
1041 |
||
1042 |
A Gordon/HOL-style type definition is a certain axiom scheme that |
|
1043 |
identifies a new type with a subset of an existing type. More |
|
42908 | 1044 |
precisely, the new type is defined by exhibiting an existing type |
1045 |
@{text \<tau>}, a set @{text "A :: \<tau> set"}, and a theorem that proves |
|
1046 |
@{prop "\<exists>x. x \<in> A"}. Thus @{text A} is a non-empty subset of @{text |
|
1047 |
\<tau>}, and the new type denotes this subset. New functions are |
|
1048 |
postulated that establish an isomorphism between the new type and |
|
1049 |
the subset. In general, the type @{text \<tau>} may involve type |
|
1050 |
variables @{text "\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>n"} which means that the type definition |
|
1051 |
produces a type constructor @{text "(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>n) t"} depending on |
|
1052 |
those type arguments. |
|
1053 |
||
57480
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1054 |
The axiomatization can be considered a ``definition'' in the sense of the |
58552 | 1055 |
particular set-theoretic interpretation of HOL @{cite pitts93}, where the |
57480
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1056 |
universe of types is required to be downwards-closed wrt.\ arbitrary |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1057 |
non-empty subsets. Thus genuinely new types introduced by @{command |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1058 |
"typedef"} stay within the range of HOL models by construction. |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1059 |
|
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1060 |
In contrast, the command @{command_ref type_synonym} from Isabelle/Pure |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1061 |
merely introduces syntactic abbreviations, without any logical |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1062 |
significance. Thus it is more faithful to the idea of a genuine type |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1063 |
definition, but less powerful in practice. |
47859 | 1064 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1065 |
@{rail \<open> |
49836
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1066 |
@@{command (HOL) typedef} abs_type '=' rep_set |
26849 | 1067 |
; |
42908 | 1068 |
abs_type: @{syntax typespec_sorts} @{syntax mixfix}? |
1069 |
; |
|
1070 |
rep_set: @{syntax term} (@'morphisms' @{syntax name} @{syntax name})? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1071 |
\<close>} |
26849 | 1072 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
1073 |
\begin{description} |
26849 | 1074 |
|
57480
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1075 |
\item @{command (HOL) "typedef"}~@{text "(\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>n) t = A"} produces an |
57487 | 1076 |
axiomatization (\secref{sec:axiomatizations}) for a type definition in the |
57480
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1077 |
background theory of the current context, depending on a non-emptiness |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1078 |
result of the set @{text A} that needs to be proven here. The set @{text |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1079 |
A} may contain type variables @{text "\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>n"} as specified on the |
d256f49b4799
clarified "axiomatization" -- minor rewording of this delicate concept;
wenzelm
parents:
56929
diff
changeset
|
1080 |
LHS, but no term variables. |
42908 | 1081 |
|
1082 |
Even though a local theory specification, the newly introduced type |
|
1083 |
constructor cannot depend on parameters or assumptions of the |
|
1084 |
context: this is structurally impossible in HOL. In contrast, the |
|
1085 |
non-emptiness proof may use local assumptions in unusual situations, |
|
1086 |
which could result in different interpretations in target contexts: |
|
1087 |
the meaning of the bijection between the representing set @{text A} |
|
1088 |
and the new type @{text t} may then change in different application |
|
1089 |
contexts. |
|
1090 |
||
49836
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1091 |
For @{command (HOL) "typedef"}~@{text "t = A"} the newly introduced |
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1092 |
type @{text t} is accompanied by a pair of morphisms to relate it to |
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1093 |
the representing set over the old type. By default, the injection |
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1094 |
from type to set is called @{text Rep_t} and its inverse @{text |
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1095 |
Abs_t}: An explicit @{keyword (HOL) "morphisms"} specification |
c13b39542972
simplified 'typedef' specifications: discontinued implicit set definition and alternative name;
wenzelm
parents:
49834
diff
changeset
|
1096 |
allows to provide alternative names. |
26849 | 1097 |
|
42908 | 1098 |
The core axiomatization uses the locale predicate @{const |
1099 |
type_definition} as defined in Isabelle/HOL. Various basic |
|
1100 |
consequences of that are instantiated accordingly, re-using the |
|
1101 |
locale facts with names derived from the new type constructor. Thus |
|
1102 |
the generic @{thm type_definition.Rep} is turned into the specific |
|
1103 |
@{text "Rep_t"}, for example. |
|
1104 |
||
1105 |
Theorems @{thm type_definition.Rep}, @{thm |
|
1106 |
type_definition.Rep_inverse}, and @{thm type_definition.Abs_inverse} |
|
1107 |
provide the most basic characterization as a corresponding |
|
1108 |
injection/surjection pair (in both directions). The derived rules |
|
1109 |
@{thm type_definition.Rep_inject} and @{thm |
|
1110 |
type_definition.Abs_inject} provide a more convenient version of |
|
1111 |
injectivity, suitable for automated proof tools (e.g.\ in |
|
1112 |
declarations involving @{attribute simp} or @{attribute iff}). |
|
1113 |
Furthermore, the rules @{thm type_definition.Rep_cases}~/ @{thm |
|
1114 |
type_definition.Rep_induct}, and @{thm type_definition.Abs_cases}~/ |
|
1115 |
@{thm type_definition.Abs_induct} provide alternative views on |
|
1116 |
surjectivity. These rules are already declared as set or type rules |
|
1117 |
for the generic @{method cases} and @{method induct} methods, |
|
1118 |
respectively. |
|
1119 |
||
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
1120 |
\end{description} |
58618 | 1121 |
\<close> |
1122 |
||
1123 |
subsubsection \<open>Examples\<close> |
|
1124 |
||
1125 |
text \<open>Type definitions permit the introduction of abstract data |
|
42908 | 1126 |
types in a safe way, namely by providing models based on already |
1127 |
existing types. Given some abstract axiomatic description @{text P} |
|
1128 |
of a type, this involves two steps: |
|
1129 |
||
1130 |
\begin{enumerate} |
|
1131 |
||
1132 |
\item Find an appropriate type @{text \<tau>} and subset @{text A} which |
|
1133 |
has the desired properties @{text P}, and make a type definition |
|
1134 |
based on this representation. |
|
1135 |
||
1136 |
\item Prove that @{text P} holds for @{text \<tau>} by lifting @{text P} |
|
1137 |
from the representation. |
|
26849 | 1138 |
|
42908 | 1139 |
\end{enumerate} |
1140 |
||
1141 |
You can later forget about the representation and work solely in |
|
1142 |
terms of the abstract properties @{text P}. |
|
1143 |
||
1144 |
\medskip The following trivial example pulls a three-element type |
|
58618 | 1145 |
into existence within the formal logical environment of HOL.\<close> |
42908 | 1146 |
|
49834 | 1147 |
typedef three = "{(True, True), (True, False), (False, True)}" |
42908 | 1148 |
by blast |
1149 |
||
1150 |
definition "One = Abs_three (True, True)" |
|
1151 |
definition "Two = Abs_three (True, False)" |
|
1152 |
definition "Three = Abs_three (False, True)" |
|
1153 |
||
1154 |
lemma three_distinct: "One \<noteq> Two" "One \<noteq> Three" "Two \<noteq> Three" |
|
49812
e3945ddcb9aa
eliminated some remaining uses of typedef with implicit set definition;
wenzelm
parents:
48985
diff
changeset
|
1155 |
by (simp_all add: One_def Two_def Three_def Abs_three_inject) |
42908 | 1156 |
|
1157 |
lemma three_cases: |
|
1158 |
fixes x :: three obtains "x = One" | "x = Two" | "x = Three" |
|
49812
e3945ddcb9aa
eliminated some remaining uses of typedef with implicit set definition;
wenzelm
parents:
48985
diff
changeset
|
1159 |
by (cases x) (auto simp: One_def Two_def Three_def Abs_three_inject) |
42908 | 1160 |
|
58618 | 1161 |
text \<open>Note that such trivial constructions are better done with |
1162 |
derived specification mechanisms such as @{command datatype}:\<close> |
|
58310 | 1163 |
|
1164 |
datatype three' = One' | Two' | Three' |
|
42908 | 1165 |
|
58618 | 1166 |
text \<open>This avoids re-doing basic definitions and proofs from the |
1167 |
primitive @{command typedef} above.\<close> |
|
1168 |
||
1169 |
||
1170 |
||
1171 |
section \<open>Functorial structure of types\<close> |
|
1172 |
||
1173 |
text \<open> |
|
41396 | 1174 |
\begin{matharray}{rcl} |
55467
a5c9002bc54d
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
blanchet
parents:
55372
diff
changeset
|
1175 |
@{command_def (HOL) "functor"} & : & @{text "local_theory \<rightarrow> proof(prove)"} |
41396 | 1176 |
\end{matharray} |
1177 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1178 |
@{rail \<open> |
55467
a5c9002bc54d
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
blanchet
parents:
55372
diff
changeset
|
1179 |
@@{command (HOL) functor} (@{syntax name} ':')? @{syntax term} |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1180 |
\<close>} |
41396 | 1181 |
|
1182 |
\begin{description} |
|
1183 |
||
55467
a5c9002bc54d
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
blanchet
parents:
55372
diff
changeset
|
1184 |
\item @{command (HOL) "functor"}~@{text "prefix: m"} allows to |
42617 | 1185 |
prove and register properties about the functorial structure of type |
1186 |
constructors. These properties then can be used by other packages |
|
1187 |
to deal with those type constructors in certain type constructions. |
|
1188 |
Characteristic theorems are noted in the current local theory. By |
|
1189 |
default, they are prefixed with the base name of the type |
|
1190 |
constructor, an explicit prefix can be given alternatively. |
|
41396 | 1191 |
|
1192 |
The given term @{text "m"} is considered as \emph{mapper} for the |
|
1193 |
corresponding type constructor and must conform to the following |
|
1194 |
type pattern: |
|
1195 |
||
1196 |
\begin{matharray}{lll} |
|
1197 |
@{text "m"} & @{text "::"} & |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1198 |
@{text "\<sigma>\<^sub>1 \<Rightarrow> \<dots> \<sigma>\<^sub>k \<Rightarrow> (\<^vec>\<alpha>\<^sub>n) t \<Rightarrow> (\<^vec>\<beta>\<^sub>n) t"} \\ |
41396 | 1199 |
\end{matharray} |
1200 |
||
1201 |
\noindent where @{text t} is the type constructor, @{text |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1202 |
"\<^vec>\<alpha>\<^sub>n"} and @{text "\<^vec>\<beta>\<^sub>n"} are distinct |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1203 |
type variables free in the local theory and @{text "\<sigma>\<^sub>1"}, |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1204 |
\ldots, @{text "\<sigma>\<^sub>k"} is a subsequence of @{text "\<alpha>\<^sub>1 \<Rightarrow> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1205 |
\<beta>\<^sub>1"}, @{text "\<beta>\<^sub>1 \<Rightarrow> \<alpha>\<^sub>1"}, \ldots, |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1206 |
@{text "\<alpha>\<^sub>n \<Rightarrow> \<beta>\<^sub>n"}, @{text "\<beta>\<^sub>n \<Rightarrow> |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1207 |
\<alpha>\<^sub>n"}. |
41396 | 1208 |
|
1209 |
\end{description} |
|
58618 | 1210 |
\<close> |
1211 |
||
1212 |
||
1213 |
section \<open>Quotient types\<close> |
|
1214 |
||
1215 |
text \<open> |
|
50109 | 1216 |
\begin{matharray}{rcl} |
1217 |
@{command_def (HOL) "quotient_type"} & : & @{text "local_theory \<rightarrow> proof(prove)"}\\ |
|
1218 |
@{command_def (HOL) "quotient_definition"} & : & @{text "local_theory \<rightarrow> proof(prove)"}\\ |
|
1219 |
@{command_def (HOL) "print_quotmapsQ3"} & : & @{text "context \<rightarrow>"}\\ |
|
1220 |
@{command_def (HOL) "print_quotientsQ3"} & : & @{text "context \<rightarrow>"}\\ |
|
1221 |
@{command_def (HOL) "print_quotconsts"} & : & @{text "context \<rightarrow>"}\\ |
|
1222 |
@{method_def (HOL) "lifting"} & : & @{text method} \\ |
|
1223 |
@{method_def (HOL) "lifting_setup"} & : & @{text method} \\ |
|
1224 |
@{method_def (HOL) "descending"} & : & @{text method} \\ |
|
1225 |
@{method_def (HOL) "descending_setup"} & : & @{text method} \\ |
|
1226 |
@{method_def (HOL) "partiality_descending"} & : & @{text method} \\ |
|
1227 |
@{method_def (HOL) "partiality_descending_setup"} & : & @{text method} \\ |
|
1228 |
@{method_def (HOL) "regularize"} & : & @{text method} \\ |
|
1229 |
@{method_def (HOL) "injection"} & : & @{text method} \\ |
|
1230 |
@{method_def (HOL) "cleaning"} & : & @{text method} \\ |
|
1231 |
@{attribute_def (HOL) "quot_thm"} & : & @{text attribute} \\ |
|
1232 |
@{attribute_def (HOL) "quot_lifted"} & : & @{text attribute} \\ |
|
1233 |
@{attribute_def (HOL) "quot_respect"} & : & @{text attribute} \\ |
|
1234 |
@{attribute_def (HOL) "quot_preserve"} & : & @{text attribute} \\ |
|
1235 |
\end{matharray} |
|
1236 |
||
1237 |
The quotient package defines a new quotient type given a raw type |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1238 |
and a partial equivalence relation. The package also historically |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1239 |
includes automation for transporting definitions and theorems. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1240 |
But most of this automation was superseded by the Lifting and Transfer |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1241 |
packages. The user should consider using these two new packages for |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1242 |
lifting definitions and transporting theorems. |
50109 | 1243 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1244 |
@{rail \<open> |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1245 |
@@{command (HOL) quotient_type} (spec) |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1246 |
; |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
1247 |
spec: @{syntax typespec} @{syntax mixfix}? '=' \<newline> |
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
1248 |
@{syntax type} '/' ('partial' ':')? @{syntax term} \<newline> |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1249 |
(@'morphisms' @{syntax name} @{syntax name})? (@'parametric' @{syntax thmref})? |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1250 |
\<close>} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1251 |
|
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1252 |
@{rail \<open> |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
1253 |
@@{command (HOL) quotient_definition} constdecl? @{syntax thmdecl}? \<newline> |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1254 |
@{syntax term} 'is' @{syntax term} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1255 |
; |
50109 | 1256 |
constdecl: @{syntax name} ('::' @{syntax type})? @{syntax mixfix}? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1257 |
\<close>} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1258 |
|
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1259 |
@{rail \<open> |
50109 | 1260 |
@@{method (HOL) lifting} @{syntax thmrefs}? |
1261 |
; |
|
1262 |
@@{method (HOL) lifting_setup} @{syntax thmrefs}? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1263 |
\<close>} |
50109 | 1264 |
|
1265 |
\begin{description} |
|
1266 |
||
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1267 |
\item @{command (HOL) "quotient_type"} defines a new quotient type @{text \<tau>}. The |
50109 | 1268 |
injection from a quotient type to a raw type is called @{text |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1269 |
rep_\<tau>}, its inverse @{text abs_\<tau>} unless explicit @{keyword (HOL) |
50109 | 1270 |
"morphisms"} specification provides alternative names. @{command |
1271 |
(HOL) "quotient_type"} requires the user to prove that the relation |
|
1272 |
is an equivalence relation (predicate @{text equivp}), unless the |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1273 |
user specifies explicitly @{text partial} in which case the |
50109 | 1274 |
obligation is @{text part_equivp}. A quotient defined with @{text |
1275 |
partial} is weaker in the sense that less things can be proved |
|
1276 |
automatically. |
|
1277 |
||
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1278 |
The command internally proves a Quotient theorem and sets up the Lifting |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1279 |
package by the command @{command (HOL) setup_lifting}. Thus the Lifting |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1280 |
and Transfer packages can be used also with quotient types defined by |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1281 |
@{command (HOL) "quotient_type"} without any extra set-up. The parametricity |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1282 |
theorem for the equivalence relation R can be provided as an extra argument |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1283 |
of the command and is passed to the corresponding internal call of @{command (HOL) setup_lifting}. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1284 |
This theorem allows the Lifting package to generate a stronger transfer rule for equality. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1285 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1286 |
\end{description} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1287 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1288 |
The most of the rest of the package was superseded by the Lifting and Transfer |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1289 |
packages. The user should consider using these two new packages for |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1290 |
lifting definitions and transporting theorems. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1291 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1292 |
\begin{description} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1293 |
|
50109 | 1294 |
\item @{command (HOL) "quotient_definition"} defines a constant on |
1295 |
the quotient type. |
|
1296 |
||
1297 |
\item @{command (HOL) "print_quotmapsQ3"} prints quotient map |
|
1298 |
functions. |
|
1299 |
||
1300 |
\item @{command (HOL) "print_quotientsQ3"} prints quotients. |
|
1301 |
||
1302 |
\item @{command (HOL) "print_quotconsts"} prints quotient constants. |
|
1303 |
||
1304 |
\item @{method (HOL) "lifting"} and @{method (HOL) "lifting_setup"} |
|
1305 |
methods match the current goal with the given raw theorem to be |
|
1306 |
lifted producing three new subgoals: regularization, injection and |
|
1307 |
cleaning subgoals. @{method (HOL) "lifting"} tries to apply the |
|
1308 |
heuristics for automatically solving these three subgoals and |
|
1309 |
leaves only the subgoals unsolved by the heuristics to the user as |
|
1310 |
opposed to @{method (HOL) "lifting_setup"} which leaves the three |
|
1311 |
subgoals unsolved. |
|
1312 |
||
1313 |
\item @{method (HOL) "descending"} and @{method (HOL) |
|
1314 |
"descending_setup"} try to guess a raw statement that would lift |
|
1315 |
to the current subgoal. Such statement is assumed as a new subgoal |
|
1316 |
and @{method (HOL) "descending"} continues in the same way as |
|
1317 |
@{method (HOL) "lifting"} does. @{method (HOL) "descending"} tries |
|
1318 |
to solve the arising regularization, injection and cleaning |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1319 |
subgoals with the analogous method @{method (HOL) |
50109 | 1320 |
"descending_setup"} which leaves the four unsolved subgoals. |
1321 |
||
1322 |
\item @{method (HOL) "partiality_descending"} finds the regularized |
|
1323 |
theorem that would lift to the current subgoal, lifts it and |
|
1324 |
leaves as a subgoal. This method can be used with partial |
|
1325 |
equivalence quotients where the non regularized statements would |
|
1326 |
not be true. @{method (HOL) "partiality_descending_setup"} leaves |
|
1327 |
the injection and cleaning subgoals unchanged. |
|
1328 |
||
1329 |
\item @{method (HOL) "regularize"} applies the regularization |
|
1330 |
heuristics to the current subgoal. |
|
1331 |
||
1332 |
\item @{method (HOL) "injection"} applies the injection heuristics |
|
1333 |
to the current goal using the stored quotient respectfulness |
|
1334 |
theorems. |
|
1335 |
||
1336 |
\item @{method (HOL) "cleaning"} applies the injection cleaning |
|
1337 |
heuristics to the current subgoal using the stored quotient |
|
1338 |
preservation theorems. |
|
1339 |
||
1340 |
\item @{attribute (HOL) quot_lifted} attribute tries to |
|
1341 |
automatically transport the theorem to the quotient type. |
|
1342 |
The attribute uses all the defined quotients types and quotient |
|
1343 |
constants often producing undesired results or theorems that |
|
1344 |
cannot be lifted. |
|
1345 |
||
1346 |
\item @{attribute (HOL) quot_respect} and @{attribute (HOL) |
|
1347 |
quot_preserve} attributes declare a theorem as a respectfulness |
|
1348 |
and preservation theorem respectively. These are stored in the |
|
1349 |
local theory store and used by the @{method (HOL) "injection"} |
|
1350 |
and @{method (HOL) "cleaning"} methods respectively. |
|
1351 |
||
1352 |
\item @{attribute (HOL) quot_thm} declares that a certain theorem |
|
1353 |
is a quotient extension theorem. Quotient extension theorems |
|
1354 |
allow for quotienting inside container types. Given a polymorphic |
|
1355 |
type that serves as a container, a map function defined for this |
|
55467
a5c9002bc54d
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
blanchet
parents:
55372
diff
changeset
|
1356 |
container using @{command (HOL) "functor"} and a relation |
50109 | 1357 |
map defined for for the container type, the quotient extension |
1358 |
theorem should be @{term "Quotient3 R Abs Rep \<Longrightarrow> Quotient3 |
|
1359 |
(rel_map R) (map Abs) (map Rep)"}. Quotient extension theorems |
|
1360 |
are stored in a database and are used all the steps of lifting |
|
1361 |
theorems. |
|
1362 |
||
1363 |
\end{description} |
|
58618 | 1364 |
\<close> |
1365 |
||
1366 |
||
1367 |
section \<open>Definition by specification \label{sec:hol-specification}\<close> |
|
1368 |
||
1369 |
text \<open> |
|
50109 | 1370 |
\begin{matharray}{rcl} |
1371 |
@{command_def (HOL) "specification"} & : & @{text "theory \<rightarrow> proof(prove)"} \\ |
|
1372 |
\end{matharray} |
|
1373 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1374 |
@{rail \<open> |
56270
ce9c7a527c4b
removed unused 'ax_specification', to give 'specification' a chance to become localized;
wenzelm
parents:
55944
diff
changeset
|
1375 |
@@{command (HOL) specification} '(' (decl +) ')' \<newline> |
ce9c7a527c4b
removed unused 'ax_specification', to give 'specification' a chance to become localized;
wenzelm
parents:
55944
diff
changeset
|
1376 |
(@{syntax thmdecl}? @{syntax prop} +) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1377 |
; |
56270
ce9c7a527c4b
removed unused 'ax_specification', to give 'specification' a chance to become localized;
wenzelm
parents:
55944
diff
changeset
|
1378 |
decl: (@{syntax name} ':')? @{syntax term} ('(' @'overloaded' ')')? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1379 |
\<close>} |
50109 | 1380 |
|
1381 |
\begin{description} |
|
1382 |
||
1383 |
\item @{command (HOL) "specification"}~@{text "decls \<phi>"} sets up a |
|
1384 |
goal stating the existence of terms with the properties specified to |
|
1385 |
hold for the constants given in @{text decls}. After finishing the |
|
1386 |
proof, the theory will be augmented with definitions for the given |
|
1387 |
constants, as well as with theorems stating the properties for these |
|
1388 |
constants. |
|
1389 |
||
56270
ce9c7a527c4b
removed unused 'ax_specification', to give 'specification' a chance to become localized;
wenzelm
parents:
55944
diff
changeset
|
1390 |
@{text decl} declares a constant to be defined by the |
50109 | 1391 |
specification given. The definition for the constant @{text c} is |
1392 |
bound to the name @{text c_def} unless a theorem name is given in |
|
1393 |
the declaration. Overloaded constants should be declared as such. |
|
1394 |
||
1395 |
\end{description} |
|
58618 | 1396 |
\<close> |
1397 |
||
1398 |
||
1399 |
section \<open>Adhoc overloading of constants\<close> |
|
1400 |
||
1401 |
text \<open> |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1402 |
\begin{tabular}{rcll} |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1403 |
@{command_def "adhoc_overloading"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1404 |
@{command_def "no_adhoc_overloading"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1405 |
@{attribute_def "show_variants"} & : & @{text "attribute"} & default @{text false} \\ |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1406 |
\end{tabular} |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1407 |
|
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1408 |
\medskip |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1409 |
|
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1410 |
Adhoc overloading allows to overload a constant depending on |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1411 |
its type. Typically this involves the introduction of an |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1412 |
uninterpreted constant (used for input and output) and the addition |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1413 |
of some variants (used internally). For examples see |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1414 |
@{file "~~/src/HOL/ex/Adhoc_Overloading_Examples.thy"} and |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1415 |
@{file "~~/src/HOL/Library/Monad_Syntax.thy"}. |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1416 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1417 |
@{rail \<open> |
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1418 |
(@@{command adhoc_overloading} | @@{command no_adhoc_overloading}) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1419 |
(@{syntax nameref} (@{syntax term} + ) + @'and') |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1420 |
\<close>} |
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1421 |
|
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1422 |
\begin{description} |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1423 |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1424 |
\item @{command "adhoc_overloading"}~@{text "c v\<^sub>1 ... v\<^sub>n"} |
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1425 |
associates variants with an existing constant. |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1426 |
|
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1427 |
\item @{command "no_adhoc_overloading"} is similar to |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1428 |
@{command "adhoc_overloading"}, but removes the specified variants |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1429 |
from the present context. |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1430 |
|
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1431 |
\item @{attribute "show_variants"} controls printing of variants |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1432 |
of overloaded constants. If enabled, the internally used variants |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1433 |
are printed instead of their respective overloaded constants. This |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1434 |
is occasionally useful to check whether the system agrees with a |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1435 |
user's expectations about derived variants. |
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1436 |
|
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
1437 |
\end{description} |
58618 | 1438 |
\<close> |
1439 |
||
1440 |
||
1441 |
chapter \<open>Proof tools\<close> |
|
1442 |
||
1443 |
section \<open>Adhoc tuples\<close> |
|
1444 |
||
1445 |
text \<open> |
|
50109 | 1446 |
\begin{matharray}{rcl} |
1447 |
@{attribute_def (HOL) split_format}@{text "\<^sup>*"} & : & @{text attribute} \\ |
|
1448 |
\end{matharray} |
|
1449 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1450 |
@{rail \<open> |
50109 | 1451 |
@@{attribute (HOL) split_format} ('(' 'complete' ')')? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1452 |
\<close>} |
50109 | 1453 |
|
1454 |
\begin{description} |
|
1455 |
||
1456 |
\item @{attribute (HOL) split_format}\ @{text "(complete)"} causes |
|
1457 |
arguments in function applications to be represented canonically |
|
1458 |
according to their tuple type structure. |
|
1459 |
||
1460 |
Note that this operation tends to invent funny names for new local |
|
1461 |
parameters introduced. |
|
1462 |
||
1463 |
\end{description} |
|
58618 | 1464 |
\<close> |
1465 |
||
1466 |
||
1467 |
section \<open>Transfer package\<close> |
|
1468 |
||
1469 |
text \<open> |
|
47821 | 1470 |
\begin{matharray}{rcl} |
1471 |
@{method_def (HOL) "transfer"} & : & @{text method} \\ |
|
1472 |
@{method_def (HOL) "transfer'"} & : & @{text method} \\ |
|
1473 |
@{method_def (HOL) "transfer_prover"} & : & @{text method} \\ |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1474 |
@{attribute_def (HOL) "Transfer.transferred"} & : & @{text attribute} \\ |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1475 |
@{attribute_def (HOL) "untransferred"} & : & @{text attribute} \\ |
47821 | 1476 |
@{attribute_def (HOL) "transfer_rule"} & : & @{text attribute} \\ |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1477 |
@{attribute_def (HOL) "transfer_domain_rule"} & : & @{text attribute} \\ |
47821 | 1478 |
@{attribute_def (HOL) "relator_eq"} & : & @{text attribute} \\ |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1479 |
@{attribute_def (HOL) "relator_domain"} & : & @{text attribute} \\ |
47821 | 1480 |
\end{matharray} |
1481 |
||
1482 |
\begin{description} |
|
1483 |
||
1484 |
\item @{method (HOL) "transfer"} method replaces the current subgoal |
|
1485 |
with a logically equivalent one that uses different types and |
|
1486 |
constants. The replacement of types and constants is guided by the |
|
1487 |
database of transfer rules. Goals are generalized over all free |
|
1488 |
variables by default; this is necessary for variables whose types |
|
1489 |
change, but can be overridden for specific variables with e.g. |
|
1490 |
@{text "transfer fixing: x y z"}. |
|
1491 |
||
1492 |
\item @{method (HOL) "transfer'"} is a variant of @{method (HOL) |
|
1493 |
transfer} that allows replacing a subgoal with one that is |
|
1494 |
logically stronger (rather than equivalent). For example, a |
|
1495 |
subgoal involving equality on a quotient type could be replaced |
|
1496 |
with a subgoal involving equality (instead of the corresponding |
|
1497 |
equivalence relation) on the underlying raw type. |
|
1498 |
||
1499 |
\item @{method (HOL) "transfer_prover"} method assists with proving |
|
1500 |
a transfer rule for a new constant, provided the constant is |
|
1501 |
defined in terms of other constants that already have transfer |
|
1502 |
rules. It should be applied after unfolding the constant |
|
1503 |
definitions. |
|
1504 |
||
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1505 |
\item @{attribute (HOL) "untransferred"} proves the same equivalent theorem |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1506 |
as @{method (HOL) "transfer"} internally does. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1507 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1508 |
\item @{attribute (HOL) Transfer.transferred} works in the opposite |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1509 |
direction than @{method (HOL) "transfer'"}. E.g., given the transfer |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1510 |
relation @{text "ZN x n \<equiv> (x = int n)"}, corresponding transfer rules and the theorem |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1511 |
@{text "\<forall>x::int \<in> {0..}. x < x + 1"}, the attribute would prove |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1512 |
@{text "\<forall>n::nat. n < n + 1"}. The attribute is still in experimental |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1513 |
phase of development. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1514 |
|
47821 | 1515 |
\item @{attribute (HOL) "transfer_rule"} attribute maintains a |
1516 |
collection of transfer rules, which relate constants at two |
|
1517 |
different types. Typical transfer rules may relate different type |
|
1518 |
instances of the same polymorphic constant, or they may relate an |
|
1519 |
operation on a raw type to a corresponding operation on an |
|
1520 |
abstract type (quotient or subtype). For example: |
|
1521 |
||
1522 |
@{text "((A ===> B) ===> list_all2 A ===> list_all2 B) map map"}\\ |
|
1523 |
@{text "(cr_int ===> cr_int ===> cr_int) (\<lambda>(x,y) (u,v). (x+u, y+v)) plus"} |
|
1524 |
||
1525 |
Lemmas involving predicates on relations can also be registered |
|
1526 |
using the same attribute. For example: |
|
1527 |
||
1528 |
@{text "bi_unique A \<Longrightarrow> (list_all2 A ===> op =) distinct distinct"}\\ |
|
55944 | 1529 |
@{text "\<lbrakk>bi_unique A; bi_unique B\<rbrakk> \<Longrightarrow> bi_unique (rel_prod A B)"} |
47821 | 1530 |
|
57829 | 1531 |
Preservation of predicates on relations (@{text "bi_unique, bi_total, |
1532 |
right_unique, right_total, left_unique, left_total"}) with the respect to a relator |
|
58552 | 1533 |
is proved automatically if the involved type is BNF |
1534 |
@{cite "isabelle-datatypes"} without dead variables. |
|
57829 | 1535 |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1536 |
\item @{attribute (HOL) "transfer_domain_rule"} attribute maintains a collection |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1537 |
of rules, which specify a domain of a transfer relation by a predicate. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1538 |
E.g., given the transfer relation @{text "ZN x n \<equiv> (x = int n)"}, |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1539 |
one can register the following transfer domain rule: |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1540 |
@{text "Domainp ZN = (\<lambda>x. x \<ge> 0)"}. The rules allow the package to produce |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1541 |
more readable transferred goals, e.g., when quantifiers are transferred. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1542 |
|
47821 | 1543 |
\item @{attribute (HOL) relator_eq} attribute collects identity laws |
57829 | 1544 |
for relators of various type constructors, e.g. @{term "rel_set |
47821 | 1545 |
(op =) = (op =)"}. The @{method (HOL) transfer} method uses these |
1546 |
lemmas to infer transfer rules for non-polymorphic constants on |
|
57829 | 1547 |
the fly. For examples see @{file |
1548 |
"~~/src/HOL/Lifting_Set.thy"} or @{file "~~/src/HOL/Lifting.thy"}. |
|
1549 |
This property is proved automatically if the involved type is BNF without dead variables. |
|
47821 | 1550 |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1551 |
\item @{attribute_def (HOL) "relator_domain"} attribute collects rules |
57829 | 1552 |
describing domains of relators by predicators. E.g., |
1553 |
@{term "Domainp (rel_set T) = (\<lambda>A. Ball A (Domainp T))"}. This allows the package |
|
1554 |
to lift transfer domain rules through type constructors. For examples see @{file |
|
1555 |
"~~/src/HOL/Lifting_Set.thy"} or @{file "~~/src/HOL/Lifting.thy"}. |
|
1556 |
This property is proved automatically if the involved type is BNF without dead variables. |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1557 |
|
47821 | 1558 |
\end{description} |
1559 |
||
58552 | 1560 |
Theoretical background can be found in @{cite "Huffman-Kuncar:2013:lifting_transfer"}. |
58618 | 1561 |
\<close> |
1562 |
||
1563 |
||
1564 |
section \<open>Lifting package\<close> |
|
1565 |
||
1566 |
text \<open> |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1567 |
The Lifting package allows users to lift terms of the raw type to the abstract type, which is |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1568 |
a necessary step in building a library for an abstract type. Lifting defines a new constant |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1569 |
by combining coercion functions (Abs and Rep) with the raw term. It also proves an appropriate |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1570 |
transfer rule for the Transfer package and, if possible, an equation for the code generator. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1571 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1572 |
The Lifting package provides two main commands: @{command (HOL) "setup_lifting"} for initializing |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1573 |
the package to work with a new type, and @{command (HOL) "lift_definition"} for lifting constants. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1574 |
The Lifting package works with all four kinds of type abstraction: type copies, subtypes, |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1575 |
total quotients and partial quotients. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1576 |
|
58552 | 1577 |
Theoretical background can be found in @{cite "Huffman-Kuncar:2013:lifting_transfer"}. |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1578 |
|
47802 | 1579 |
\begin{matharray}{rcl} |
1580 |
@{command_def (HOL) "setup_lifting"} & : & @{text "local_theory \<rightarrow> local_theory"}\\ |
|
1581 |
@{command_def (HOL) "lift_definition"} & : & @{text "local_theory \<rightarrow> proof(prove)"}\\ |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1582 |
@{command_def (HOL) "lifting_forget"} & : & @{text "local_theory \<rightarrow> local_theory"}\\ |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1583 |
@{command_def (HOL) "lifting_update"} & : & @{text "local_theory \<rightarrow> local_theory"}\\ |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
53015
diff
changeset
|
1584 |
@{command_def (HOL) "print_quot_maps"} & : & @{text "context \<rightarrow>"}\\ |
47802 | 1585 |
@{command_def (HOL) "print_quotients"} & : & @{text "context \<rightarrow>"}\\ |
1586 |
@{attribute_def (HOL) "quot_map"} & : & @{text attribute} \\ |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
1587 |
@{attribute_def (HOL) "relator_eq_onp"} & : & @{text attribute} \\ |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1588 |
@{attribute_def (HOL) "relator_mono"} & : & @{text attribute} \\ |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1589 |
@{attribute_def (HOL) "relator_distr"} & : & @{text attribute} \\ |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1590 |
@{attribute_def (HOL) "quot_del"} & : & @{text attribute} \\ |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1591 |
@{attribute_def (HOL) "lifting_restore"} & : & @{text attribute} \\ |
47802 | 1592 |
\end{matharray} |
1593 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1594 |
@{rail \<open> |
59487
adaa430fc0f7
default abstypes and default abstract equations make technical (no_code) annotation superfluous
haftmann
parents:
58618
diff
changeset
|
1595 |
@@{command (HOL) setup_lifting} \<newline> |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1596 |
@{syntax thmref} @{syntax thmref}? (@'parametric' @{syntax thmref})?; |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1597 |
\<close>} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1598 |
|
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1599 |
@{rail \<open> |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
1600 |
@@{command (HOL) lift_definition} @{syntax name} '::' @{syntax type} @{syntax mixfix}? \<newline> |
57829 | 1601 |
'is' @{syntax term} (@'parametric' (@{syntax thmref}+))?; |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1602 |
\<close>} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1603 |
|
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1604 |
@{rail \<open> |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1605 |
@@{command (HOL) lifting_forget} @{syntax nameref}; |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1606 |
\<close>} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1607 |
|
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1608 |
@{rail \<open> |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1609 |
@@{command (HOL) lifting_update} @{syntax nameref}; |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1610 |
\<close>} |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1611 |
|
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1612 |
@{rail \<open> |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1613 |
@@{attribute (HOL) lifting_restore} @{syntax thmref} (@{syntax thmref} @{syntax thmref})?; |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1614 |
\<close>} |
47802 | 1615 |
|
1616 |
\begin{description} |
|
1617 |
||
47859 | 1618 |
\item @{command (HOL) "setup_lifting"} Sets up the Lifting package |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1619 |
to work with a user-defined type. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1620 |
The command supports two modes. The first one is a low-level mode when |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1621 |
the user must provide as a first |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1622 |
argument of @{command (HOL) "setup_lifting"} a |
57829 | 1623 |
quotient theorem @{term "Quotient R Abs Rep T"}. The |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1624 |
package configures a transfer rule for equality, a domain transfer |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1625 |
rules and sets up the @{command_def (HOL) "lift_definition"} |
57829 | 1626 |
command to work with the abstract type. An optional theorem @{term "reflp R"}, which certifies that |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1627 |
the equivalence relation R is total, |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1628 |
can be provided as a second argument. This allows the package to generate stronger transfer |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1629 |
rules. And finally, the parametricity theorem for R can be provided as a third argument. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1630 |
This allows the package to generate a stronger transfer rule for equality. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1631 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1632 |
Users generally will not prove the @{text Quotient} theorem manually for |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1633 |
new types, as special commands exist to automate the process. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1634 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1635 |
When a new subtype is defined by @{command (HOL) typedef}, @{command (HOL) "lift_definition"} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1636 |
can be used in its |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1637 |
second mode, where only the type_definition theorem @{text "type_definition Rep Abs A"} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1638 |
is used as an argument of the command. The command internally proves the corresponding |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1639 |
Quotient theorem and registers it with @{command (HOL) setup_lifting} using its first mode. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1640 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1641 |
For quotients, the command @{command (HOL) quotient_type} can be used. The command defines |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1642 |
a new quotient type and similarly to the previous case, the corresponding Quotient theorem is proved |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1643 |
and registered by @{command (HOL) setup_lifting}. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1644 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1645 |
The command @{command (HOL) "setup_lifting"} also sets up the code generator |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1646 |
for the new type. Later on, when a new constant is defined by @{command (HOL) "lift_definition"}, |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1647 |
the Lifting package proves and registers a code equation (if there is one) for the new constant. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1648 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1649 |
\item @{command (HOL) "lift_definition"} @{text "f :: \<tau>"} @{keyword (HOL) "is"} @{text t} |
47859 | 1650 |
Defines a new function @{text f} with an abstract type @{text \<tau>} |
1651 |
in terms of a corresponding operation @{text t} on a |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1652 |
representation type. More formally, if @{text "t :: \<sigma>"}, then |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1653 |
the command builds a term @{text "F"} as a corresponding combination of abstraction |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1654 |
and representation functions such that @{text "F :: \<sigma> \<Rightarrow> \<tau>" } and |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1655 |
defines @{text f} is as @{text "f \<equiv> F t"}. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1656 |
The term @{text t} does not have to be necessarily a constant but it can be any term. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1657 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1658 |
The command opens a proof environment and the user must discharge |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1659 |
a respectfulness proof obligation. For a type copy, i.e., a typedef with @{text |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1660 |
UNIV}, the obligation is discharged automatically. The proof goal is |
47802 | 1661 |
presented in a user-friendly, readable form. A respectfulness |
47859 | 1662 |
theorem in the standard format @{text f.rsp} and a transfer rule |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1663 |
@{text f.transfer} for the Transfer package are generated by the |
47859 | 1664 |
package. |
47802 | 1665 |
|
57829 | 1666 |
The user can specify a parametricity theorems for @{text t} after the keyword |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1667 |
@{keyword "parametric"}, which allows the command |
57829 | 1668 |
to generate parametric transfer rules for @{text f}. |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1669 |
|
50879 | 1670 |
For each constant defined through trivial quotients (type copies or |
1671 |
subtypes) @{text f.rep_eq} is generated. The equation is a code certificate |
|
1672 |
that defines @{text f} using the representation function. |
|
1673 |
||
1674 |
For each constant @{text f.abs_eq} is generated. The equation is unconditional |
|
1675 |
for total quotients. The equation defines @{text f} using |
|
1676 |
the abstraction function. |
|
1677 |
||
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1678 |
Integration with [@{attribute code} abstract]: For subtypes (e.g., |
47859 | 1679 |
corresponding to a datatype invariant, such as dlist), @{command |
50879 | 1680 |
(HOL) "lift_definition"} uses a code certificate theorem |
1681 |
@{text f.rep_eq} as a code equation. |
|
1682 |
||
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1683 |
Integration with [@{attribute code} equation]: For total quotients, @{command |
50879 | 1684 |
(HOL) "lift_definition"} uses @{text f.abs_eq} as a code equation. |
47802 | 1685 |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1686 |
\item @{command (HOL) lifting_forget} and @{command (HOL) lifting_update} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1687 |
These two commands serve for storing and deleting the set-up of |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1688 |
the Lifting package and corresponding transfer rules defined by this package. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1689 |
This is useful for hiding of type construction details of an abstract type |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1690 |
when the construction is finished but it still allows additions to this construction |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1691 |
when this is later necessary. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1692 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1693 |
Whenever the Lifting package is set up with a new abstract type @{text "\<tau>"} by |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1694 |
@{command_def (HOL) "lift_definition"}, the package defines a new bundle |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1695 |
that is called @{text "\<tau>.lifting"}. This bundle already includes set-up for the Lifting package. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1696 |
The new transfer rules |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1697 |
introduced by @{command (HOL) "lift_definition"} can be stored in the bundle by |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1698 |
the command @{command (HOL) "lifting_update"} @{text "\<tau>.lifting"}. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1699 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1700 |
The command @{command (HOL) "lifting_forget"} @{text "\<tau>.lifting"} deletes set-up of the Lifting |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1701 |
package |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1702 |
for @{text \<tau>} and deletes all the transfer rules that were introduced |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1703 |
by @{command (HOL) "lift_definition"} using @{text \<tau>} as an abstract type. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1704 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1705 |
The stored set-up in a bundle can be reintroduced by the Isar commands for including a bundle |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1706 |
(@{command "include"}, @{keyword "includes"} and @{command "including"}). |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1707 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
53015
diff
changeset
|
1708 |
\item @{command (HOL) "print_quot_maps"} prints stored quotient map |
47859 | 1709 |
theorems. |
1710 |
||
1711 |
\item @{command (HOL) "print_quotients"} prints stored quotient |
|
1712 |
theorems. |
|
1713 |
||
1714 |
\item @{attribute (HOL) quot_map} registers a quotient map |
|
57829 | 1715 |
theorem, a theorem showing how to "lift" quotients over type constructors. |
1716 |
E.g., @{term "Quotient R Abs Rep T \<Longrightarrow> |
|
1717 |
Quotient (rel_set R) (image Abs) (image Rep) (rel_set T)"}. |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1718 |
For examples see @{file |
57829 | 1719 |
"~~/src/HOL/Lifting_Set.thy"} or @{file "~~/src/HOL/Lifting.thy"}. |
1720 |
This property is proved automatically if the involved type is BNF without dead variables. |
|
47859 | 1721 |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
1722 |
\item @{attribute (HOL) relator_eq_onp} registers a theorem that |
57829 | 1723 |
shows that a relator applied to an equality restricted by a predicate @{term P} (i.e., @{term |
1724 |
"eq_onp P"}) is equal |
|
1725 |
to a predicator applied to the @{term P}. The combinator @{const eq_onp} is used for |
|
1726 |
internal encoding of proper subtypes. Such theorems allows the package to hide @{text |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
1727 |
eq_onp} from a user in a user-readable form of a |
47859 | 1728 |
respectfulness theorem. For examples see @{file |
57829 | 1729 |
"~~/src/HOL/Lifting_Set.thy"} or @{file "~~/src/HOL/Lifting.thy"}. |
1730 |
This property is proved automatically if the involved type is BNF without dead variables. |
|
47802 | 1731 |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1732 |
\item @{attribute (HOL) "relator_mono"} registers a property describing a monotonicity of a relator. |
57829 | 1733 |
E.g., @{term "A \<le> B \<Longrightarrow> rel_set A \<le> rel_set B"}. |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1734 |
This property is needed for proving a stronger transfer rule in @{command_def (HOL) "lift_definition"} |
57829 | 1735 |
when a parametricity theorem for the raw term is specified and also for the reflexivity prover. |
1736 |
For examples see @{file |
|
1737 |
"~~/src/HOL/Lifting_Set.thy"} or @{file "~~/src/HOL/Lifting.thy"}. |
|
1738 |
This property is proved automatically if the involved type is BNF without dead variables. |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1739 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1740 |
\item @{attribute (HOL) "relator_distr"} registers a property describing a distributivity |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1741 |
of the relation composition and a relator. E.g., |
57829 | 1742 |
@{text "rel_set R \<circ>\<circ> rel_set S = rel_set (R \<circ>\<circ> S)"}. |
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1743 |
This property is needed for proving a stronger transfer rule in @{command_def (HOL) "lift_definition"} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1744 |
when a parametricity theorem for the raw term is specified. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1745 |
When this equality does not hold unconditionally (e.g., for the function type), the user can specified |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1746 |
each direction separately and also register multiple theorems with different set of assumptions. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1747 |
This attribute can be used only after the monotonicity property was already registered by |
57829 | 1748 |
@{attribute (HOL) "relator_mono"}. For examples see @{file |
1749 |
"~~/src/HOL/Lifting_Set.thy"} or @{file "~~/src/HOL/Lifting.thy"}. |
|
1750 |
This property is proved automatically if the involved type is BNF without dead variables. |
|
50877 | 1751 |
|
1752 |
\item @{attribute (HOL) quot_del} deletes a corresponding Quotient theorem |
|
1753 |
from the Lifting infrastructure and thus de-register the corresponding quotient. |
|
1754 |
This effectively causes that @{command (HOL) lift_definition} will not |
|
54334
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1755 |
do any lifting for the corresponding type. This attribute is rather used for low-level |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1756 |
manipulation with set-up of the Lifting package because @{command (HOL) lifting_forget} is |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1757 |
preferred for normal usage. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1758 |
|
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1759 |
\item @{attribute (HOL) lifting_restore} @{text "Quotient_thm pcr_def pcr_cr_eq_thm"} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1760 |
registers the Quotient theorem @{text Quotient_thm} in the Lifting infrastructure |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1761 |
and thus sets up lifting for an abstract type @{text \<tau>} (that is defined by @{text Quotient_thm}). |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1762 |
Optional theorems @{text pcr_def} and @{text pcr_cr_eq_thm} can be specified to register |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1763 |
the parametrized |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1764 |
correspondence relation for @{text \<tau>}. E.g., for @{text "'a dlist"}, @{text pcr_def} is |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1765 |
@{text "pcr_dlist A \<equiv> list_all2 A \<circ>\<circ> cr_dlist"} and @{text pcr_cr_eq_thm} is |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1766 |
@{text "pcr_dlist op= = op="}. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1767 |
This attribute is rather used for low-level |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1768 |
manipulation with set-up of the Lifting package because using of the bundle @{text \<tau>.lifting} |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1769 |
together with the commands @{command (HOL) lifting_forget} and @{command (HOL) lifting_update} is |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1770 |
preferred for normal usage. |
409d7f7247f4
update documentation of Lifting/Transfer and Quotient
kuncar
parents:
54017
diff
changeset
|
1771 |
|
58552 | 1772 |
\item Integration with the BNF package @{cite "isabelle-datatypes"}: |
57829 | 1773 |
As already mentioned, the theorems that are registered |
1774 |
by the following attributes are proved and registered automatically if the involved type |
|
1775 |
is BNF without dead variables: @{attribute (HOL) quot_map}, @{attribute (HOL) relator_eq_onp}, |
|
1776 |
@{attribute (HOL) "relator_mono"}, @{attribute (HOL) "relator_distr"}. Also the definition of a |
|
1777 |
relator and predicator is provided automatically. Moreover, if the BNF represents a datatype, |
|
1778 |
simplification rules for a predicator are again proved automatically. |
|
1779 |
||
47802 | 1780 |
\end{description} |
58618 | 1781 |
\<close> |
1782 |
||
1783 |
||
1784 |
section \<open>Coercive subtyping\<close> |
|
1785 |
||
1786 |
text \<open> |
|
43994 | 1787 |
\begin{matharray}{rcl} |
1788 |
@{attribute_def (HOL) coercion} & : & @{text attribute} \\ |
|
1789 |
@{attribute_def (HOL) coercion_enabled} & : & @{text attribute} \\ |
|
1790 |
@{attribute_def (HOL) coercion_map} & : & @{text attribute} \\ |
|
1791 |
\end{matharray} |
|
1792 |
||
46280 | 1793 |
Coercive subtyping allows the user to omit explicit type |
1794 |
conversions, also called \emph{coercions}. Type inference will add |
|
1795 |
them as necessary when parsing a term. See |
|
58552 | 1796 |
@{cite "traytel-berghofer-nipkow-2011"} for details. |
46280 | 1797 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1798 |
@{rail \<open> |
43994 | 1799 |
@@{attribute (HOL) coercion} (@{syntax term})? |
1800 |
; |
|
1801 |
@@{attribute (HOL) coercion_map} (@{syntax term})? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1802 |
\<close>} |
43994 | 1803 |
|
1804 |
\begin{description} |
|
1805 |
||
1806 |
\item @{attribute (HOL) "coercion"}~@{text "f"} registers a new |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1807 |
coercion function @{text "f :: \<sigma>\<^sub>1 \<Rightarrow> \<sigma>\<^sub>2"} where @{text "\<sigma>\<^sub>1"} and |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1808 |
@{text "\<sigma>\<^sub>2"} are type constructors without arguments. Coercions are |
46280 | 1809 |
composed by the inference algorithm if needed. Note that the type |
1810 |
inference algorithm is complete only if the registered coercions |
|
1811 |
form a lattice. |
|
43994 | 1812 |
|
46280 | 1813 |
\item @{attribute (HOL) "coercion_map"}~@{text "map"} registers a |
1814 |
new map function to lift coercions through type constructors. The |
|
1815 |
function @{text "map"} must conform to the following type pattern |
|
43994 | 1816 |
|
1817 |
\begin{matharray}{lll} |
|
1818 |
@{text "map"} & @{text "::"} & |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1819 |
@{text "f\<^sub>1 \<Rightarrow> \<dots> \<Rightarrow> f\<^sub>n \<Rightarrow> (\<alpha>\<^sub>1, \<dots>, \<alpha>\<^sub>n) t \<Rightarrow> (\<beta>\<^sub>1, \<dots>, \<beta>\<^sub>n) t"} \\ |
43994 | 1820 |
\end{matharray} |
1821 |
||
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1822 |
where @{text "t"} is a type constructor and @{text "f\<^sub>i"} is of type |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
1823 |
@{text "\<alpha>\<^sub>i \<Rightarrow> \<beta>\<^sub>i"} or @{text "\<beta>\<^sub>i \<Rightarrow> \<alpha>\<^sub>i"}. Registering a map function |
46280 | 1824 |
overwrites any existing map function for this particular type |
1825 |
constructor. |
|
43994 | 1826 |
|
1827 |
\item @{attribute (HOL) "coercion_enabled"} enables the coercion |
|
1828 |
inference algorithm. |
|
1829 |
||
1830 |
\end{description} |
|
58618 | 1831 |
\<close> |
1832 |
||
1833 |
||
1834 |
section \<open>Arithmetic proof support\<close> |
|
1835 |
||
1836 |
text \<open> |
|
26849 | 1837 |
\begin{matharray}{rcl} |
28761
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
1838 |
@{method_def (HOL) arith} & : & @{text method} \\ |
30863 | 1839 |
@{attribute_def (HOL) arith} & : & @{text attribute} \\ |
28761
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
1840 |
@{attribute_def (HOL) arith_split} & : & @{text attribute} \\ |
26849 | 1841 |
\end{matharray} |
1842 |
||
46280 | 1843 |
\begin{description} |
26849 | 1844 |
|
46280 | 1845 |
\item @{method (HOL) arith} decides linear arithmetic problems (on |
1846 |
types @{text nat}, @{text int}, @{text real}). Any current facts |
|
1847 |
are inserted into the goal before running the procedure. |
|
26849 | 1848 |
|
46280 | 1849 |
\item @{attribute (HOL) arith} declares facts that are supplied to |
1850 |
the arithmetic provers implicitly. |
|
1851 |
||
1852 |
\item @{attribute (HOL) arith_split} attribute declares case split |
|
30865 | 1853 |
rules to be expanded before @{method (HOL) arith} is invoked. |
30863 | 1854 |
|
46280 | 1855 |
\end{description} |
1856 |
||
1857 |
Note that a simpler (but faster) arithmetic prover is already |
|
1858 |
invoked by the Simplifier. |
|
58618 | 1859 |
\<close> |
1860 |
||
1861 |
||
1862 |
section \<open>Intuitionistic proof search\<close> |
|
1863 |
||
1864 |
text \<open> |
|
30169 | 1865 |
\begin{matharray}{rcl} |
30171 | 1866 |
@{method_def (HOL) iprover} & : & @{text method} \\ |
30169 | 1867 |
\end{matharray} |
1868 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1869 |
@{rail \<open> |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1870 |
@@{method (HOL) iprover} (@{syntax rulemod} *) |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1871 |
\<close>} |
30169 | 1872 |
|
46280 | 1873 |
\begin{description} |
1874 |
||
1875 |
\item @{method (HOL) iprover} performs intuitionistic proof search, |
|
1876 |
depending on specifically declared rules from the context, or given |
|
1877 |
as explicit arguments. Chained facts are inserted into the goal |
|
1878 |
before commencing proof search. |
|
35613 | 1879 |
|
30169 | 1880 |
Rules need to be classified as @{attribute (Pure) intro}, |
1881 |
@{attribute (Pure) elim}, or @{attribute (Pure) dest}; here the |
|
1882 |
``@{text "!"}'' indicator refers to ``safe'' rules, which may be |
|
1883 |
applied aggressively (without considering back-tracking later). |
|
1884 |
Rules declared with ``@{text "?"}'' are ignored in proof search (the |
|
42626 | 1885 |
single-step @{method (Pure) rule} method still observes these). An |
30169 | 1886 |
explicit weight annotation may be given as well; otherwise the |
1887 |
number of rule premises will be taken into account here. |
|
46280 | 1888 |
|
1889 |
\end{description} |
|
58618 | 1890 |
\<close> |
1891 |
||
1892 |
||
1893 |
section \<open>Model Elimination and Resolution\<close> |
|
1894 |
||
1895 |
text \<open> |
|
43578
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1896 |
\begin{matharray}{rcl} |
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1897 |
@{method_def (HOL) "meson"} & : & @{text method} \\ |
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1898 |
@{method_def (HOL) "metis"} & : & @{text method} \\ |
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1899 |
\end{matharray} |
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1900 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1901 |
@{rail \<open> |
43578
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1902 |
@@{method (HOL) meson} @{syntax thmrefs}? |
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1903 |
; |
46280 | 1904 |
@@{method (HOL) metis} |
1905 |
('(' ('partial_types' | 'full_types' | 'no_types' | @{syntax name}) ')')? |
|
1906 |
@{syntax thmrefs}? |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1907 |
\<close>} |
43578
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1908 |
|
46280 | 1909 |
\begin{description} |
1910 |
||
1911 |
\item @{method (HOL) meson} implements Loveland's model elimination |
|
58552 | 1912 |
procedure @{cite "loveland-78"}. See @{file |
46280 | 1913 |
"~~/src/HOL/ex/Meson_Test.thy"} for examples. |
43578
36ba44fe0781
document "meson" and "metis" in HOL specific section of the Isar ref manual
blanchet
parents:
43270
diff
changeset
|
1914 |
|
46280 | 1915 |
\item @{method (HOL) metis} combines ordered resolution and ordered |
1916 |
paramodulation to find first-order (or mildly higher-order) proofs. |
|
1917 |
The first optional argument specifies a type encoding; see the |
|
58552 | 1918 |
Sledgehammer manual @{cite "isabelle-sledgehammer"} for details. The |
46280 | 1919 |
directory @{file "~~/src/HOL/Metis_Examples"} contains several small |
1920 |
theories developed to a large extent using @{method (HOL) metis}. |
|
1921 |
||
1922 |
\end{description} |
|
58618 | 1923 |
\<close> |
1924 |
||
1925 |
||
1926 |
section \<open>Algebraic reasoning via Gr\"obner bases\<close> |
|
1927 |
||
1928 |
text \<open> |
|
50130 | 1929 |
\begin{matharray}{rcl} |
1930 |
@{method_def (HOL) "algebra"} & : & @{text method} \\ |
|
1931 |
@{attribute_def (HOL) algebra} & : & @{text attribute} \\ |
|
1932 |
\end{matharray} |
|
1933 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1934 |
@{rail \<open> |
50130 | 1935 |
@@{method (HOL) algebra} |
1936 |
('add' ':' @{syntax thmrefs})? |
|
1937 |
('del' ':' @{syntax thmrefs})? |
|
1938 |
; |
|
1939 |
@@{attribute (HOL) algebra} (() | 'add' | 'del') |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
1940 |
\<close>} |
50130 | 1941 |
|
1942 |
\begin{description} |
|
1943 |
||
1944 |
\item @{method (HOL) algebra} performs algebraic reasoning via |
|
58552 | 1945 |
Gr\"obner bases, see also @{cite "Chaieb-Wenzel:2007"} and |
1946 |
@{cite \<open>\S3.2\<close> "Chaieb-thesis"}. The method handles deals with two main |
|
50130 | 1947 |
classes of problems: |
1948 |
||
1949 |
\begin{enumerate} |
|
1950 |
||
1951 |
\item Universal problems over multivariate polynomials in a |
|
1952 |
(semi)-ring/field/idom; the capabilities of the method are augmented |
|
1953 |
according to properties of these structures. For this problem class |
|
1954 |
the method is only complete for algebraically closed fields, since |
|
1955 |
the underlying method is based on Hilbert's Nullstellensatz, where |
|
1956 |
the equivalence only holds for algebraically closed fields. |
|
1957 |
||
1958 |
The problems can contain equations @{text "p = 0"} or inequations |
|
1959 |
@{text "q \<noteq> 0"} anywhere within a universal problem statement. |
|
1960 |
||
1961 |
\item All-exists problems of the following restricted (but useful) |
|
1962 |
form: |
|
1963 |
||
1964 |
@{text [display] "\<forall>x\<^sub>1 \<dots> x\<^sub>n. |
|
1965 |
e\<^sub>1(x\<^sub>1, \<dots>, x\<^sub>n) = 0 \<and> \<dots> \<and> e\<^sub>m(x\<^sub>1, \<dots>, x\<^sub>n) = 0 \<longrightarrow> |
|
1966 |
(\<exists>y\<^sub>1 \<dots> y\<^sub>k. |
|
1967 |
p\<^sub>1\<^sub>1(x\<^sub>1, \<dots> ,x\<^sub>n) * y\<^sub>1 + \<dots> + p\<^sub>1\<^sub>k(x\<^sub>1, \<dots>, x\<^sub>n) * y\<^sub>k = 0 \<and> |
|
1968 |
\<dots> \<and> |
|
1969 |
p\<^sub>t\<^sub>1(x\<^sub>1, \<dots>, x\<^sub>n) * y\<^sub>1 + \<dots> + p\<^sub>t\<^sub>k(x\<^sub>1, \<dots>, x\<^sub>n) * y\<^sub>k = 0)"} |
|
1970 |
||
1971 |
Here @{text "e\<^sub>1, \<dots>, e\<^sub>n"} and the @{text "p\<^sub>i\<^sub>j"} are multivariate |
|
1972 |
polynomials only in the variables mentioned as arguments. |
|
1973 |
||
1974 |
\end{enumerate} |
|
1975 |
||
1976 |
The proof method is preceded by a simplification step, which may be |
|
1977 |
modified by using the form @{text "(algebra add: ths\<^sub>1 del: ths\<^sub>2)"}. |
|
1978 |
This acts like declarations for the Simplifier |
|
1979 |
(\secref{sec:simplifier}) on a private simpset for this tool. |
|
1980 |
||
1981 |
\item @{attribute algebra} (as attribute) manages the default |
|
1982 |
collection of pre-simplification rules of the above proof method. |
|
1983 |
||
1984 |
\end{description} |
|
58618 | 1985 |
\<close> |
1986 |
||
1987 |
||
1988 |
subsubsection \<open>Example\<close> |
|
1989 |
||
1990 |
text \<open>The subsequent example is from geometry: collinearity is |
|
1991 |
invariant by rotation.\<close> |
|
50130 | 1992 |
|
1993 |
type_synonym point = "int \<times> int" |
|
1994 |
||
1995 |
fun collinear :: "point \<Rightarrow> point \<Rightarrow> point \<Rightarrow> bool" where |
|
1996 |
"collinear (Ax, Ay) (Bx, By) (Cx, Cy) \<longleftrightarrow> |
|
1997 |
(Ax - Bx) * (By - Cy) = (Ay - By) * (Bx - Cx)" |
|
1998 |
||
1999 |
lemma collinear_inv_rotation: |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
52895
diff
changeset
|
2000 |
assumes "collinear (Ax, Ay) (Bx, By) (Cx, Cy)" and "c\<^sup>2 + s\<^sup>2 = 1" |
50130 | 2001 |
shows "collinear (Ax * c - Ay * s, Ay * c + Ax * s) |
2002 |
(Bx * c - By * s, By * c + Bx * s) (Cx * c - Cy * s, Cy * c + Cx * s)" |
|
2003 |
using assms by (algebra add: collinear.simps) |
|
2004 |
||
58618 | 2005 |
text \<open> |
53982 | 2006 |
See also @{file "~~/src/HOL/ex/Groebner_Examples.thy"}. |
58618 | 2007 |
\<close> |
2008 |
||
2009 |
||
2010 |
section \<open>Coherent Logic\<close> |
|
2011 |
||
2012 |
text \<open> |
|
30171 | 2013 |
\begin{matharray}{rcl} |
2014 |
@{method_def (HOL) "coherent"} & : & @{text method} \\ |
|
2015 |
\end{matharray} |
|
2016 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2017 |
@{rail \<open> |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2018 |
@@{method (HOL) coherent} @{syntax thmrefs}? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2019 |
\<close>} |
30171 | 2020 |
|
46280 | 2021 |
\begin{description} |
2022 |
||
2023 |
\item @{method (HOL) coherent} solves problems of \emph{Coherent |
|
58552 | 2024 |
Logic} @{cite "Bezem-Coquand:2005"}, which covers applications in |
46280 | 2025 |
confluence theory, lattice theory and projective geometry. See |
2026 |
@{file "~~/src/HOL/ex/Coherent.thy"} for some examples. |
|
2027 |
||
2028 |
\end{description} |
|
58618 | 2029 |
\<close> |
2030 |
||
2031 |
||
2032 |
section \<open>Proving propositions\<close> |
|
2033 |
||
2034 |
text \<open> |
|
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2035 |
In addition to the standard proof methods, a number of diagnosis |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2036 |
tools search for proofs and provide an Isar proof snippet on success. |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2037 |
These tools are available via the following commands. |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2038 |
|
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2039 |
\begin{matharray}{rcl} |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2040 |
@{command_def (HOL) "solve_direct"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\ |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2041 |
@{command_def (HOL) "try"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\ |
46641 | 2042 |
@{command_def (HOL) "try0"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\ |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2043 |
@{command_def (HOL) "sledgehammer"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\ |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2044 |
@{command_def (HOL) "sledgehammer_params"} & : & @{text "theory \<rightarrow> theory"} |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2045 |
\end{matharray} |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2046 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2047 |
@{rail \<open> |
43040 | 2048 |
@@{command (HOL) try} |
2049 |
; |
|
2050 |
||
46641 | 2051 |
@@{command (HOL) try0} ( ( ( 'simp' | 'intro' | 'elim' | 'dest' ) ':' @{syntax thmrefs} ) + ) ? |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2052 |
@{syntax nat}? |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2053 |
; |
43040 | 2054 |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2055 |
@@{command (HOL) sledgehammer} ( '[' args ']' )? facts? @{syntax nat}? |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2056 |
; |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2057 |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2058 |
@@{command (HOL) sledgehammer_params} ( ( '[' args ']' ) ? ) |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2059 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2060 |
args: ( @{syntax name} '=' value + ',' ) |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2061 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2062 |
facts: '(' ( ( ( ( 'add' | 'del' ) ':' ) ? @{syntax thmrefs} ) + ) ? ')' |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2063 |
\<close>} % FIXME check args "value" |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2064 |
|
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2065 |
\begin{description} |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2066 |
|
46283 | 2067 |
\item @{command (HOL) "solve_direct"} checks whether the current |
2068 |
subgoals can be solved directly by an existing theorem. Duplicate |
|
2069 |
lemmas can be detected in this way. |
|
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2070 |
|
46641 | 2071 |
\item @{command (HOL) "try0"} attempts to prove a subgoal |
46283 | 2072 |
using a combination of standard proof methods (@{method auto}, |
2073 |
@{method simp}, @{method blast}, etc.). Additional facts supplied |
|
2074 |
via @{text "simp:"}, @{text "intro:"}, @{text "elim:"}, and @{text |
|
2075 |
"dest:"} are passed to the appropriate proof methods. |
|
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2076 |
|
43914
64819f353c53
updating documentation about quickcheck; adding information about try
bulwahn
parents:
43578
diff
changeset
|
2077 |
\item @{command (HOL) "try"} attempts to prove or disprove a subgoal |
46283 | 2078 |
using a combination of provers and disprovers (@{command (HOL) |
2079 |
"solve_direct"}, @{command (HOL) "quickcheck"}, @{command (HOL) |
|
46641 | 2080 |
"try0"}, @{command (HOL) "sledgehammer"}, @{command (HOL) |
46283 | 2081 |
"nitpick"}). |
43914
64819f353c53
updating documentation about quickcheck; adding information about try
bulwahn
parents:
43578
diff
changeset
|
2082 |
|
46283 | 2083 |
\item @{command (HOL) "sledgehammer"} attempts to prove a subgoal |
2084 |
using external automatic provers (resolution provers and SMT |
|
58552 | 2085 |
solvers). See the Sledgehammer manual @{cite "isabelle-sledgehammer"} |
46283 | 2086 |
for details. |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2087 |
|
46283 | 2088 |
\item @{command (HOL) "sledgehammer_params"} changes @{command (HOL) |
2089 |
"sledgehammer"} configuration options persistently. |
|
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2090 |
|
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2091 |
\end{description} |
58618 | 2092 |
\<close> |
2093 |
||
2094 |
||
2095 |
section \<open>Checking and refuting propositions\<close> |
|
2096 |
||
2097 |
text \<open> |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2098 |
Identifying incorrect propositions usually involves evaluation of |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2099 |
particular assignments and systematic counterexample search. This |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2100 |
is supported by the following commands. |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2101 |
|
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2102 |
\begin{matharray}{rcl} |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2103 |
@{command_def (HOL) "value"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
45409
5abb0e738b00
adding some documentation about the values command to the isar reference
bulwahn
parents:
45408
diff
changeset
|
2104 |
@{command_def (HOL) "values"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2105 |
@{command_def (HOL) "quickcheck"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\ |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2106 |
@{command_def (HOL) "nitpick"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow>"} \\ |
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2107 |
@{command_def (HOL) "quickcheck_params"} & : & @{text "theory \<rightarrow> theory"} \\ |
45943
8c4a5e664fbc
adding documentation about the quickcheck_generator command in the IsarRef
bulwahn
parents:
45839
diff
changeset
|
2108 |
@{command_def (HOL) "nitpick_params"} & : & @{text "theory \<rightarrow> theory"} \\ |
46592
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2109 |
@{command_def (HOL) "quickcheck_generator"} & : & @{text "theory \<rightarrow> theory"} \\ |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2110 |
@{command_def (HOL) "find_unused_assms"} & : & @{text "context \<rightarrow>"} |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2111 |
\end{matharray} |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2112 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2113 |
@{rail \<open> |
58100
f54a8a4134d3
restored generic value slot, retaining default behaviour and separate approximate command
haftmann
parents:
57829
diff
changeset
|
2114 |
@@{command (HOL) value} ( '[' @{syntax name} ']' )? modes? @{syntax term} |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2115 |
; |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2116 |
|
45409
5abb0e738b00
adding some documentation about the values command to the isar reference
bulwahn
parents:
45408
diff
changeset
|
2117 |
@@{command (HOL) values} modes? @{syntax nat}? @{syntax term} |
5abb0e738b00
adding some documentation about the values command to the isar reference
bulwahn
parents:
45408
diff
changeset
|
2118 |
; |
5abb0e738b00
adding some documentation about the values command to the isar reference
bulwahn
parents:
45408
diff
changeset
|
2119 |
|
49993
80402e0e78e3
removed "refute" command from Isar manual, now that it has been moved outside "Main"
blanchet
parents:
49836
diff
changeset
|
2120 |
(@@{command (HOL) quickcheck} | @@{command (HOL) nitpick}) |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2121 |
( '[' args ']' )? @{syntax nat}? |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2122 |
; |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2123 |
|
49993
80402e0e78e3
removed "refute" command from Isar manual, now that it has been moved outside "Main"
blanchet
parents:
49836
diff
changeset
|
2124 |
(@@{command (HOL) quickcheck_params} | |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2125 |
@@{command (HOL) nitpick_params}) ( '[' args ']' )? |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2126 |
; |
46592
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2127 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2128 |
@@{command (HOL) quickcheck_generator} @{syntax nameref} \<newline> |
45943
8c4a5e664fbc
adding documentation about the quickcheck_generator command in the IsarRef
bulwahn
parents:
45839
diff
changeset
|
2129 |
'operations:' ( @{syntax term} +) |
8c4a5e664fbc
adding documentation about the quickcheck_generator command in the IsarRef
bulwahn
parents:
45839
diff
changeset
|
2130 |
; |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2131 |
|
46628 | 2132 |
@@{command (HOL) find_unused_assms} @{syntax name}? |
46592
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2133 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2134 |
modes: '(' (@{syntax name} +) ')' |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2135 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2136 |
args: ( @{syntax name} '=' value + ',' ) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2137 |
\<close>} % FIXME check "value" |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2138 |
|
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2139 |
\begin{description} |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2140 |
|
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2141 |
\item @{command (HOL) "value"}~@{text t} evaluates and prints a |
46283 | 2142 |
term; optionally @{text modes} can be specified, which are appended |
2143 |
to the current print mode; see \secref{sec:print-modes}. |
|
56927 | 2144 |
Evaluation is tried first using ML, falling |
2145 |
back to normalization by evaluation if this fails. |
|
58100
f54a8a4134d3
restored generic value slot, retaining default behaviour and separate approximate command
haftmann
parents:
57829
diff
changeset
|
2146 |
Alternatively a specific evaluator can be selected using square |
f54a8a4134d3
restored generic value slot, retaining default behaviour and separate approximate command
haftmann
parents:
57829
diff
changeset
|
2147 |
brackets; typical evaluators use the current set of code equations |
f54a8a4134d3
restored generic value slot, retaining default behaviour and separate approximate command
haftmann
parents:
57829
diff
changeset
|
2148 |
to normalize and include @{text simp} for fully symbolic evaluation |
f54a8a4134d3
restored generic value slot, retaining default behaviour and separate approximate command
haftmann
parents:
57829
diff
changeset
|
2149 |
using the simplifier, @{text nbe} for \emph{normalization by |
f54a8a4134d3
restored generic value slot, retaining default behaviour and separate approximate command
haftmann
parents:
57829
diff
changeset
|
2150 |
evaluation} and \emph{code} for code generation in SML. |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2151 |
|
46283 | 2152 |
\item @{command (HOL) "values"}~@{text t} enumerates a set |
2153 |
comprehension by evaluation and prints its values up to the given |
|
2154 |
number of solutions; optionally @{text modes} can be specified, |
|
2155 |
which are appended to the current print mode; see |
|
2156 |
\secref{sec:print-modes}. |
|
45409
5abb0e738b00
adding some documentation about the values command to the isar reference
bulwahn
parents:
45408
diff
changeset
|
2157 |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2158 |
\item @{command (HOL) "quickcheck"} tests the current goal for |
46283 | 2159 |
counterexamples using a series of assignments for its free |
2160 |
variables; by default the first subgoal is tested, an other can be |
|
2161 |
selected explicitly using an optional goal index. Assignments can |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
2162 |
be chosen exhausting the search space up to a given size, or using a |
46283 | 2163 |
fixed number of random assignments in the search space, or exploring |
2164 |
the search space symbolically using narrowing. By default, |
|
2165 |
quickcheck uses exhaustive testing. A number of configuration |
|
2166 |
options are supported for @{command (HOL) "quickcheck"}, notably: |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2167 |
|
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2168 |
\begin{description} |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2169 |
|
43914
64819f353c53
updating documentation about quickcheck; adding information about try
bulwahn
parents:
43578
diff
changeset
|
2170 |
\item[@{text tester}] specifies which testing approach to apply. |
46283 | 2171 |
There are three testers, @{text exhaustive}, @{text random}, and |
2172 |
@{text narrowing}. An unknown configuration option is treated as |
|
2173 |
an argument to tester, making @{text "tester ="} optional. When |
|
2174 |
multiple testers are given, these are applied in parallel. If no |
|
2175 |
tester is specified, quickcheck uses the testers that are set |
|
2176 |
active, i.e., configurations @{attribute |
|
2177 |
quickcheck_exhaustive_active}, @{attribute |
|
2178 |
quickcheck_random_active}, @{attribute |
|
2179 |
quickcheck_narrowing_active} are set to true. |
|
2180 |
||
40254 | 2181 |
\item[@{text size}] specifies the maximum size of the search space |
2182 |
for assignment values. |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2183 |
|
45758
6210c350d88b
documenting the genuine_only option in quickcheck;
bulwahn
parents:
45701
diff
changeset
|
2184 |
\item[@{text genuine_only}] sets quickcheck only to return genuine |
46283 | 2185 |
counterexample, but not potentially spurious counterexamples due |
2186 |
to underspecified functions. |
|
46498
2754784e9153
adding documentation for abort_potential option in quickcheck
bulwahn
parents:
46494
diff
changeset
|
2187 |
|
2754784e9153
adding documentation for abort_potential option in quickcheck
bulwahn
parents:
46494
diff
changeset
|
2188 |
\item[@{text abort_potential}] sets quickcheck to abort once it |
2754784e9153
adding documentation for abort_potential option in quickcheck
bulwahn
parents:
46494
diff
changeset
|
2189 |
found a potentially spurious counterexample and to not continue |
2754784e9153
adding documentation for abort_potential option in quickcheck
bulwahn
parents:
46494
diff
changeset
|
2190 |
to search for a further genuine counterexample. |
2754784e9153
adding documentation for abort_potential option in quickcheck
bulwahn
parents:
46494
diff
changeset
|
2191 |
For this option to be effective, the @{text genuine_only} option |
2754784e9153
adding documentation for abort_potential option in quickcheck
bulwahn
parents:
46494
diff
changeset
|
2192 |
must be set to false. |
47859 | 2193 |
|
42092
f07b373f25d3
adding documentation about the eval option in quickcheck
bulwahn
parents:
41846
diff
changeset
|
2194 |
\item[@{text eval}] takes a term or a list of terms and evaluates |
46283 | 2195 |
these terms under the variable assignment found by quickcheck. |
48159 | 2196 |
This option is currently only supported by the default |
2197 |
(exhaustive) tester. |
|
42123 | 2198 |
|
40254 | 2199 |
\item[@{text iterations}] sets how many sets of assignments are |
2200 |
generated for each particular size. |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2201 |
|
40254 | 2202 |
\item[@{text no_assms}] specifies whether assumptions in |
2203 |
structured proofs should be ignored. |
|
35331 | 2204 |
|
47349
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2205 |
\item[@{text locale}] specifies how to process conjectures in |
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2206 |
a locale context, i.e., they can be interpreted or expanded. |
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2207 |
The option is a whitespace-separated list of the two words |
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2208 |
@{text interpret} and @{text expand}. The list determines the |
47859 | 2209 |
order they are employed. The default setting is to first use |
47349
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2210 |
interpretations and then test the expanded conjecture. |
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2211 |
The option is only provided as attribute declaration, but not |
47859 | 2212 |
as parameter to the command. |
47349
803729c9fd4d
documenting options quickcheck_locale; adjusting IsarRef documentation of Quotient predicate; NEWS
bulwahn
parents:
46641
diff
changeset
|
2213 |
|
40254 | 2214 |
\item[@{text timeout}] sets the time limit in seconds. |
40245
59f011c1877a
updating documentation on quickcheck in the Isar reference
bulwahn
parents:
40171
diff
changeset
|
2215 |
|
40254 | 2216 |
\item[@{text default_type}] sets the type(s) generally used to |
2217 |
instantiate type variables. |
|
40245
59f011c1877a
updating documentation on quickcheck in the Isar reference
bulwahn
parents:
40171
diff
changeset
|
2218 |
|
40254 | 2219 |
\item[@{text report}] if set quickcheck reports how many tests |
2220 |
fulfilled the preconditions. |
|
40245
59f011c1877a
updating documentation on quickcheck in the Isar reference
bulwahn
parents:
40171
diff
changeset
|
2221 |
|
46592
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2222 |
\item[@{text use_subtype}] if set quickcheck automatically lifts |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2223 |
conjectures to registered subtypes if possible, and tests the |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2224 |
lifted conjecture. |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2225 |
|
45766
46046d8e9659
updating documentation about quiet and verbose options in quickcheck
bulwahn
parents:
45758
diff
changeset
|
2226 |
\item[@{text quiet}] if set quickcheck does not output anything |
46046d8e9659
updating documentation about quiet and verbose options in quickcheck
bulwahn
parents:
45758
diff
changeset
|
2227 |
while testing. |
47859 | 2228 |
|
46283 | 2229 |
\item[@{text verbose}] if set quickcheck informs about the current |
2230 |
size and cardinality while testing. |
|
40245
59f011c1877a
updating documentation on quickcheck in the Isar reference
bulwahn
parents:
40171
diff
changeset
|
2231 |
|
40254 | 2232 |
\item[@{text expect}] can be used to check if the user's |
2233 |
expectation was met (@{text no_expectation}, @{text |
|
2234 |
no_counterexample}, or @{text counterexample}). |
|
40245
59f011c1877a
updating documentation on quickcheck in the Isar reference
bulwahn
parents:
40171
diff
changeset
|
2235 |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2236 |
\end{description} |
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2237 |
|
46283 | 2238 |
These option can be given within square brackets. |
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2239 |
|
56363
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2240 |
Using the following type classes, the testers generate values and convert |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2241 |
them back into Isabelle terms for displaying counterexamples. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2242 |
\begin{description} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2243 |
\item[@{text exhaustive}] The parameters of the type classes @{class exhaustive} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2244 |
and @{class full_exhaustive} implement the testing. They take a |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2245 |
testing function as a parameter, which takes a value of type @{typ "'a"} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2246 |
and optionally produces a counterexample, and a size parameter for the test values. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2247 |
In @{class full_exhaustive}, the testing function parameter additionally |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2248 |
expects a lazy term reconstruction in the type @{typ Code_Evaluation.term} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2249 |
of the tested value. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2250 |
|
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2251 |
The canonical implementation for @{text exhaustive} testers calls the given |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2252 |
testing function on all values up to the given size and stops as soon |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2253 |
as a counterexample is found. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2254 |
|
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2255 |
\item[@{text random}] The operation @{const Quickcheck_Random.random} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2256 |
of the type class @{class random} generates a pseudo-random |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2257 |
value of the given size and a lazy term reconstruction of the value |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2258 |
in the type @{typ Code_Evaluation.term}. A pseudo-randomness generator |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2259 |
is defined in theory @{theory Random}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2260 |
|
58552 | 2261 |
\item[@{text narrowing}] implements Haskell's Lazy Smallcheck @{cite "runciman-naylor-lindblad"} |
56363
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2262 |
using the type classes @{class narrowing} and @{class partial_term_of}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2263 |
Variables in the current goal are initially represented as symbolic variables. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2264 |
If the execution of the goal tries to evaluate one of them, the test engine |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2265 |
replaces it with refinements provided by @{const narrowing}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2266 |
Narrowing views every value as a sum-of-products which is expressed using the operations |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2267 |
@{const Quickcheck_Narrowing.cons} (embedding a value), |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2268 |
@{const Quickcheck_Narrowing.apply} (product) and @{const Quickcheck_Narrowing.sum} (sum). |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2269 |
The refinement should enable further evaluation of the goal. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2270 |
|
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2271 |
For example, @{const narrowing} for the list type @{typ "'a :: narrowing list"} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2272 |
can be recursively defined as |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2273 |
@{term "Quickcheck_Narrowing.sum (Quickcheck_Narrowing.cons []) |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2274 |
(Quickcheck_Narrowing.apply |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2275 |
(Quickcheck_Narrowing.apply |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2276 |
(Quickcheck_Narrowing.cons (op #)) |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2277 |
narrowing) |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2278 |
narrowing)"}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2279 |
If a symbolic variable of type @{typ "_ list"} is evaluated, it is replaced by (i)~the empty |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2280 |
list @{term "[]"} and (ii)~by a non-empty list whose head and tail can then be recursively |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2281 |
refined if needed. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2282 |
|
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2283 |
To reconstruct counterexamples, the operation @{const partial_term_of} transforms |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2284 |
@{text narrowing}'s deep representation of terms to the type @{typ Code_Evaluation.term}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2285 |
The deep representation models symbolic variables as |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2286 |
@{const Quickcheck_Narrowing.Narrowing_variable}, which are normally converted to |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2287 |
@{const Code_Evaluation.Free}, and refined values as |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2288 |
@{term "Quickcheck_Narrowing.Narrowing_constructor i args"}, where @{term "i :: integer"} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2289 |
denotes the index in the sum of refinements. In the above example for lists, |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2290 |
@{term "0"} corresponds to @{term "[]"} and @{term "1"} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2291 |
to @{term "op #"}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2292 |
|
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2293 |
The command @{command (HOL) "code_datatype"} sets up @{const partial_term_of} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2294 |
such that the @{term "i"}-th refinement is interpreted as the @{term "i"}-th constructor, |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2295 |
but it does not ensures consistency with @{const narrowing}. |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2296 |
\end{description} |
89e0264adf79
document value generation for quickcheck's testers
Andreas Lochbihler
parents:
56270
diff
changeset
|
2297 |
|
46283 | 2298 |
\item @{command (HOL) "quickcheck_params"} changes @{command (HOL) |
2299 |
"quickcheck"} configuration options persistently. |
|
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2300 |
|
45943
8c4a5e664fbc
adding documentation about the quickcheck_generator command in the IsarRef
bulwahn
parents:
45839
diff
changeset
|
2301 |
\item @{command (HOL) "quickcheck_generator"} creates random and |
46283 | 2302 |
exhaustive value generators for a given type and operations. It |
2303 |
generates values by using the operations as if they were |
|
2304 |
constructors of that type. |
|
45943
8c4a5e664fbc
adding documentation about the quickcheck_generator command in the IsarRef
bulwahn
parents:
45839
diff
changeset
|
2305 |
|
46283 | 2306 |
\item @{command (HOL) "nitpick"} tests the current goal for |
2307 |
counterexamples using a reduction to first-order relational |
|
58552 | 2308 |
logic. See the Nitpick manual @{cite "isabelle-nitpick"} for details. |
42215
de9d43c427ae
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
blanchet
parents:
42123
diff
changeset
|
2309 |
|
46283 | 2310 |
\item @{command (HOL) "nitpick_params"} changes @{command (HOL) |
2311 |
"nitpick"} configuration options persistently. |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2312 |
|
46592
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2313 |
\item @{command (HOL) "find_unused_assms"} finds potentially superfluous |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2314 |
assumptions in theorems using quickcheck. |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2315 |
It takes the theory name to be checked for superfluous assumptions as |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2316 |
optional argument. If not provided, it checks the current theory. |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2317 |
Options to the internal quickcheck invocations can be changed with |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2318 |
common configuration declarations. |
d5d49bd4a7b4
adding documentation about find_unused_assms command and use_subtype option in the IsarRef
bulwahn
parents:
46498
diff
changeset
|
2319 |
|
31912
f5bd306f5e9d
more friendly wrt. PGs interpretation of compound *); added dedicated section on value and quickcheck
haftmann
parents:
31254
diff
changeset
|
2320 |
\end{description} |
58618 | 2321 |
\<close> |
2322 |
||
2323 |
||
2324 |
section \<open>Unstructured case analysis and induction \label{sec:hol-induct-tac}\<close> |
|
2325 |
||
2326 |
text \<open> |
|
27123
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2327 |
The following tools of Isabelle/HOL support cases analysis and |
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2328 |
induction in unstructured tactic scripts; see also |
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2329 |
\secref{sec:cases-induct} for proper Isar versions of similar ideas. |
26849 | 2330 |
|
2331 |
\begin{matharray}{rcl} |
|
28761
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
2332 |
@{method_def (HOL) case_tac}@{text "\<^sup>*"} & : & @{text method} \\ |
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
2333 |
@{method_def (HOL) induct_tac}@{text "\<^sup>*"} & : & @{text method} \\ |
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
2334 |
@{method_def (HOL) ind_cases}@{text "\<^sup>*"} & : & @{text method} \\ |
9ec4482c9201
updated/refined types of Isar language elements, removed special LaTeX macros;
wenzelm
parents:
28760
diff
changeset
|
2335 |
@{command_def (HOL) "inductive_cases"}@{text "\<^sup>*"} & : & @{text "local_theory \<rightarrow> local_theory"} \\ |
26849 | 2336 |
\end{matharray} |
2337 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2338 |
@{rail \<open> |
42705 | 2339 |
@@{method (HOL) case_tac} @{syntax goal_spec}? @{syntax term} rule? |
26849 | 2340 |
; |
42705 | 2341 |
@@{method (HOL) induct_tac} @{syntax goal_spec}? (@{syntax insts} * @'and') rule? |
26849 | 2342 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2343 |
@@{method (HOL) ind_cases} (@{syntax prop}+) (@'for' (@{syntax name}+))? |
26849 | 2344 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2345 |
@@{command (HOL) inductive_cases} (@{syntax thmdecl}? (@{syntax prop}+) + @'and') |
26849 | 2346 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2347 |
rule: 'rule' ':' @{syntax thmref} |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2348 |
\<close>} |
26849 | 2349 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2350 |
\begin{description} |
26849 | 2351 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2352 |
\item @{method (HOL) case_tac} and @{method (HOL) induct_tac} admit |
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2353 |
to reason about inductive types. Rules are selected according to |
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2354 |
the declarations by the @{attribute cases} and @{attribute induct} |
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2355 |
attributes, cf.\ \secref{sec:cases-induct}. The @{command (HOL) |
58310 | 2356 |
datatype} package already takes care of this. |
27123
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2357 |
|
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2358 |
These unstructured tactics feature both goal addressing and dynamic |
26849 | 2359 |
instantiation. Note that named rule cases are \emph{not} provided |
27123
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2360 |
as would be by the proper @{method cases} and @{method induct} proof |
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2361 |
methods (see \secref{sec:cases-induct}). Unlike the @{method |
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2362 |
induct} method, @{method induct_tac} does not handle structured rule |
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2363 |
statements, only the compact object-logic conclusion of the subgoal |
11fcdd5897dd
case_tac/induct_tac: use same declarations as cases/induct;
wenzelm
parents:
27103
diff
changeset
|
2364 |
being addressed. |
42123 | 2365 |
|
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2366 |
\item @{method (HOL) ind_cases} and @{command (HOL) |
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2367 |
"inductive_cases"} provide an interface to the internal @{ML_text |
26860 | 2368 |
mk_cases} operation. Rules are simplified in an unrestricted |
2369 |
forward manner. |
|
26849 | 2370 |
|
2371 |
While @{method (HOL) ind_cases} is a proof method to apply the |
|
2372 |
result immediately as elimination rules, @{command (HOL) |
|
2373 |
"inductive_cases"} provides case split theorems at the theory level |
|
2374 |
for later use. The @{keyword "for"} argument of the @{method (HOL) |
|
2375 |
ind_cases} method allows to specify a list of variables that should |
|
2376 |
be generalized before applying the resulting rule. |
|
2377 |
||
28760
cbc435f7b16b
unified use of declaration environment with IsarImplementation;
wenzelm
parents:
28752
diff
changeset
|
2378 |
\end{description} |
58618 | 2379 |
\<close> |
2380 |
||
2381 |
||
2382 |
chapter \<open>Executable code\<close> |
|
2383 |
||
2384 |
text \<open>For validation purposes, it is often useful to \emph{execute} |
|
42627
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2385 |
specifications. In principle, execution could be simulated by |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2386 |
Isabelle's inference kernel, i.e. by a combination of resolution and |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2387 |
simplification. Unfortunately, this approach is rather inefficient. |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2388 |
A more efficient way of executing specifications is to translate |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2389 |
them into a functional programming language such as ML. |
26849 | 2390 |
|
45192 | 2391 |
Isabelle provides a generic framework to support code generation |
42627
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2392 |
from executable specifications. Isabelle/HOL instantiates these |
45192 | 2393 |
mechanisms in a way that is amenable to end-user applications. Code |
2394 |
can be generated for functional programs (including overloading |
|
58552 | 2395 |
using type classes) targeting SML @{cite SML}, OCaml @{cite OCaml}, |
2396 |
Haskell @{cite "haskell-revised-report"} and Scala |
|
2397 |
@{cite "scala-overview-tech-report"}. Conceptually, code generation is |
|
42627
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2398 |
split up in three steps: \emph{selection} of code theorems, |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2399 |
\emph{translation} into an abstract executable view and |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2400 |
\emph{serialization} to a specific \emph{target language}. |
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2401 |
Inductive specifications can be executed using the predicate |
58552 | 2402 |
compiler which operates within HOL. See @{cite "isabelle-codegen"} for |
42627
8749742785b8
moved material about old codegen to isar-ref manual;
wenzelm
parents:
42626
diff
changeset
|
2403 |
an introduction. |
37422 | 2404 |
|
2405 |
\begin{matharray}{rcl} |
|
2406 |
@{command_def (HOL) "export_code"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
|
2407 |
@{attribute_def (HOL) code} & : & @{text attribute} \\ |
|
2408 |
@{command_def (HOL) "code_datatype"} & : & @{text "theory \<rightarrow> theory"} \\ |
|
2409 |
@{command_def (HOL) "print_codesetup"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
|
45232
eb56e1774c26
updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
bulwahn
parents:
45192
diff
changeset
|
2410 |
@{attribute_def (HOL) code_unfold} & : & @{text attribute} \\ |
37422 | 2411 |
@{attribute_def (HOL) code_post} & : & @{text attribute} \\ |
46028
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2412 |
@{attribute_def (HOL) code_abbrev} & : & @{text attribute} \\ |
37422 | 2413 |
@{command_def (HOL) "print_codeproc"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
2414 |
@{command_def (HOL) "code_thms"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
|
2415 |
@{command_def (HOL) "code_deps"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\ |
|
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2416 |
@{command_def (HOL) "code_reserved"} & : & @{text "theory \<rightarrow> theory"} \\ |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2417 |
@{command_def (HOL) "code_printing"} & : & @{text "theory \<rightarrow> theory"} \\ |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2418 |
@{command_def (HOL) "code_identifier"} & : & @{text "theory \<rightarrow> theory"} \\ |
37422 | 2419 |
@{command_def (HOL) "code_monad"} & : & @{text "theory \<rightarrow> theory"} \\ |
45408
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2420 |
@{command_def (HOL) "code_reflect"} & : & @{text "theory \<rightarrow> theory"} \\ |
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2421 |
@{command_def (HOL) "code_pred"} & : & @{text "theory \<rightarrow> proof(prove)"} |
37422 | 2422 |
\end{matharray} |
2423 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2424 |
@{rail \<open> |
55686
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2425 |
@@{command (HOL) export_code} ( @'open' ) ? ( constexpr + ) \<newline> |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2426 |
( ( @'in' target ( @'module_name' @{syntax string} ) ? \<newline> |
52435
6646bb548c6b
migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
haftmann
parents:
52378
diff
changeset
|
2427 |
( @'file' @{syntax string} ) ? ( '(' args ')' ) ?) + ) ? |
37422 | 2428 |
; |
2429 |
||
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2430 |
const: @{syntax term} |
37422 | 2431 |
; |
2432 |
||
40711
81bc73585eec
globbing constant expressions use more idiomatic underscore rather than star
haftmann
parents:
40709
diff
changeset
|
2433 |
constexpr: ( const | 'name._' | '_' ) |
37422 | 2434 |
; |
2435 |
||
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2436 |
typeconstructor: @{syntax nameref} |
37422 | 2437 |
; |
2438 |
||
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2439 |
class: @{syntax nameref} |
37422 | 2440 |
; |
2441 |
||
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2442 |
target: 'SML' | 'OCaml' | 'Haskell' | 'Scala' | 'Eval' |
37422 | 2443 |
; |
2444 |
||
54890
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2445 |
@@{attribute (HOL) code} ( 'del' | 'equation' | 'abstype' | 'abstract' |
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2446 |
| 'drop:' ( const + ) | 'abort:' ( const + ) )? |
37422 | 2447 |
; |
2448 |
||
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2449 |
@@{command (HOL) code_datatype} ( const + ) |
37422 | 2450 |
; |
2451 |
||
45232
eb56e1774c26
updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
bulwahn
parents:
45192
diff
changeset
|
2452 |
@@{attribute (HOL) code_unfold} ( 'del' ) ? |
37422 | 2453 |
; |
2454 |
||
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2455 |
@@{attribute (HOL) code_post} ( 'del' ) ? |
37422 | 2456 |
; |
2457 |
||
46028
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2458 |
@@{attribute (HOL) code_abbrev} |
45232
eb56e1774c26
updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
bulwahn
parents:
45192
diff
changeset
|
2459 |
; |
eb56e1774c26
updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
bulwahn
parents:
45192
diff
changeset
|
2460 |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2461 |
@@{command (HOL) code_thms} ( constexpr + ) ? |
37422 | 2462 |
; |
2463 |
||
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2464 |
@@{command (HOL) code_deps} ( constexpr + ) ? |
37422 | 2465 |
; |
2466 |
||
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2467 |
@@{command (HOL) code_reserved} target ( @{syntax string} + ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2468 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2469 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2470 |
symbol_const: ( @'constant' const ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2471 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2472 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2473 |
symbol_typeconstructor: ( @'type_constructor' typeconstructor ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2474 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2475 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2476 |
symbol_class: ( @'type_class' class ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2477 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2478 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2479 |
symbol_class_relation: ( @'class_relation' class ( '<' | '\<subseteq>' ) class ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2480 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2481 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2482 |
symbol_class_instance: ( @'class_instance' typeconstructor @'::' class ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2483 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2484 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2485 |
symbol_module: ( @'code_module' name ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2486 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2487 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2488 |
syntax: @{syntax string} | ( @'infix' | @'infixl' | @'infixr' ) @{syntax nat} @{syntax string} |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2489 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2490 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2491 |
printing_const: symbol_const ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2492 |
( '(' target ')' syntax ? + @'and' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2493 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2494 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2495 |
printing_typeconstructor: symbol_typeconstructor ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2496 |
( '(' target ')' syntax ? + @'and' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2497 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2498 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2499 |
printing_class: symbol_class ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2500 |
( '(' target ')' @{syntax string} ? + @'and' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2501 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2502 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2503 |
printing_class_relation: symbol_class_relation ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2504 |
( '(' target ')' @{syntax string} ? + @'and' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2505 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2506 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2507 |
printing_class_instance: symbol_class_instance ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2508 |
( '(' target ')' '-' ? + @'and' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2509 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2510 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2511 |
printing_module: symbol_module ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2512 |
( '(' target ')' ( @{syntax string} ( @'attach' ( const + ) ) ? ) ? + @'and' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2513 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2514 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2515 |
@@{command (HOL) code_printing} ( ( printing_const | printing_typeconstructor |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2516 |
| printing_class | printing_class_relation | printing_class_instance |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2517 |
| printing_module ) + '|' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2518 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2519 |
|
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2520 |
@@{command (HOL) code_identifier} ( ( symbol_const | symbol_typeconstructor |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2521 |
| symbol_class | symbol_class_relation | symbol_class_instance |
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2522 |
| symbol_module ) ( '\<rightharpoonup>' | '=>' ) \<newline> |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2523 |
( '(' target ')' @{syntax string} ? + @'and' ) + '|' ) |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2524 |
; |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2525 |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2526 |
@@{command (HOL) code_monad} const const target |
37422 | 2527 |
; |
2528 |
||
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2529 |
@@{command (HOL) code_reflect} @{syntax string} \<newline> |
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2530 |
( @'datatypes' ( @{syntax string} '=' ( '_' | ( @{syntax string} + '|' ) + @'and' ) ) ) ? \<newline> |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
42215
diff
changeset
|
2531 |
( @'functions' ( @{syntax string} + ) ) ? ( @'file' @{syntax string} ) ? |
37422 | 2532 |
; |
2533 |
||
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2534 |
@@{command (HOL) code_pred} \<newline> ('(' @'modes' ':' modedecl ')')? \<newline> const |
45408
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2535 |
; |
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2536 |
|
55029
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2537 |
modedecl: (modes | ((const ':' modes) \<newline> |
61a6bf7d4b02
clarified @{rail} syntax: prefer explicit \<newline> symbol;
wenzelm
parents:
54890
diff
changeset
|
2538 |
(@'and' ((const ':' modes @'and') +))?)) |
45408
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2539 |
; |
47859 | 2540 |
|
45408
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2541 |
modes: mode @'as' const |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
2542 |
\<close>} |
37422 | 2543 |
|
2544 |
\begin{description} |
|
2545 |
||
2546 |
\item @{command (HOL) "export_code"} generates code for a given list |
|
39608 | 2547 |
of constants in the specified target language(s). If no |
2548 |
serialization instruction is given, only abstract code is generated |
|
2549 |
internally. |
|
37422 | 2550 |
|
2551 |
Constants may be specified by giving them literally, referring to |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
2552 |
all executable constants within a certain theory by giving @{text |
55686
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2553 |
"name._"}, or referring to \emph{all} executable constants currently |
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2554 |
available by giving @{text "_"}. |
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2555 |
|
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2556 |
By default, exported identifiers are minimized per module. This |
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2557 |
can be suppressed by prepending @{keyword "open"} before the list |
e99ed112d303
NEWS and documentation, including correction of long-overseen "*"
haftmann
parents:
55677
diff
changeset
|
2558 |
of contants. |
37422 | 2559 |
|
2560 |
By default, for each involved theory one corresponding name space |
|
52895
a806aa7a5370
some documentation for adhoc overloading;
Christian Sternagel
parents:
52637
diff
changeset
|
2561 |
module is generated. Alternatively, a module name may be specified |
37422 | 2562 |
after the @{keyword "module_name"} keyword; then \emph{all} code is |
2563 |
placed in this module. |
|
2564 |
||
39608 | 2565 |
For \emph{SML}, \emph{OCaml} and \emph{Scala} the file specification |
2566 |
refers to a single file; for \emph{Haskell}, it refers to a whole |
|
2567 |
directory, where code is generated in multiple files reflecting the |
|
2568 |
module hierarchy. Omitting the file specification denotes standard |
|
37749 | 2569 |
output. |
37422 | 2570 |
|
55677 | 2571 |
Serializers take an optional list of arguments in parentheses. |
39608 | 2572 |
For \emph{Haskell} a module name prefix may be given using the |
2573 |
``@{text "root:"}'' argument; ``@{text string_classes}'' adds a |
|
2574 |
``@{verbatim "deriving (Read, Show)"}'' clause to each appropriate |
|
2575 |
datatype declaration. |
|
37422 | 2576 |
|
52637
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2577 |
\item @{attribute (HOL) code} declare code equations for code |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2578 |
generation. Variant @{text "code equation"} declares a conventional |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2579 |
equation as code equation. Variants @{text "code abstype"} and |
38462
34d3de1254cd
formally document `code abstype` and `code abstract` attributes
haftmann
parents:
37820
diff
changeset
|
2580 |
@{text "code abstract"} declare abstract datatype certificates or |
34d3de1254cd
formally document `code abstype` and `code abstract` attributes
haftmann
parents:
37820
diff
changeset
|
2581 |
code equations on abstract datatype representations respectively. |
52637
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2582 |
Vanilla @{text "code"} falls back to @{text "code equation"} |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2583 |
or @{text "code abstype"} depending on the syntactic shape |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2584 |
of the underlying equation. Variant @{text "code del"} |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2585 |
deselects a code equation for code generation. |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2586 |
|
54890
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2587 |
Variants @{text "code drop:"} and @{text "code abort:"} take |
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2588 |
a list of constant as arguments and drop all code equations declared |
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2589 |
for them. In the case of {text abort}, these constants then are |
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2590 |
are not required to have a definition by means of code equations; |
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2591 |
if needed these are implemented by program abort (exception) instead. |
cb892d835803
fundamental treatment of undefined vs. universally partial replaces code_abort
haftmann
parents:
54338
diff
changeset
|
2592 |
|
52637
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2593 |
Usually packages introducing code equations provide a reasonable |
1501ebe39711
attribute "code" declares concrete and abstract code equations uniformly; added explicit "code equation" instead
haftmann
parents:
52476
diff
changeset
|
2594 |
default setup for selection. |
37422 | 2595 |
|
2596 |
\item @{command (HOL) "code_datatype"} specifies a constructor set |
|
2597 |
for a logical type. |
|
2598 |
||
2599 |
\item @{command (HOL) "print_codesetup"} gives an overview on |
|
2600 |
selected code equations and code generator datatypes. |
|
2601 |
||
45232
eb56e1774c26
updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
bulwahn
parents:
45192
diff
changeset
|
2602 |
\item @{attribute (HOL) code_unfold} declares (or with option |
46028
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2603 |
``@{text "del"}'' removes) theorems which during preprocessing |
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2604 |
are applied as rewrite rules to any code equation or evaluation |
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2605 |
input. |
37422 | 2606 |
|
39608 | 2607 |
\item @{attribute (HOL) code_post} declares (or with option ``@{text |
2608 |
"del"}'' removes) theorems which are applied as rewrite rules to any |
|
2609 |
result of an evaluation. |
|
37422 | 2610 |
|
56929 | 2611 |
\item @{attribute (HOL) code_abbrev} declares (or with option ``@{text |
2612 |
"del"}'' removes) equations which are |
|
46028
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2613 |
applied as rewrite rules to any result of an evaluation and |
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2614 |
symmetrically during preprocessing to any code equation or evaluation |
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2615 |
input. |
9f113cdf3d66
attribute code_abbrev superseedes code_unfold_post
haftmann
parents:
45944
diff
changeset
|
2616 |
|
39608 | 2617 |
\item @{command (HOL) "print_codeproc"} prints the setup of the code |
2618 |
generator preprocessor. |
|
37422 | 2619 |
|
2620 |
\item @{command (HOL) "code_thms"} prints a list of theorems |
|
2621 |
representing the corresponding program containing all given |
|
2622 |
constants after preprocessing. |
|
2623 |
||
2624 |
\item @{command (HOL) "code_deps"} visualizes dependencies of |
|
2625 |
theorems representing the corresponding program containing all given |
|
2626 |
constants after preprocessing. |
|
2627 |
||
2628 |
\item @{command (HOL) "code_reserved"} declares a list of names as |
|
2629 |
reserved for a given target, preventing it to be shadowed by any |
|
2630 |
generated code. |
|
2631 |
||
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2632 |
\item @{command (HOL) "code_printing"} associates a series of symbols |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2633 |
(constants, type constructors, classes, class relations, instances, |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2634 |
module names) with target-specific serializations; omitting a serialization |
55372 | 2635 |
deletes an existing serialization. |
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2636 |
|
37422 | 2637 |
\item @{command (HOL) "code_monad"} provides an auxiliary mechanism |
2638 |
to generate monadic code for Haskell. |
|
2639 |
||
52378
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2640 |
\item @{command (HOL) "code_identifier"} associates a a series of symbols |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2641 |
(constants, type constructors, classes, class relations, instances, |
08dbf9ff2140
documentation on code_printing and code_identifier
haftmann
parents:
50879
diff
changeset
|
2642 |
module names) with target-specific hints how these symbols shall be named. |
55293
42cf5802d36a
code generation: explicitly declared identifiers gain predence over implicit ones
haftmann
parents:
55112
diff
changeset
|
2643 |
These hints gain precedence over names for symbols with no hints at all. |
42cf5802d36a
code generation: explicitly declared identifiers gain predence over implicit ones
haftmann
parents:
55112
diff
changeset
|
2644 |
Conflicting hints are subject to name disambiguation. |
42cf5802d36a
code generation: explicitly declared identifiers gain predence over implicit ones
haftmann
parents:
55112
diff
changeset
|
2645 |
\emph{Warning:} It is at the discretion |
52476 | 2646 |
of the user to ensure that name prefixes of identifiers in compound |
2647 |
statements like type classes or datatypes are still the same. |
|
37422 | 2648 |
|
39608 | 2649 |
\item @{command (HOL) "code_reflect"} without a ``@{text "file"}'' |
2650 |
argument compiles code into the system runtime environment and |
|
2651 |
modifies the code generator setup that future invocations of system |
|
2652 |
runtime code generation referring to one of the ``@{text |
|
47859 | 2653 |
"datatypes"}'' or ``@{text "functions"}'' entities use these |
2654 |
precompiled entities. With a ``@{text "file"}'' argument, the |
|
2655 |
corresponding code is generated into that specified file without |
|
2656 |
modifying the code generator setup. |
|
2657 |
||
2658 |
\item @{command (HOL) "code_pred"} creates code equations for a |
|
2659 |
predicate given a set of introduction rules. Optional mode |
|
2660 |
annotations determine which arguments are supposed to be input or |
|
2661 |
output. If alternative introduction rules are declared, one must |
|
2662 |
prove a corresponding elimination rule. |
|
45408
7156f63ce3c2
adding a minimal documentation about the code_pred command to the isar reference
bulwahn
parents:
45232
diff
changeset
|
2663 |
|
37422 | 2664 |
\end{description} |
58618 | 2665 |
\<close> |
37422 | 2666 |
|
26840 | 2667 |
end |