127
+ − 1
theory Ind_Prelims
244
+ − 2
imports Main "../Base"
32
+ − 3
begin
+ − 4
127
+ − 5
section{* Preliminaries *}
+ − 6
32
+ − 7
text {*
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 8
The user will just give a specification of inductive predicate(s) and
129
+ − 9
expects from the package to produce a convenient reasoning
+ − 10
infrastructure. This infrastructure needs to be derived from the definition
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 11
that correspond to the specified predicate(s). Before we start with
219
+ − 12
explaining all parts of the package, let us first give some examples
+ − 13
showing how to define inductive predicates and then also how
+ − 14
to generate a reasoning infrastructure for them. From the examples
+ − 15
we will figure out a general method for
+ − 16
defining inductive predicates. The aim in this section is \emph{not} to
+ − 17
write proofs that are as beautiful as possible, but as close as possible to
244
+ − 18
the ML-implementation we will develop in later sections.
219
+ − 19
+ − 20
We first consider the transitive closure of a relation @{text R}. The
+ − 21
``pencil-and-paper'' specification for the transitive closure is:
+ − 22
127
+ − 23
\begin{center}\small
116
+ − 24
@{prop[mode=Axiom] "trcl R x x"} \hspace{5mm}
+ − 25
@{prop[mode=Rule] "R x y \<Longrightarrow> trcl R y z \<Longrightarrow> trcl R x z"}
88
+ − 26
\end{center}
+ − 27
224
+ − 28
The package has to make an appropriate definition for @{term "trcl"}.
+ − 29
Since an inductively
127
+ − 30
defined predicate is the least predicate closed under a collection of
+ − 31
introduction rules, the predicate @{text "trcl R x y"} can be defined so
+ − 32
that it holds if and only if @{text "P x y"} holds for every predicate
+ − 33
@{text P} closed under the rules above. This gives rise to the definition
32
+ − 34
*}
+ − 35
127
+ − 36
definition "trcl \<equiv>
+ − 37
\<lambda>R x y. \<forall>P. (\<forall>x. P x x)
+ − 38
\<longrightarrow> (\<forall>x y z. R x y \<longrightarrow> P y z \<longrightarrow> P x z) \<longrightarrow> P x y"
32
+ − 39
+ − 40
text {*
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 41
We have to use the object implication @{text "\<longrightarrow>"} and object quantification
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 42
@{text "\<forall>"} for stating this definition (there is no other way for
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 43
definitions in HOL). However, the introduction rules and induction
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 44
principles associated with the transitive closure should use the meta-connectives,
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 45
since they simplify the reasoning for the user.
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 46
32
+ − 47
127
+ − 48
With this definition, the proof of the induction principle for @{term trcl}
129
+ − 49
is almost immediate. It suffices to convert all the meta-level
116
+ − 50
connectives in the lemma to object-level connectives using the
219
+ − 51
proof method @{text atomize} (Line 4 below), expand the definition of @{term trcl}
127
+ − 52
(Line 5 and 6), eliminate the universal quantifier contained in it (Line~7),
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 53
and then solve the goal by @{text assumption} (Line 8).
113
+ − 54
32
+ − 55
*}
+ − 56
114
+ − 57
lemma %linenos trcl_induct:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 58
assumes "trcl R x y"
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 59
shows "(\<And>x. P x x) \<Longrightarrow> (\<And>x y z. R x y \<Longrightarrow> P y z \<Longrightarrow> P x z) \<Longrightarrow> P x y"
113
+ − 60
apply(atomize (full))
165
+ − 61
apply(cut_tac prems)
113
+ − 62
apply(unfold trcl_def)
+ − 63
apply(drule spec[where x=P])
+ − 64
apply(assumption)
+ − 65
done
88
+ − 66
113
+ − 67
text {*
127
+ − 68
The proofs for the introduction rules are slightly more complicated.
+ − 69
For the first one, we need to prove the following lemma:
+ − 70
*}
+ − 71
+ − 72
lemma %linenos trcl_base:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 73
shows "trcl R x x"
127
+ − 74
apply(unfold trcl_def)
+ − 75
apply(rule allI impI)+
+ − 76
apply(drule spec)
+ − 77
apply(assumption)
+ − 78
done
+ − 79
+ − 80
text {*
+ − 81
We again unfold first the definition and apply introduction rules
+ − 82
for @{text "\<forall>"} and @{text "\<longrightarrow>"} as often as possible (Lines 3 and 4).
116
+ − 83
We then end up in the goal state:
113
+ − 84
*}
88
+ − 85
113
+ − 86
(*<*)lemma "trcl R x x"
115
+ − 87
apply (unfold trcl_def)
+ − 88
apply (rule allI impI)+(*>*)
113
+ − 89
txt {* @{subgoals [display]} *}
32
+ − 90
(*<*)oops(*>*)
88
+ − 91
113
+ − 92
text {*
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 93
The two assumptions come from the definition of @{term trcl} and correspond
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 94
to the introduction rules. Thus, all we have to do is to eliminate the
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 95
universal quantifier in front of the first assumption (Line 5), and then
219
+ − 96
solve the goal by @{text assumption} (Line 6).
113
+ − 97
*}
+ − 98
+ − 99
text {*
127
+ − 100
Next we have to show that the second introduction rule also follows from the
+ − 101
definition. Since this rule has premises, the proof is a bit more
+ − 102
involved. After unfolding the definitions and applying the introduction
+ − 103
rules for @{text "\<forall>"} and @{text "\<longrightarrow>"}
113
+ − 104
*}
+ − 105
127
+ − 106
lemma trcl_step:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 107
shows "R x y \<Longrightarrow> trcl R y z \<Longrightarrow> trcl R x z"
115
+ − 108
apply (unfold trcl_def)
127
+ − 109
apply (rule allI impI)+
113
+ − 110
127
+ − 111
txt {*
+ − 112
we obtain the goal state
+ − 113
+ − 114
@{subgoals [display]}
+ − 115
+ − 116
To see better where we are, let us explicitly name the assumptions
+ − 117
by starting a subproof.
115
+ − 118
*}
+ − 119
+ − 120
proof -
+ − 121
case (goal1 P)
127
+ − 122
have p1: "R x y" by fact
+ − 123
have p2: "\<forall>P. (\<forall>x. P x x)
+ − 124
\<longrightarrow> (\<forall>x y z. R x y \<longrightarrow> P y z \<longrightarrow> P x z) \<longrightarrow> P y z" by fact
+ − 125
have r1: "\<forall>x. P x x" by fact
+ − 126
have r2: "\<forall>x y z. R x y \<longrightarrow> P y z \<longrightarrow> P x z" by fact
+ − 127
show "P x z"
+ − 128
+ − 129
txt {*
+ − 130
The assumptions @{text "p1"} and @{text "p2"} correspond to the premises of
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 131
the second introduction rule (unfolded); the assumptions @{text "r1"} and @{text "r2"}
219
+ − 132
come from the definition of @{term trcl}. We apply @{text "r2"} to the goal
+ − 133
@{term "P x z"}. In order for this assumption to be applicable as a rule, we
127
+ − 134
have to eliminate the universal quantifier and turn the object-level
+ − 135
implications into meta-level ones. This can be accomplished using the @{text
+ − 136
rule_format} attribute. So we continue the proof with:
115
+ − 137
32
+ − 138
*}
113
+ − 139
127
+ − 140
apply (rule r2[rule_format])
88
+ − 141
127
+ − 142
txt {*
+ − 143
This gives us two new subgoals
+ − 144
+ − 145
@{subgoals [display]}
+ − 146
+ − 147
which can be solved using assumptions @{text p1} and @{text p2}. The latter
+ − 148
involves a quantifier and implications that have to be eliminated before it
+ − 149
can be applied. To avoid potential problems with higher-order unification,
+ − 150
we explicitly instantiate the quantifier to @{text "P"} and also match
+ − 151
explicitly the implications with @{text "r1"} and @{text "r2"}. This gives
+ − 152
the proof:
+ − 153
*}
+ − 154
+ − 155
apply(rule p1)
+ − 156
apply(rule p2[THEN spec[where x=P], THEN mp, THEN mp, OF r1, OF r2])
115
+ − 157
done
+ − 158
qed
32
+ − 159
+ − 160
text {*
127
+ − 161
Now we are done. It might be surprising that we are not using the automatic
244
+ − 162
tactics available in Isabelle/HOL for proving this lemmas. After all @{text
127
+ − 163
"blast"} would easily dispense of it.
115
+ − 164
*}
88
+ − 165
127
+ − 166
lemma trcl_step_blast:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 167
shows "R x y \<Longrightarrow> trcl R y z \<Longrightarrow> trcl R x z"
115
+ − 168
apply(unfold trcl_def)
+ − 169
apply(blast)
+ − 170
done
+ − 171
+ − 172
text {*
116
+ − 173
Experience has shown that it is generally a bad idea to rely heavily on
+ − 174
@{text blast}, @{text auto} and the like in automated proofs. The reason is
+ − 175
that you do not have precise control over them (the user can, for example,
+ − 176
declare new intro- or simplification rules that can throw automatic tactics
+ − 177
off course) and also it is very hard to debug proofs involving automatic
+ − 178
tactics whenever something goes wrong. Therefore if possible, automatic
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 179
tactics should be avoided or be constrained sufficiently.
115
+ − 180
116
+ − 181
The method of defining inductive predicates by impredicative quantification
+ − 182
also generalises to mutually inductive predicates. The next example defines
219
+ − 183
the predicates @{text even} and @{text odd} given by
32
+ − 184
219
+ − 185
\begin{center}\small
+ − 186
@{prop[mode=Axiom] "even (0::nat)"} \hspace{5mm}
+ − 187
@{prop[mode=Rule] "odd n \<Longrightarrow> even (Suc n)"} \hspace{5mm}
+ − 188
@{prop[mode=Rule] "even n \<Longrightarrow> odd (Suc n)"}
+ − 189
\end{center}
32
+ − 190
127
+ − 191
Since the predicates @{term even} and @{term odd} are mutually inductive, each
+ − 192
corresponding definition must quantify over both predicates (we name them
+ − 193
below @{text "P"} and @{text "Q"}).
+ − 194
*}
+ − 195
219
+ − 196
definition "even \<equiv>
127
+ − 197
\<lambda>n. \<forall>P Q. P 0 \<longrightarrow> (\<forall>m. Q m \<longrightarrow> P (Suc m))
+ − 198
\<longrightarrow> (\<forall>m. P m \<longrightarrow> Q (Suc m)) \<longrightarrow> P n"
+ − 199
219
+ − 200
definition "odd \<equiv>
127
+ − 201
\<lambda>n. \<forall>P Q. P 0 \<longrightarrow> (\<forall>m. Q m \<longrightarrow> P (Suc m))
+ − 202
\<longrightarrow> (\<forall>m. P m \<longrightarrow> Q (Suc m)) \<longrightarrow> Q n"
32
+ − 203
+ − 204
text {*
116
+ − 205
For proving the induction principles, we use exactly the same technique
+ − 206
as in the transitive closure example, namely:
32
+ − 207
*}
+ − 208
+ − 209
lemma even_induct:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 210
assumes "even n"
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 211
shows "P 0 \<Longrightarrow> (\<And>m. Q m \<Longrightarrow> P (Suc m)) \<Longrightarrow> (\<And>m. P m \<Longrightarrow> Q (Suc m)) \<Longrightarrow> P n"
115
+ − 212
apply(atomize (full))
165
+ − 213
apply(cut_tac prems)
115
+ − 214
apply(unfold even_def)
+ − 215
apply(drule spec[where x=P])
+ − 216
apply(drule spec[where x=Q])
+ − 217
apply(assumption)
+ − 218
done
32
+ − 219
+ − 220
text {*
127
+ − 221
The only difference with the proof @{text "trcl_induct"} is that we have to
+ − 222
instantiate here two universal quantifiers. We omit the other induction
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 223
principle that has @{prop "even n"} as premise and @{term "Q n"} as conclusion.
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 224
The proofs of the introduction rules are also very similar to the ones in
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 225
the @{text "trcl"}-example. We only show the proof of the second introduction
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 226
rule.
32
+ − 227
*}
+ − 228
127
+ − 229
lemma %linenos evenS:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 230
shows "odd m \<Longrightarrow> even (Suc m)"
115
+ − 231
apply (unfold odd_def even_def)
+ − 232
apply (rule allI impI)+
+ − 233
proof -
165
+ − 234
case (goal1 P Q)
127
+ − 235
have p1: "\<forall>P Q. P 0 \<longrightarrow> (\<forall>m. Q m \<longrightarrow> P (Suc m))
115
+ − 236
\<longrightarrow> (\<forall>m. P m \<longrightarrow> Q (Suc m)) \<longrightarrow> Q m" by fact
127
+ − 237
have r1: "P 0" by fact
+ − 238
have r2: "\<forall>m. Q m \<longrightarrow> P (Suc m)" by fact
+ − 239
have r3: "\<forall>m. P m \<longrightarrow> Q (Suc m)" by fact
115
+ − 240
show "P (Suc m)"
127
+ − 241
apply(rule r2[rule_format])
+ − 242
apply(rule p1[THEN spec[where x=P], THEN spec[where x=Q],
+ − 243
THEN mp, THEN mp, THEN mp, OF r1, OF r2, OF r3])
115
+ − 244
done
+ − 245
qed
88
+ − 246
32
+ − 247
text {*
219
+ − 248
The interesting lines are 7 to 15. The assumptions fall into two categories:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 249
@{text p1} corresponds to the premise of the introduction rule; @{text "r1"}
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 250
to @{text "r3"} come from the definition of @{text "even"}.
127
+ − 251
In Line 13, we apply the assumption @{text "r2"} (since we prove the second
+ − 252
introduction rule). In Lines 14 and 15 we apply assumption @{text "p1"} (if
+ − 253
the second introduction rule had more premises we have to do that for all
+ − 254
of them). In order for this assumption to be applicable, the quantifiers
+ − 255
need to be instantiated and then also the implications need to be resolved
+ − 256
with the other rules.
+ − 257
219
+ − 258
Next we define the accessible part of a relation @{text R} given by
+ − 259
the single rule:
+ − 260
+ − 261
\begin{center}\small
+ − 262
\mbox{\inferrule{@{term "\<And>y. R y x \<Longrightarrow> accpart R y"}}{@{term "accpart R x"}}}
+ − 263
\end{center}
+ − 264
+ − 265
The definition of @{text "accpart"} is:
32
+ − 266
*}
+ − 267
127
+ − 268
definition "accpart \<equiv> \<lambda>R x. \<forall>P. (\<forall>x. (\<forall>y. R y x \<longrightarrow> P y) \<longrightarrow> P x) \<longrightarrow> P x"
32
+ − 269
+ − 270
text {*
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 271
The proof of the induction principle is again straightforward and omitted.
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 272
Proving the introduction rule is a little more complicated, because the
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 273
quantifier and the implication in the premise. The proof is as follows.
115
+ − 274
*}
+ − 275
127
+ − 276
lemma %linenos accpartI:
218
7ff7325e3b4e
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 277
shows "(\<And>y. R y x \<Longrightarrow> accpart R y) \<Longrightarrow> accpart R x"
115
+ − 278
apply (unfold accpart_def)
+ − 279
apply (rule allI impI)+
+ − 280
proof -
+ − 281
case (goal1 P)
127
+ − 282
have p1: "\<And>y. R y x \<Longrightarrow>
115
+ − 283
(\<forall>P. (\<forall>x. (\<forall>y. R y x \<longrightarrow> P y) \<longrightarrow> P x) \<longrightarrow> P y)" by fact
127
+ − 284
have r1: "\<forall>x. (\<forall>y. R y x \<longrightarrow> P y) \<longrightarrow> P x" by fact
115
+ − 285
show "P x"
127
+ − 286
apply(rule r1[rule_format])
115
+ − 287
proof -
+ − 288
case (goal1 y)
127
+ − 289
have r1_prem: "R y x" by fact
115
+ − 290
show "P y"
127
+ − 291
apply(rule p1[OF r1_prem, THEN spec[where x=P], THEN mp, OF r1])
115
+ − 292
done
+ − 293
qed
+ − 294
qed
+ − 295
+ − 296
text {*
219
+ − 297
As you can see, there are now two subproofs. The assumptions fall again into
+ − 298
two categories (Lines 7 to 9). In Line 11, applying the assumption @{text
+ − 299
"r1"} generates a goal state with the new local assumption @{term "R y x"},
+ − 300
named @{text "r1_prem"} in the second subproof (Line 14). This local assumption is
+ − 301
used to solve the goal @{term "P y"} with the help of assumption @{text
+ − 302
"p1"}.
+ − 303
124
+ − 304
219
+ − 305
\begin{exercise}
+ − 306
Give the definition for the freshness predicate for lambda-terms. The rules
+ − 307
for this predicate are:
+ − 308
+ − 309
\begin{center}\small
+ − 310
@{prop[mode=Rule] "a\<noteq>b \<Longrightarrow> fresh a (Var b)"}\hspace{5mm}
+ − 311
@{prop[mode=Rule] "\<lbrakk>fresh a t; fresh a s\<rbrakk> \<Longrightarrow> fresh a (App t s)"}\\[2mm]
+ − 312
@{prop[mode=Axiom] "fresh a (Lam a t)"}\hspace{5mm}
+ − 313
@{prop[mode=Rule] "\<lbrakk>a\<noteq>b; fresh a t\<rbrakk> \<Longrightarrow> fresh a (Lam b t)"}
+ − 314
\end{center}
+ − 315
+ − 316
From the definition derive the induction principle and the introduction
+ − 317
rules.
+ − 318
\end{exercise}
+ − 319
+ − 320
The point of all these examples is to get a feeling what the automatic
+ − 321
proofs should do in order to solve all inductive definitions we throw at
+ − 322
them. This is usually the first step in writing a package. We next explain
129
+ − 323
the parsing and typing part of the package.
127
+ − 324
115
+ − 325
*}
129
+ − 326
(*<*)end(*>*)