Скачиваний:
37
Добавлен:
10.08.2013
Размер:
7.33 Mб
Скачать

278

6/Gentzen’s Cut Elimination Theorem And Applications

A G1nnf -proof T of

Γ, Λ , Θ

can be constructed, such that

depth(T ) ≤ depth(T1) + depth(T2) and c(T ) ≤ |A|.

Proof : We proceed by induction on depth(T1) + depth(T2).

Case 1: Either A is not the principal formula of the last inference of T1, or A is not the principal formula of the last inference of T2. By symmetry, we can assume the former. There are several subcases, depending on the last inference. Let us consider the : right rule, the other subcases being similar and left as an exercise. The proof has the form

S1

 

S2

 

Γ , C, A

Γ , D, A

Γ , C D, A

By the induction hypothesis, we can find proofs T1 for Γ, Λ , Θ, C and T2 for Γ, Λ , Θ, D, such that depth(Ti ) < depth(T1) + depth(T2) and c(Ti ) ≤ |A|, for i=1,2. The result follows by the inference

Γ, Λ , Θ, C Γ, Λ , Θ, D

Γ, Λ , C D, Θ

Case 2: A is the principal formula of the last inference of both T1 and

T2.

Case 2.1: A is a literal; that is, an atomic formula, or the negation of an atomic formula. In this case, both Γ , A and A, Λ Θ are axioms. By considering all possible cases, it can be verified that Γ, Λ , Θ is an axiom. For example, if A is atomic, ∆ contains ¬A and Λ contains ¬A, Γ, Λ , Θ is an axiom.

Case 2.2: A is of the form (B C). Using the weakening lemma, we can make sure that the last inference of T1 is of the form

S0

Γ, A, B

Γ, A

or

6.4 Gentzen’s Hauptsatz for Sequents in NNF

279

S0

Γ, A, C

Γ, A

replacing T1 by (T1, A) if necessary. Consider the first case, the other being

similar. By the induction hypothesis, we can find a proof T1 for Γ, Λ , Θ, B, such that depth(T1) < depth(T1) + depth(T2) and c(T1) ≤ |A|. By the inversion lemma, we can find a proof T2 of B, Λ Θ such that depth(T2)

depth(T2) and c(T2) ≤ |A|. The following proof T

T1

 

T2

 

Γ, Λ , Θ, B

B, Λ Θ

Γ, Λ , Θ

 

 

is such that depth(T ) ≤ depth(T1) + depth(T2) and has cut-rank c(T ) ≤ |A|, since |B| < |A|.

Case 2.3: A is of the form (B C). This case is symmetric to case 2.2.

Case 2.4: A is of the form xB. As in case 2.2, we can assume that A belongs to the premise of the last inference in T1, so that T1 is of the form

S0

Γ, A, B[t/x]

Γ, A

By the induction hypothesis, we can find a proof tree T1 for Γ, Λ , Θ, B[t/x], such that depth(T1) < depth(T1) + depth(T2) and c(T1) ≤ |A|. By the inversion lemma, for any variable y not bound in T2 and distinct from

all eigenvariables in T2, there is a proof T2 for B[y/x], Λ Θ, such that depth(T2) ≤ depth(T2) and c(T2) ≤ |A|. By the substitution lemma, we can

construct a proof T2 for B[t/x], Λ Θ, also such that depth(T2 ) ≤ depth(T2) and c(T2 ) ≤ |A|. Since |B[t/x]| < |A|, the proof obtained from T1 and T2 by

applying a cut to B[t/x] has cut-rank ≤ |A|.

Case 2.5: A is of the form xB. This case is symmetric to case 2.4. This concludes all the cases.

Finally, we can prove the cut elimination theorem.

The function exp(m, n, p) is defined recursively as follows:

exp(m, 0, p) = p; exp(m, n + 1, p) = mexp(m,n,p).

280

6/Gentzen’s Cut Elimination Theorem And Applications

This function grows extremely fast in the argument n. Indeed, exp(m, 1, p) = mp, exp(m, 2, p) = mmp , and in general, exp(m, n, p) is an iterated stack of exponentials of height n, topped with a p:

exp(m, n, p) = mmm···mp n

The Tait-Schwichtenberg’s version of the cut elimination theorem for G1nnf follows.

Theorem 6.4.1 (Cut elimination theorem for G1nnf ) Let T be a G1nnf - proof with cut-rank c(T ) of a sequent Γ ∆. A cut-free proof T for Γ ∆ such that depth(T ) ≤ exp(2, c(T ), depth(T )) can be constructed.

Proof : We prove the following claim by induction on the depth of proof

trees.

Claim: Let T be a G1nnf -proof with cut-rank c(T ) for a sequent Γ ∆. If c(T ) > 0 then we can construct a proof T for Γ ∆, such that

c(T ) < c(T ) and depth(T ) 2depth(T ).

Proof of Claim: If either the last inference of T is not a cut, or it is a cut and c(T ) > |A| + 1, where A is the cut formula of the last inference, we can apply the induction hypothesis to the immediate subtrees T1 or T2 (or T1) of T . We are left with the case in which the last inference is a cut and c(T ) = |A| + 1. The proof is of the form

T1

 

 

T2

 

Γ , A

 

A, Γ

 

 

Γ

 

By the induction hypothesis, we can construct a proof T1 for Γ , A and a proof T2 for A, Γ ∆, such that c(Ti ) ≤ |A| and depth(Ti ) 2depth(Ti), for i = 1, 2. Applying the reduction lemma, we obtain a proof T such that, c(T ) ≤ |A| and depth(T ) ≤ depth(T1) + depth(T2). But

depth(T1) + depth(T2) 2depth(T1) + 2depth(T2)

2max(depth(T1),depth(T2))+1 = 2depth(T ).

Hence, the claim holds for T .

The proof of the theorem follows by induction on c(T ), and by the definition of exp(2, m, n).

It is remarkable that theorem 6.4.1 provides an upper bound on the depth of cut-free proofs obtained by converting a proof with cuts. Note that the “blow up” in the size of the proof can be very large.

6.4 Gentzen’s Hauptsatz for Sequents in NNF

281

Cut-free proofs are “direct” (or analytic), in the sense that all inferences are purely mechanical, and thus require no ingenuity. Proofs with cuts are “indirect” (or nonanalytic), in the sense that the cut formula in a cut rule may not be a subformula of any of the formulae in the conclusion of the inference. Theorem 6.4.1 suggests that if some ingenuity is exercised in constructing proofs with cuts, the size of a proof can be reduced significantly. It gives a measure of the complexity of proofs. Without being very rigorous, we can say that theorem 6.4.1 suggests that there are theorems that have no easy proofs, in the sense that if the steps are straightforward, the proof is very long, or else if the proof is short, the cuts are very ingenious. Such an example is given in Statman, 1979.

We now add equality axioms to the system G1nnf .

6.4.5 The System G1nnf=

The axioms and inference rules of the system G1nnf= are defined as follows.

Definition 6.4.6 The system G1nnf= is obtained by adding to G1nnf the following sequents as axioms. All sequents of the form

.

(i) Γ , t = t;

(ii) For every n-ary function symbol f ,

 

 

 

 

 

 

.

.

.

, f s1

.

 

 

 

 

Γ, s1 = t1, s2

= t2, ..., sn = tn

...sn = f t1...tn

 

 

 

 

 

 

 

 

 

.

 

 

 

(iii) For every n-ary predicate symbol P (including =),

 

 

 

.

.

.

, P s1...sn

, P t1...tn

 

 

 

Γ, s1 = t1, s2

= t2

, ..., sn = tn

 

 

 

and all sequents obtained from the above

sequents by applications of

¬

: lef t

.

 

.

 

.

 

and ¬ : right rules to the atomic formulae t = t, si = ti, f s1...sn

= f t1...tn,

P s1...sn and P t1...tn.

 

 

 

 

 

 

 

 

 

 

.

.

 

equality axiom. It is obvious

For example, → ¬(s = t), f (s) = f (t) is an

 

nnf

is sound.

 

 

 

that these sequents are valid and that the system G1=

 

 

 

Lemma 6.4.8 (Completeness of G1nnf= ) For the system G1nnf= , every valid sequent is provable.

Proof : The lemma can be proved using the completeness of LKe (theorem 6.3.1). First, we can show that in an LKe-proof, all weakenings can be moved above all other inferences. Then, we can show how such a proof can be simulated by a G1nnf= -proof. The details are rather straighforward and are left as an exercise.

282 6/Gentzen’s Cut Elimination Theorem And Applications

6.4.6 The Cut Elimination Theorem for G1nnf=

Gentzen’s cut elimination theorem also holds for G1nnf= if an inessential cut

as a cut in which the cut formula is a literal

B or

¬

B, where B is

is defined .

 

 

equation s = t (but not an atomic formula of the form P s1...sn, where P is a

.

 

 

 

predicate symbol di erent from =). This has interesting applications, such as

the completeness of equational logic (see the problems). The proof requires a modification of lemma 6.4.6. The cut-rank of a proof is now defined by considering essential cuts only.

Lemma 6.4.9 (Reduction lemma for G1nnf= ) Let T1 be a G1nnf= -proof of Γ , A, and T2 a G1nnf= -proof of A, Λ Θ, and assume that c(T1), c(T2)

that some

|A|. Let m be the maximal rank of all predicate symbols P such nnf

 

literal P t1...tn or ¬P t1...tn is a cut formula in either T1 or T2. A G1=

-proof

T of Γ, Λ , Θ can be constructed such that

 

c(T ) ≤ |A| and depth(T ) ≤ depth(T1) + depth(T2) + m.

 

Proof : We proceed by induction on depth(T1) + depth(T2). The only new case is the case in which A is a literal of the form P t1...tn or ¬P t1...tn, and one of the two axioms Γ , A and A, Λ Θ is an equality axiom. Assume that A = P t1...tn, the other case being similar. If Γ ∆ or Λ Θ is an axiom, then Γ, Λ , Θ is an axiom. Otherwise, we have three cases.

Case 1: Γ , A is an equality axiom, but A, Λ Θ is not. Then, either ¬A is in Λ or A is in Θ, and Γ , A is obtained from some equality

axiom of the form

 

 

 

 

.

, s2

.

.

...sn , P t1...tn

Γ , s1 = t1

= t2

, ..., sn = tn, P s1

by application of ¬ : rules.

Since either P t1...tn is in Θ or ¬P t1...tn is in

Λ, the sequent Γ, Λ , Θ is an equality axiom also obtained from some sequent of the form

.

, s2

.

.

...sn , P t1

...tn.

Γ , s1 = t1

= t2

, ..., sn = tn, P s1

Case 2: Γ , A is not an equality axiom, but A, Λ Θ is. This is similar to case 1.

Case 3: Both Γ , A and A, Λ Θ are equality axioms. In this case, Γ , A is obtained from some equality axiom of the form

.

, s2

.

.

...sn , P t1...tn

Γ , s1 = t1

= t2

, ..., sn = tn, P s1

by application of ¬ : rules, and A, Λ Θ is obtained from some equality axiom of the form

.

, t2

.

.

...tn Θ , P r1

...rn

Λ , t1 = r1

= r2

, ..., tn = rn, P t1

6.4 Gentzen’s Hauptsatz for Sequents in NNF

283

by applications of ¬ : rules.

Then, Γ, Λ , Θ is obtained by applying negation rules to the sequent

.

, s2

.

.

.

, t2

.

.

...sn

Γ , Λ , s1 = t1

= t2

, ..., sn = tn, t1

= r1

= r2

, ..., tn = rn, P s1

, Θ , P r1...rn.

A proof with only inessential cuts can be given using axioms derived by applying ¬ : rules to the provable (with no essential cuts) sequents

 

.

.

.

 

 

si = ti, ti = ri → si = ri,

 

for i = 1, ..., n, and the axiom

 

 

 

.

 

.

...sn , Θ , P r1

...rn,

Γ , Λ , s1 = r1

, ..., sn = rn, P s1

 

 

 

.

.

and n inessential cuts (the i-th cut with cut formula si = ri or ¬si = ri). The

depth of this proof is n, which is bounded by m. The rest of the proof is left as an exercise.

We obtain the following cut elimination theorem.

Theorem 6.4.2 (Cut elimination theorem for G1nnf= ) Let T be a G1nnf= - proof with cut-rank c(T ) for a sequent Γ ∆, and let m be defined as in lemma 6.4.9. A G1nnf= -proof T for Γ ∆ without essential cuts such that depth(T ) ≤ exp(m + 2, c(T ), depth(T )) can be constructed.

Proof : The following claim can be shown by induction on the depth of proof trees:

Claim: Let T be a G1nnf= -proof with cut-rank c(T ) for a sequent Γ ∆. If c(T ) > 0 then we can construct a G1nnf= -proof T for Γ ∆, such that

c(T ) < c(T ) and depth(T ) (m + 2)depth(T ).

The details are left as an exercise.

Note: The cut elimination theorem with inessential cuts (with atomic

.

cut formulae of the form s = t) also holds for LKe. The interested reader is refered to Takeuti, 1975.

As an application of theorem 6.3.1, we shall prove Craig’s interpolation theorem in the next section. The significance of a proof of Craig’s theorem using theorem 6.3.1 is that an interpolant can actually be constructed. In turn, Craig’s interpolation theorem implies two other important results: Beth’s definability theorem, and Robinson’s joint consistency theorem.

284

6/Gentzen’s Cut Elimination Theorem And Applications

PROBLEMS

6.4.1. Convert the following formulae to NNF:

(¬xP (x, y) xR(x, y))x(P (x) ¬yR(x, y))

(¬x¬y¬zP (x, y) ¬x¬y(¬zQ(x, y, z) R(x, y)))

6.4.2. Convert the following formulae to NNF:

( x yP (x, y) y xP (y, x))

(¬( xP (x) y¬Q(y)) ( zG(z) w¬Q(w)))

(¬x(P (x) y¬Q(y)) ( zP (z) w¬Q(w)))

6.4.3.Write a computer program for converting a formula to NNF.

6.4.4.Give the details of the proof of lemma 6.4.2.

6.4.5.Finish the proof of the cases that have been left out in the proof of lemma 6.4.3.

6.4.6.Prove lemma 6.4.4.

6.4.7.Prove lemma 6.4.5.

6.4.8.Finish the proof of the cases that have been left out in the proof of lemma 6.4.6.

6.4.9.Finish the proof of the cases that have been left out in the proof of lemma 6.4.7.

6.4.10.Prove that for any LKe-proof, all weakenings can be moved above all other kinds of inferences. Use this result to prove lemma 6.4.8.

6.4.11.Finish the proof of the cases that have been left out in the proof of lemma 6.4.9.

6.4.12.Give the details of the proof of theorem 6.4.2.

6.4.13.Given a set S of formulae, let Des(S) be the set of immediate descendants of formulae in S as defined in problem 5.5.18, and define Sn by induction as follows:

S0 = S;

Sn+1 = Des(Sn).

Let S = Sn.

n≥0

S is called the set of descendants of S.

PROBLEMS

285

(a) Prove that for every deduction tree without essential cuts for a sequent Γ0 0, the formulae in the sets of formulae Γ {¬B | B

} for all sequents Γ ∆ occurring in that tree, belong to S or are

.

equations of the form s = t, where S = Γ0 {¬B | B 0}.

(b) Deduce from (a) that not all G1nnf= -formulae are provable.

6.4.14. Let L be a first-order language with equality and with function symbols and constant symbols, but no predicate symbols. Such a language will be called equational .

Let e1, ..., em → e be a sequent where each ei is a closed formula of the

.

form x1... xn(s = t), called a universal equation, where {x1, ..., xn}

.

is the set of variables free in s = t, and e is an atomic formula of

.

the form s = t, called an equation. Using theorem 6.4.2, prove that if e1, ..., en → e is G1nnf= -provable, then it is provable using only axioms

(including the equality axioms), the cut rule applied to equations (of

.

the form s = t), weakenings, and the : lef t rule.

6.4.15. Let L be an equational language as defined in problem 6.4.14. A substitution function (for short, a substitution) is any function σ :

V → T ERML assigning terms to the variables in V. By theorem 2.4.1, there is a unique homomorphism σ : T ERML → T ERML extending σ and defined recursively as follows:

For every variable x V, σ(x) = s(x).

For every constant c, σ(c) = c.

For every term f t1...tn T ERML,

σ(f t1...tn) = f σ(t1)...σ(tn).

By abuse of language and notation, the function σ will also be called a substitution, and will often be denoted by σ.

The subset X of V consisting of the variables such that s(x) = x is called the support of the substitution. In what follows, we will be dealing with substitutions of finite support. If a substitution σ has finite support {y1, ..., yn} and σ(yi) = si, for i = 1, .., n, for any term t, the substitution instance σ(t) is also denoted as t[s1/y1, ..., sn/yn].

Let E =< e1, ..., en > be a sequence of equations, and E the sequence of their universal closures. (Recall that for a formula A with set of free variables F V (A) = {x1, ..., xn}, x1... xnA is the universal closure of A.)

We define the relation −→E on the set T ERML of terms as follows. For any two terms t1, t2,

t1 −→E t2

286

6/Gentzen’s Cut Elimination Theorem And Applications

.

i there is some term r, some equation s = t E, some substitution σ with support F V (s) F V (t), and some tree address u in r, such that,

t1 = r[u ← σ(s)], and t2 = r[u ← σ(t)].

When t1 −→E t2, we say that t1 rewrites to t2. In words, t1 rewrites to t2 i t2 is obtained from t1 by finding a subterm σ(s) of t1 (called

a pattern) which is a substitution instance of the left hand side s of

.

an equation s = t E, and replacing this subterm by the subterm σ(t) obtained by applying the same substitution σ to the right hand side t of the equation.

Let ←→E be the relation defined such

that

 

t1 ←→E t2

i

 

either t1 −→E t2 or

t2 −→E t1,

 

be the reflexive and transitive closure of ←→E .

and let ←→E

Our goal is to prove that for every sequence E =< e1, ..., en > of equa-

 

.

 

 

tions and for every equation s = t, if E is the sequence of universal

closures of equations in E, then

 

 

.

nnf

-provable i

 

E → s = t

is G1=

s ←→E t.

During the proof that proceeds by induction, we will have to consider formulae which are universally quantified equations of the form

.

 

y1... ym(s = t),

 

where {y1, ..., ym} is a subset of F V (s) F V (t),

including the case

.

m = 0 which corresponds to the quantifier-free equation s = t. Hence, we will prove two facts.

For every sequence T consisting of (partially) universally quantified equations from E,

(1)

If

.

nnf

-provable then

 

 

T → s = t

is G1=

s ←→E t.

(2)

If

 

 

.

nnf

-provable,

s ←→E t

then E → s = t

is G1=

 

where E is the universal closure of E.

This is done as follows:

 

t, then the sequent E

(a) Prove that if s ←→E

provable, where E is the universal closure of E.

. nnf

s = t is G1= -

6.5 Craig’s Interpolation Theorem

 

 

 

287

Hint: Use induction on the structure of the term r in the definition

 

 

 

 

 

 

of ←→E .

.

 

.

 

 

and any equation v = w, let

{

E, v = w

}

(b) Given a set E of equations .

 

 

 

denote the union of E and {v = w}.

 

 

 

 

 

Prove that

 

 

 

 

 

 

 

 

 

 

 

(i) If si ←→E ti, for 1 ≤ i ≤ n, then

 

 

 

 

 

 

f (s1, ..., sn).

 

 

 

 

f (t1, ..., tn) ←→E

 

 

 

 

(ii) If t1 ←→E t2, then for every substitution σ with support F V (t1)

F V (t2),

 

 

 

σ(t

)

 

σ(t2).

 

 

(iii) If v

 

w and s

1

 

←→.

Et, then s

 

t.

 

←→E

 

←→{E,v=w}

←→E

 

.

Hint: Show that every rewrite step involving v = w as an equation

can be simulated using the steps in v ←→E w.

(c) Prove that,

for every sequence T consisting of (partially) uni-

 

 

.

versally quantified equations from E, for any equation s = t, if the

.

nnf

 

sequent T → s = t is G1=

-provable then s ←→E t.

Hint: Proceed by induction on G1nnf= proofs without essential cuts. One of the cases is that of an inessential cut. If the bottom inference is a cut, it must be of the form

 

S1

 

 

 

 

S2

 

 

 

.

 

 

 

 

.

 

.

 

 

T1 → v = w

 

 

v = w, T2

→ s = t

 

 

 

 

 

.

 

 

 

 

 

 

 

 

T → s = t

 

 

 

where T1 and T2

are subsets of T . By the induction hypothesis,

 

 

.

t. Conclude using (b).

v ←→E w and s ←→{E,v=w}

 

 

 

 

 

.

nnf

 

 

(d) Prove that the sequent E → s = t is G1=

-provable i s ←→E t.

The above problem shows the completeness of the rewrite rule method for (universal) equational logic. This is an important current area of research. For more on this approach, see the article by Huet and Oppen, in Book, 1980, and Huet, 1980.

6.5 Craig’s Interpolation Theorem

First, we define the concept of an interpolant.