7 Completeness

We want to show that the deductive system is complete, that is, that given a set of formulas Γ and a formula φ. Γφ if Γφ.

Theorem 7.1 (Completeness) Given a set of formulas Γ and a formula φ, if Γφ, then Γφ.

We take an indirect route to the theorem. In particular, we set out to establish:

Proposition 7.1 If a set of formulas Γ is consistent, then Γ is satisfiable.

That will suffice for our purposes. For given a set of formulas Γ and a formula φ, if Γφ, then by proposition 3.6, Γ,¬φ is consistent. Given the link between consistency and satisfiability, we would infer that Γ,¬φ is satisfiable, whence Γφ.

We procced in two steps:

Γ consistentΓ satisfiableΣ (ΓΣΣ maxcon)Σ (ΓΣΣ satisfiable)

One step enables us to move from the consistency of a set Γ to the existence of a maximal consistent extension Σ of that set.

Theorem 7.2 (Lindenbaum Lemma) Each consistent set Γ is a subset of a maximal consistent set of formulas Σ.

Proof. We begin with an enumeration of the formulas of propositional logic: φ0,φ1,,φn, Given Γ be a consistent set of formulas, we build a maximal consistent superset Σ by the recursion: Σ0=ΓΣn+1={Σn,φnif that set is consistentΣnotherwise We let Σ=nNΣn. We now argue that Σ is a maximal consistent superset of Γ. We proceed in several steps.

Lemma 7.1 ΓΣ

This is because Γ=Σ0 and Σ0Σ.

Lemma 7.2 For each natural number n, Γn is consistent.

Proof. A simple induction on n:

  • Σ0 is consistent on the assumption Γ is consistent.

  • If Σn is consistent, then Σn+1 is Σn,φn if consistent, or else Σn. Either way, Σn+1 is consistent.

Lemma 7.3 For each natural number n, for every m<n, ΣmΣn.

Proof. A simple induction on n:

  • Σ0 is vacuously a superset of any predecessors in the sequence.

  • Σn+1 is Σn,φn if consistent, or else Σn. Either way, since by inductive hypothesis, for every m<n ΣmΣn and ΣnΣn+1, we conclude that for every m<n ΣmΣn+1.

Lemma 7.4 For every finite subset ΔΣ, there is some natural number n such that ΔΣn.

Proof. If Δ is a finite subset of Σ, then let φn be the member of Δ of highest index. That is for all m, if φmΔ, then mn. Notice that for each natural number m, if φmΣ, then φmΣm+1. That is, a formula φm is accepted into Σ via Σm+1 if at all. So, it follows that ΔΣn+1 if n is the highest index of a formula in Δ.

Lemma 7.5 Σ is consistent.

Proof. It follows from the preceding lemmas that every finite subset of Σ is consistent. We now argue that Σ is consistent as well.

For a reductio, suppose Σ. That means that there is a finite derivation (χ1,,χn) of from Σ. That is therefore a derivation of from a finite subset of Σ, which would require a finite subset of Σ to be inconsistent. That contradicts the observation that every finite subset of Σ is consistent.

Lemma 7.6 Given a formula φ, if Σ,φ is consistent, then φΣ.

Proof. A formula φ will be assigned an index by the enumeration, which means φ=φn. Now, if Σ,φn is consistent, then Σn,φn will be consistent as well. But that means that by construction of Σ, φnΣn+1Σ.

We conclude that Σ is a maximal consistent superset of Γ.

The interest of this observation is that every maximal consistent set Σ is satisfiable.

Theorem 7.3 (Henkin Lemma) Every maximal consistent set Σ is satisfiable.

Proof. Given a maximal consistent set Σ, consider a valuation V based on an assignment v such that: v(pn)=1iffpnΣ. We use an induction on the complexity of φ to establish:
V(φ)=1iffφΣ.
- Base Case:

V(pn)=1iffv(pn)=1iffpnΣ.definition of v
- Inductive Step for ¬:

V(¬φ)=1iffV(φ)=0iffφΣInductive Hypothesisiff¬φΣProposition 3.7, 2
- Inductive Step for :

V(φψ)=1iffV(φ)=0 or V(ψ)=1iffφΣ or ψΣInductive HypothesisiffφψΣProposition 3.7, 3
We conclude that V verifies exactly those formulas in Σ. So, it follows that Σ is satisfiable.