8745
|
1 |
(*<*)
|
9792
|
2 |
theory Nested = ABexpr:
|
8745
|
3 |
(*>*)
|
|
4 |
|
|
5 |
text{*
|
|
6 |
So far, all datatypes had the property that on the right-hand side of their
|
|
7 |
definition they occurred only at the top-level, i.e.\ directly below a
|
|
8 |
constructor. This is not the case any longer for the following model of terms
|
|
9 |
where function symbols can be applied to a list of arguments:
|
|
10 |
*}
|
9933
|
11 |
(*<*)hide const Var(*>*)
|
8745
|
12 |
datatype ('a,'b)"term" = Var 'a | App 'b "('a,'b)term list";
|
|
13 |
|
|
14 |
text{*\noindent
|
9792
|
15 |
Note that we need to quote @{text"term"} on the left to avoid confusion with
|
8745
|
16 |
the command \isacommand{term}.
|
9792
|
17 |
Parameter @{typ"'a"} is the type of variables and @{typ"'b"} the type of
|
8745
|
18 |
function symbols.
|
9541
|
19 |
A mathematical term like $f(x,g(y))$ becomes @{term"App f [Var x, App g
|
9792
|
20 |
[Var y]]"}, where @{term"f"}, @{term"g"}, @{term"x"}, @{term"y"} are
|
8745
|
21 |
suitable values, e.g.\ numbers or strings.
|
|
22 |
|
9792
|
23 |
What complicates the definition of @{text"term"} is the nested occurrence of
|
|
24 |
@{text"term"} inside @{text"list"} on the right-hand side. In principle,
|
8745
|
25 |
nested recursion can be eliminated in favour of mutual recursion by unfolding
|
9792
|
26 |
the offending datatypes, here @{text"list"}. The result for @{text"term"}
|
8745
|
27 |
would be something like
|
8751
|
28 |
\medskip
|
|
29 |
|
|
30 |
\input{Datatype/document/unfoldnested.tex}
|
|
31 |
\medskip
|
|
32 |
|
|
33 |
\noindent
|
8745
|
34 |
Although we do not recommend this unfolding to the user, it shows how to
|
|
35 |
simulate nested recursion by mutual recursion.
|
9792
|
36 |
Now we return to the initial definition of @{text"term"} using
|
8745
|
37 |
nested recursion.
|
|
38 |
|
|
39 |
Let us define a substitution function on terms. Because terms involve term
|
|
40 |
lists, we need to define two substitution functions simultaneously:
|
|
41 |
*}
|
|
42 |
|
|
43 |
consts
|
|
44 |
subst :: "('a\\<Rightarrow>('a,'b)term) \\<Rightarrow> ('a,'b)term \\<Rightarrow> ('a,'b)term"
|
|
45 |
substs:: "('a\\<Rightarrow>('a,'b)term) \\<Rightarrow> ('a,'b)term list \\<Rightarrow> ('a,'b)term list";
|
|
46 |
|
|
47 |
primrec
|
|
48 |
"subst s (Var x) = s x"
|
9644
|
49 |
subst_App:
|
8745
|
50 |
"subst s (App f ts) = App f (substs s ts)"
|
|
51 |
|
|
52 |
"substs s [] = []"
|
|
53 |
"substs s (t # ts) = subst s t # substs s ts";
|
|
54 |
|
|
55 |
text{*\noindent
|
9933
|
56 |
(Please ignore the label @{thm[source]subst_App} for the moment.)
|
9644
|
57 |
|
8745
|
58 |
Similarly, when proving a statement about terms inductively, we need
|
|
59 |
to prove a related statement about term lists simultaneously. For example,
|
|
60 |
the fact that the identity substitution does not change a term needs to be
|
|
61 |
strengthened and proved as follows:
|
|
62 |
*}
|
|
63 |
|
|
64 |
lemma "subst Var t = (t ::('a,'b)term) \\<and>
|
|
65 |
substs Var ts = (ts::('a,'b)term list)";
|
9689
|
66 |
by(induct_tac t and ts, simp_all);
|
8745
|
67 |
|
|
68 |
text{*\noindent
|
9792
|
69 |
Note that @{term"Var"} is the identity substitution because by definition it
|
|
70 |
leaves variables unchanged: @{prop"subst Var (Var x) = Var x"}. Note also
|
8745
|
71 |
that the type annotations are necessary because otherwise there is nothing in
|
|
72 |
the goal to enforce that both halves of the goal talk about the same type
|
9792
|
73 |
parameters @{text"('a,'b)"}. As a result, induction would fail
|
8745
|
74 |
because the two halves of the goal would be unrelated.
|
|
75 |
|
|
76 |
\begin{exercise}
|
|
77 |
The fact that substitution distributes over composition can be expressed
|
|
78 |
roughly as follows:
|
9792
|
79 |
@{text[display]"subst (f o g) t = subst f (subst g t)"}
|
8745
|
80 |
Correct this statement (you will find that it does not type-check),
|
9792
|
81 |
strengthen it, and prove it. (Note: \isaindexbold{o} is function composition;
|
|
82 |
its definition is found in theorem @{thm[source]o_def}).
|
8745
|
83 |
\end{exercise}
|
9644
|
84 |
\begin{exercise}\label{ex:trev-trev}
|
9792
|
85 |
Define a function @{text"trev"} of type @{typ"('a,'b)term => ('a,'b)term"}
|
|
86 |
that recursively reverses the order of arguments of all function symbols in a
|
|
87 |
term. Prove that @{prop"trev(trev t) = t"}.
|
9644
|
88 |
\end{exercise}
|
|
89 |
|
|
90 |
The experienced functional programmer may feel that our above definition of
|
9792
|
91 |
@{term"subst"} is unnecessarily complicated in that @{term"substs"} is
|
|
92 |
completely unnecessary. The @{term"App"}-case can be defined directly as
|
9644
|
93 |
@{term[display]"subst s (App f ts) = App f (map (subst s) ts)"}
|
|
94 |
where @{term"map"} is the standard list function such that
|
9792
|
95 |
@{text"map f [x1,...,xn] = [f x1,...,f xn]"}. This is true, but Isabelle
|
|
96 |
insists on the above fixed format. Fortunately, we can easily \emph{prove}
|
|
97 |
that the suggested equation holds:
|
9644
|
98 |
*}
|
|
99 |
|
|
100 |
lemma [simp]: "subst s (App f ts) = App f (map (subst s) ts)"
|
9689
|
101 |
by(induct_tac ts, simp_all)
|
9644
|
102 |
|
9689
|
103 |
text{*\noindent
|
9644
|
104 |
What is more, we can now disable the old defining equation as a
|
|
105 |
simplification rule:
|
|
106 |
*}
|
|
107 |
|
9933
|
108 |
declare subst_App [simp del]
|
9644
|
109 |
|
|
110 |
text{*\noindent
|
9689
|
111 |
The advantage is that now we have replaced @{term"substs"} by
|
|
112 |
@{term"map"}, we can profit from the large number of pre-proved lemmas
|
|
113 |
about @{term"map"}. Unfortunately inductive proofs about type
|
9792
|
114 |
@{text"term"} are still awkward because they expect a conjunction. One
|
9689
|
115 |
could derive a new induction principle as well (see
|
|
116 |
\S\ref{sec:derive-ind}), but turns out to be simpler to define
|
|
117 |
functions by \isacommand{recdef} instead of \isacommand{primrec}.
|
|
118 |
The details are explained in \S\ref{sec:advanced-recdef} below.
|
8745
|
119 |
|
|
120 |
Of course, you may also combine mutual and nested recursion. For example,
|
9792
|
121 |
constructor @{text"Sum"} in \S\ref{sec:datatype-mut-rec} could take a list of
|
|
122 |
expressions as its argument: @{text"Sum"}~@{typ[quotes]"'a aexp list"}.
|
8745
|
123 |
*}
|
|
124 |
(*<*)
|
|
125 |
end
|
|
126 |
(*>*)
|