1 Substitution 2 Natural Deduction

Total Page:16

File Type:pdf, Size:1020Kb

1 Substitution 2 Natural Deduction Math 4680, Topics in Logic and Computation, Winter 2012 2. t is substitutable for x in ¬ ϕ iff t is substitutable for x in ϕ. Lecture Notes 4: Soundness, Completeness, and Consequences for t is substitutable for x in ϕ ψ iff t is substitutable for x in ϕ and t is First-Order Logic substitutable for x in ψ. Peter Selinger 3. t is substitutable for x in ∀y.ϕ iff either (a) x is not free in ∀y.ϕ or 1 Substitution (b) y is not free in t and t is substitutable for x in ϕ. t is substitutable for x in ∃y.ϕ iff either We write t1[t/x] for the result of substituting the term t for the variable x in the term t1, and ϕ[t/x] for the result of substituting t for x in the formula ϕ. Here, (a) x is not free in ∃y.ϕ or only free occurrences of x are substituted. More precisely, substitution is defined (b) is not free in and is substitutable for in . recursively as follows. On terms: y t t x ϕ Convention. From now on, whenever we write ϕ[t/x], it is always implicitly x[t/x] = t assumed that t is substitutable for x in ϕ. If t is not substitutable for x in ϕ, then y[t/x] = y if x, y are different variables we implicitly rename the bound variables in ϕ so that t becomes substitutable for f(t1,...,t )[t/x] = f(t1[t/x],...,t [t/x]) n n x in ϕ. On formulas: In the proofs of soundness and completeness, we often need to relate substitutions 1. P (t1,...,tn)[t/x] = P (t1[t/x],...,tn[t/x]) to the interpretation of the involved terms in a structure. The following lemma ≈ ≈ (t1 t2)[t/x] = t1[t/x] t2[t/x] provides the necessary facts. 2. (¬ ϕ)[t/x] = ¬(ϕ[t/x]) (ϕ ψ)[t/x] = (ϕ[t/x]) (ψ[t/x]) Lemma 1 (Substitution Lemma). Suppose A is a structure and s is a valuation. 3. (∀x.ϕ)[t/x] = ∀x.ϕ Suppose t a term, x a variable, and s¯(t)= a. Let s′ = s(a|x). Then (∀y.ϕ)[t/x] = ∀y.(ϕ[t/x]) if x, y are different variables ′ (∃x.ϕ)[t/x] = ∃x.ϕ 1. s¯(t1[t/x]) = s¯(t1) for all terms t1. ∃ ∃ ( y.ϕ)[t/x] = y.(ϕ[t/x]) if x, y are different variables ′ 2. |=A ϕ[t/x][s] iff |=A ϕ [s ], for all formulas ϕ such that t is substitutable Substitution is a more subtle notion than meets the eye. In particular, one has to for x in ϕ. be careful that t does not contain any free variables which get captured when t is substituted into some formula. Consider the formula ∃y.x 6≈ y. In a structure Proof. By induction on terms and formulas. with two or more elements, this statement is true for any x. On the other hand, if we substitute y for x, we obtain ∃y.y 6≈ y, which is false! We want to rule out situations like this. 2 Natural Deduction We say that t is substitutable for x in ϕ if we can substitute t for x in ϕ without worrying about free variables of t intruding the scope of quantifiers in ϕ. More The natural deduction rules for first-order logic are those for sentential logic, plus precisely, this concept is defined by recursion on ϕ: the rules given below. Note that since we are already using lower-case roman letters for variables, we are now using numbers to identify canceled hypotheses. 1. If ϕ is atomic, then t is always substitutable for x in ϕ. Also, in the rules for quantifiers, whenever we write ϕ[t/x], it is always implicitly 1 2 assumed that t is substitutable for x in ϕ. Note the side conditions in the (∀I) 3 Soundness and Completeness and (∃E) rules. These conditions ensure that we have not made any unwarranted assumptions about the variable a. Theorem 2 (Soundness and Completeness). If Γ is a set of formulas, and ϕ is a Rules for quantifiers: formula, then Γ ⊢ ϕ iff Γ |= ϕ. Γ The left-to-right implication is called soundness, and the right-to-left implication . is called completeness. ϕ[a/x] (∀I) if a is a variable not free in Γ or ϕ ∀x.ϕ Proof. Soundness is proved by induction on the size of derivations, and by a case distinction on what the last rule in the derivation is. The substitution lemma is Γ needed in the cases of the quantifier rules. For the proof of completeness, see e.g. van Dalen’s book [?]. ∀x.ϕ (∀E) if t is a term ϕ[t/x] 4 Compactness and consequences Γ . The following theorem is a trivial consequenceof the soundness and completeness . theorem, but it has many interesting and surprising applications. Recall that a set ϕ (∃I) if t is a term of formulas is called satisfiable if there exists a structure and a valuation that ϕ[t/x] makes all formulas in the set true. Γ Γ, [ϕ[a/x]]1 Theorem 3 (Compactness). Let Γ be a set of formulas. If every finite subset of Γ . is satisfiable, then Γ is satisfiable. ∃x.ϕ ψ 1 (∃E) if a is a variable not free in Γ, ϕ, or ψ Proof. We prove the contrapositive. Suppose Γ is not satisfiable. Then Γ |= ⊥. ψ By completeness, Γ ⊢ ⊥. But natural deductions are finite, hence any deduction ′ Rules for equality: can only use finitely many hypotheses. It follows that Γ ⊢ ⊥ for some finite Γ′ ⊆ Γ. By soundness, Γ′ |= ⊥, and thus Γ′ is not satisfiable, as desired. s ≈ t r ≈ s s ≈ t t ≈ t (refl) t ≈ s (symm) r ≈ t (trans) Several applications of the compactness theorem are demonstrated in the exercises ′ s ≈ s′ s ≈ s ϕ[s/x] of Problem Set 9. Here are some more examples of such applications: ≈ ′ (cong1) ′ (cong2) t[s/x] t[s /x] ϕ[s /x] Theorem 4. Suppose Σ is a set of sentences. If Σ has arbitrarily large finite As before, we write Γ ⊢ ϕ if there is a natural deduction derivation, all of whose models, then it has an infinite model. uncanceled hypotheses are in Γ, and whose conclusion is ϕ. Proof. Suppose Σ has arbitrarily large finite models. For every n ∈ N, let λn be the sentence that states “there are at least n distinct object”. Notice that λn is first-order definable, for instance λ3 = ∃x∃y∃z(x 6≈ y ∧ x 6≈ z ∧ y 6≈ z). 3 4 Consider the set of sentences Φ=Σ ∪{λn | n ∈ N}. Since Σ has arbitrarily Proof. “⇒”: Suppose K is finitely axiomatizable. Then surely K is axioma- c large finite models, every finite subset of Φ has a model. By compactness, Φ has tizable. To show that K is axiomatizable, let K = Mod(σ1,...,σn). Let c a model. But any model of Φ is infinite, and it is also a model of Σ. Thus, Σ has σ = σ1 ∧ ... ∧ σn. Then A ∈ K iff |=A σ. Consequently A ∈ K iff 6|=A σ, iff c an infinite model. |=A ¬ σ. Thus, K = Mod(¬ σ). “⇐”: Suppose both K and Kc are axiomatizable. Let K = Mod(Σ) and Kc = Recall that a class K of structures is called axiomatizable if K = Mod(Σ), Mod(Γ). Since no structure is in K and Kc, the set Σ ∪ Γ is unsatisfiable. By for some set of sentences Σ. Also, K is called finitely axiomatizable if K = compactness, there exists a finite subset Σ′ ∪ Γ′ which is unsatisfiable. Clearly Mod(σ1,...,σn) for finitely many sentences σ1,...,σn. every model of Σ is a model of Σ′. Conversely, let A be a model of Σ′. Then A ′ A c A Theorem 5. The class of all infinite structures is axiomatizable, but not finitely does not satisfy Γ , and hence not Γ. Thus 6∈ K , thus ∈ K. We have: axiomatizable. ′ K = Mod(Σ) ⊆ Mod(Σ ) ⊆ K, N ′ Proof. Let K be the class of infinite structures. The set {λn | n ∈ } axiomatizes and hence K = Mod(Σ ). Thus K is finitely axiomatizable, as desired. K. Suppose, on the other hand, that K was finitely axiomatizable. Then there exist sentences σ1,...,σn such that K = Mod(σ1,...,σn). Let σ = σ1 ∧ ... ∧ A σn, then K = Mod(σ). Thus, a structure is infinite iff |=A σ. Equivalently, a 5 Size of models structure A is finite iff |=A ¬ σ. But then the class of finite structures would be axiomatizable, contradicting Theorem 4. The cardinality of a set is the number of elements in the set. Different infinite The following theorem is often useful in proving that a certain class of structures sets can have different cardinalities; for instance, the set of natural numbers has is not finitely axiomatizable: a smaller cardinality than the set of real numbers. We say the cardinality of a structure A is the cardinality of its carrier |A|. The cardinality of a language L is Theorem 6. If K is a finitely axiomatizable class of structures, and if K = the cardinality of L, considered as a set of sentences. ′ ′ Mod(Σ), then there exists a finite subset Σ ⊆ Σ such that K = Mod(Σ ). Remark. If P and F are the sets of predicate symbols, respectively function sym- bols, of the language L, then the cardinality of L is κ = max(card P∪F, ℵ0).
Recommended publications
  • Proof Theory Can Be Viewed As the General Study of Formal Deductive Systems
    Proof Theory Jeremy Avigad December 19, 2017 Abstract Proof theory began in the 1920’s as a part of Hilbert’s program, which aimed to secure the foundations of mathematics by modeling infinitary mathematics with formal axiomatic systems and proving those systems consistent using restricted, finitary means. The program thus viewed mathematics as a system of reasoning with precise linguistic norms, governed by rules that can be described and studied in concrete terms. Today such a viewpoint has applications in mathematics, computer science, and the philosophy of mathematics. Keywords: proof theory, Hilbert’s program, foundations of mathematics 1 Introduction At the turn of the nineteenth century, mathematics exhibited a style of argumentation that was more explicitly computational than is common today. Over the course of the century, the introduction of abstract algebraic methods helped unify developments in analysis, number theory, geometry, and the theory of equations, and work by mathematicians like Richard Dedekind, Georg Cantor, and David Hilbert towards the end of the century introduced set-theoretic language and infinitary methods that served to downplay or suppress computational content. This shift in emphasis away from calculation gave rise to concerns as to whether such methods were meaningful and appropriate in mathematics. The discovery of paradoxes stemming from overly naive use of set-theoretic language and methods led to even more pressing concerns as to whether the modern methods were even consistent. This led to heated debates in the early twentieth century and what is sometimes called the “crisis of foundations.” In lectures presented in 1922, Hilbert launched his Beweistheorie, or Proof Theory, which aimed to justify the use of modern methods and settle the problem of foundations once and for all.
    [Show full text]
  • Systematic Construction of Natural Deduction Systems for Many-Valued Logics
    23rd International Symposium on Multiple Valued Logic. Sacramento, CA, May 1993 Proceedings. (IEEE Press, Los Alamitos, 1993) pp. 208{213 Systematic Construction of Natural Deduction Systems for Many-valued Logics Matthias Baaz∗ Christian G. Ferm¨ullery Richard Zachy Technische Universit¨atWien, Austria Abstract sion.) Each position i corresponds to one of the truth values, vm is the distinguished truth value. The in- A construction principle for natural deduction sys- tended meaning is as follows: Derive that at least tems for arbitrary finitely-many-valued first order log- one formula of Γm takes the value vm under the as- ics is exhibited. These systems are systematically ob- sumption that no formula in Γi takes the value vi tained from sequent calculi, which in turn can be au- (1 i m 1). ≤ ≤ − tomatically extracted from the truth tables of the log- Our starting point for the construction of natural ics under consideration. Soundness and cut-free com- deduction systems are sequent calculi. (A sequent is pleteness of these sequent calculi translate into sound- a tuple Γ1 ::: Γm, defined to be satisfied by an ness, completeness and normal form theorems for the interpretationj iffj for some i 1; : : : ; m at least one 2 f g natural deduction systems. formula in Γi takes the truth value vi.) For each pair of an operator 2 or quantifier Q and a truth value vi 1 Introduction we construct a rule introducing a formula of the form 2(A ;:::;A ) or (Qx)A(x), respectively, at position i The study of natural deduction systems for many- 1 n of a sequent.
    [Show full text]
  • Complexities of Proof-Theoretical Reductions
    Complexities of Proof-Theoretical Reductions Michael Toppel Submitted in accordance with the requirements for the degree of Doctor of Philosophy The University of Leeds Department of Pure Mathematics September 2016 iii The candidate confirms that the work submitted is his own and that appropriate credit has been given where reference has been made to the work of others. This copy has been supplied on the understanding that it is copyright material and that no quotation from the thesis may be published without proper acknowledgement. c 2016 The University of Leeds and Michael Toppel iv v Abstract The present thesis is a contribution to a project that is carried out by Michael Rathjen 0 and Andreas Weiermann to give a general method to study the proof-complexity of Σ1- sentences. This general method uses the generalised ordinal-analysis that was given by Buchholz, Ruede¨ and Strahm in [5] and [44] as well as the generalised characterisation of provable-recursive functions of PA + TI(≺ α) that was given by Weiermann in [60]. The present thesis links these two methods by giving an explicit elementary bound for the i proof-complexity increment that occurs after the transition from the theory IDc ! + TI(≺ α), which was used by Ruede¨ and Strahm, to the theory PA + TI(≺ α), which was analysed by Weiermann. vi vii Contents Abstract . v Contents . vii Introduction 1 1 Justifying the use of Multi-Conclusion Sequents 5 1.1 Introduction . 5 1.2 A Gentzen-semantics . 8 1.3 Multi-Conclusion Sequents . 15 1.4 Comparison with other Positions and Responses to Objections .
    [Show full text]
  • An Integration of Resolution and Natural Deduction Theorem Proving
    From: AAAI-86 Proceedings. Copyright ©1986, AAAI (www.aaai.org). All rights reserved. An Integration of Resolution and Natural Deduction Theorem Proving Dale Miller and Amy Felty Computer and Information Science University of Pennsylvania Philadelphia, PA 19104 Abstract: We present a high-level approach to the integra- ble of translating between them. In order to achieve this goal, tion of such different theorem proving technologies as resolution we have designed a programming language which permits proof and natural deduction. This system represents natural deduc- structures as values and types. This approach builds on and ex- tion proofs as X-terms and resolution refutations as the types of tends the LCF approach to natural deduction theorem provers such X-terms. These type structures, called ezpansion trees, are by replacing the LCF notion of a uakfation with explicit term essentially formulas in which substitution terms are attached to representation of proofs. The terms which represent proofs are quantifiers. As such, this approach to proofs and their types ex- given types which generalize the formulas-as-type notion found tends the formulas-as-type notion found in proof theory. The in proof theory [Howard, 19691. Resolution refutations are seen LCF notion of tactics and tacticals can also be extended to in- aa specifying the type of a natural deduction proofs. This high corporate proofs as typed X-terms. Such extended tacticals can level view of proofs as typed terms can be easily combined with be used to program different interactive and automatic natural more standard aspects of LCF to yield the integration for which Explicit representation of proofs deduction theorem provers.
    [Show full text]
  • Natural Deduction and the Curry-Howard-Isomorphism
    Natural Deduction and the Curry-Howard-Isomorphism Andreas Abel August 2016 Abstract We review constructive propositional logic and natural deduction and connect it to the simply-typed lambda-calculus with the Curry- Howard Isomorphism. Constructive Logic A fundamental property of constructive logic is the disjunction property: If the disjunction A _ B is provable, then either A is provable or B is provable. This property is not compatible with the principle of the excluded middle (tertium non datur), which states that A _:A holds for any proposition A. While each fool can state the classical tautology \aliens exist or don't", this certainly does not give us a means to decide whether aliens exist or not. A constructive proof of the fool's statement would require either showcasing an alien or a stringent argument for the impossibility of their existence.1 1 Natural deduction for propositional logic The proof calculus of natural deduction goes back to Gentzen[1935]. 1 For a more mathematical example of undecidability, refer to the continuum hypothesis CH which states that no cardinal exists between the set of the natural numbers and the set of reals. It is independent of ZFC, Zermelo-Fr¨ankel set theory with the axiom of choice, meaning that in ZFC, neither CH nor :CH is provable. 1 1.1 Propositions Formulæ of propositional logic are given by the following grammar: P; Q atomic proposition A; B; C ::= P j A ) B implication j A ^ B j > conjunction, truth j A _ B j ? disjunction, absurdity Even though we write formulas in linearized (string) form, we think of them as (abstract syntax) trees.
    [Show full text]
  • On Synthetic Undecidability in Coq, with an Application to the Entscheidungsproblem
    On Synthetic Undecidability in Coq, with an Application to the Entscheidungsproblem Yannick Forster Dominik Kirst Gert Smolka Saarland University Saarland University Saarland University Saarbrücken, Germany Saarbrücken, Germany Saarbrücken, Germany [email protected] [email protected] [email protected] Abstract like decidability, enumerability, and reductions are avail- We formalise the computational undecidability of validity, able without reference to a concrete model of computation satisfiability, and provability of first-order formulas follow- such as Turing machines, general recursive functions, or ing a synthetic approach based on the computation native the λ-calculus. For instance, representing a given decision to Coq’s constructive type theory. Concretely, we consider problem by a predicate p on a type X, a function f : X ! B Tarski and Kripke semantics as well as classical and intu- with 8x: p x $ f x = tt is a decision procedure, a function itionistic natural deduction systems and provide compact д : N ! X with 8x: p x $ ¹9n: д n = xº is an enumer- many-one reductions from the Post correspondence prob- ation, and a function h : X ! Y with 8x: p x $ q ¹h xº lem (PCP). Moreover, developing a basic framework for syn- for a predicate q on a type Y is a many-one reduction from thetic computability theory in Coq, we formalise standard p to q. Working formally with concrete models instead is results concerning decidability, enumerability, and reducibil- cumbersome, given that every defined procedure needs to ity without reference to a concrete model of computation. be shown representable by a concrete entity of the model.
    [Show full text]
  • Generating Hints and Feedback for Hilbert-Style Axiomatic Proofs
    Generating hints and feedback for Hilbert-style axiomatic proofs Josje Lodder Bastiaan Heeren Johan Jeuring Technical Report UU-CS-2016-009 December 2016 Department of Information and Computing Sciences Utrecht University, Utrecht, The Netherlands www.cs.uu.nl ISSN: 0924-3275 Department of Information and Computing Sciences Utrecht University P.O. Box 80.089 3508 TB Utrecht The Netherlands Generating hints and feedback for Hilbert-style axiomatic proofs Josje Lodder Bastiaan Heeren Johan Jeuring Open University of the Open University of the Open University of the Netherlands Netherlands Netherlands and Utrecht [email protected] [email protected] University [email protected] ABSTRACT From these students, 22 had to redo their homework exer- This paper describes an algorithm to generate Hilbert-style cise on axiomatic proofs. This is significantly higher than, axiomatic proofs. Based on this algorithm we develop lo- for example, the number of students in the same group who gax, a new interactive tutoring tool that provides hints and had to redo the exercise on semantic tableaux: 5 out of 65. feedback to a student who stepwise constructs an axiomatic A student practices axiomatic proofs by solving exercises. proof. We compare the generated proofs with expert and Since it is not always possible to have a human tutor avail- student solutions, and conclude that the quality of the gen- able, an intelligent tutoring system (ITS) might be of help. erated proofs is comparable to that of expert proofs. logax There are several ITSs supporting exercises on natural de- recognizes most steps that students take when constructing duction systems [23, 22, 6].
    [Show full text]
  • Types of Proof System
    Types of proof system Peter Smith October 13, 2010 1 Axioms, rules, and what logic is all about 1.1 Two kinds of proof system There are at least two styles of proof system for propositional logic other than trees that beginners ought to know about. The real interest here, of course, is not in learning yet more about classical proposi- tional logic per se. For how much fun is that? Rather, what we are doing { as always { is illustrating some Big Ideas using propositional logic as a baby example. The two new styles are: 1. Axiomatic systems The first system of formal logic in anything like the contempo- rary sense { Frege's system in his Begriffsschrift of 1879 { is an axiomatic one. What is meant by `axiomatic' in this context? Think of Euclid's geometry for example. In such an axiomatic theory, we are given a \starter pack" of basic as- sumptions or axioms (we are often given a package of supplementary definitions as well, enabling us to introduce new ideas as abbreviations for constructs out of old ideas). And then the theorems of the theory are those claims that can deduced by allowed moves from the axioms, perhaps invoking definitions where appropriate. In Euclid's case, the axioms and definitions are of course geometrical, and he just helps himself to whatever logical inferences he needs to execute the deductions. But, if we are going to go on to axiomatize logic itself, we are going to need to be explicit not just about the basic logical axioms we take as given starting points for deductions, but also about the rules of inference that we are permitted to use.
    [Show full text]
  • The Natural Deduction Pack
    The Natural Deduction Pack Alastair Carr March 2018 Contents 1 Using this pack2 2 Summary of rules3 3 Worked examples5 3.1 Implication..............................5 3.2 Universal quantifier..........................6 3.3 Existential quantifier.........................8 4 Practice problems 11 4.1 Core.................................. 11 4.2 Conjunction.............................. 13 4.3 Implication.............................. 14 4.4 Disjunction.............................. 15 4.5 Biconditional............................. 16 4.6 Negation................................ 17 4.7 Universal quantifier.......................... 19 4.8 Existential quantifier......................... 21 4.9 Identity................................ 23 4.10 Additional challenges......................... 24 5 Solutions 26 5.1 Core.................................. 26 5.2 Conjunction.............................. 35 5.3 Implication.............................. 36 5.4 Disjunction.............................. 42 5.5 Biconditional............................. 50 5.6 Negation................................ 55 5.7 Universal quantifier.......................... 71 5.8 Existential quantifier......................... 86 5.9 Identity................................ 106 5.10 Additional challenges......................... 117 1 1 Using this pack This pack consists of Natural Deduction problems, intended to be used alongside The Logic Manual by Volker Halbach. The pack covers Natural Deduction proofs in propositional logic (L1), predicate logic (L2) and predicate logic with
    [Show full text]
  • Natural Deduction
    Natural deduction Constructive Logic (15-317) Instructor: Giselle Reis Lecture 02 1 Some history David Hilbert was a German mathematician who published, in 1899, a very influential book called Foundations of Geometry. The thing that was so revo- lutionary about this book was the way theorems were proven. It followed very closely an axiomatic approach, meaning that a set of geometry axioms were assumed and the whole theory was developed by deriving new facts from those axioms via modus ponens basically1. Hilbert believed this was the right way to do mathematics, so in 1920 he proposed that all math- ematics be formalized using a set of axioms which needed to be proved consistent (i.e. ? cannot be derived from them). All further mathematical knowledge would follow from this set. Shortly after that, it was clear that the task would not be so easy. Several attempts were proposed, but mathematicians and philosophers alike kept running into paradoxes. The foundations of mathematics was in crisis: to have something so fundamental and powerful be inconsistent seemed like a disaster. Many scientists were compelled to prove consistency of at least some part of math, and this was the case for Gentzen (another German mathematician and logician). In 1932 he set as a personal goal to show con- sistency of logical deduction in arithmetic. Given a formal system of logical deduction, the consistency proof becomes a purely mathematical problem, so that is what he did first. He thought that later on arithmetic could be added (turns out that was not so straightforward, and he ended up devel- oping yet another system, but ultimately Gentzen did prove consistency of arithmetic).
    [Show full text]
  • Some Basics of Classical Logic
    Some Basics of Classical Logic Theodora Achourioti AUC/ILLC, University of Amsterdam [email protected] PWN Vakantiecursus 2014 Eindhoven, August 22 Amsterdam, August 29 Theodora Achourioti (AUC/ILLC, UvA) Some Basics of Classical Logic PWN Vakantiecursus 2014 1 / 47 Intro Classical Logic Propositional and first order predicate logic. A way to think about a logic (and no more than that) is as consisting of: Expressive part: Syntax & Semantics Normative part: Logical Consequence (Validity) Derivability (Syntactic Validity) Entailment (Semantic Validity) Theodora Achourioti (AUC/ILLC, UvA) Some Basics of Classical Logic PWN Vakantiecursus 2014 2 / 47 Outline 1 Intro 2 Syntax 3 Derivability (Syntactic Validity) 4 Semantics 5 Entailment (Semantic Validity) 6 Meta-theory 7 Further Reading Theodora Achourioti (AUC/ILLC, UvA) Some Basics of Classical Logic PWN Vakantiecursus 2014 3 / 47 Syntax Propositional Logic The language of classical propositional logic consists of: Propositional variables: p; q; r::: Logical operators: :, ^, _, ! Parentheses: ( , ) Theodora Achourioti (AUC/ILLC, UvA) Some Basics of Classical Logic PWN Vakantiecursus 2014 4 / 47 Syntax Propositional Logic Recursive definition of a well-formed formula (wff) in classical propositional logic: Definition 1 A propositional variable is a wff. 2 If φ and are wffs, then :φ,(φ ^ ), (φ _ ), (φ ! ) are wffs. 3 Nothing else is a wff. The recursive nature of the above definition is important in that it allows inductive proofs on the entire logical language. Exercise: Prove that all wffs have an even number of brackets. Theodora Achourioti (AUC/ILLC, UvA) Some Basics of Classical Logic PWN Vakantiecursus 2014 5 / 47 Syntax Predicate Logic The language of classical predicate logic consists of: Terms: a) constants (a; b; c:::) , b) variables (x; y; z:::)1 n-place predicates P; Q; R::: Logical operators: a) propositional connectives, b) quantifiers 8, 9 Parentheses: ( , ) 1Functions are also typically included in first order theories.
    [Show full text]
  • Natural Deduction, Inference, and Consistency
    NATURAL DEDUCTION, INFERENCE, AND CONSISTENCY ROBERT L. STANLEY 1. Introduction. This paper presents results in Quine's element- hood-restricted foundational system ML,1 which parallel the im- portant conjecture and theorem which Takeuti developed in his GLC, for type-theoretic systems, and which recur in Schütte's STT. Takeuti conjectured in GLC that his natural deduction subsystem, which does not postulate Modus Ponens or any clearly equivalent inference-rule, is nevertheless ponentially closed.2 Further, he showed that if it is closed, then the whole system, including classical arith- metic, must be absolutely consistent. It is especially easy to establish the "coherence" of suitable, very strong subsystems of ML—that is, that certain (false) formulae cannot be proven under the systems' simple, natural deduction rules. Presumably it is not known whether or not these subsystems are ponentially closed.8 If, in fact, they are closed, then they are all equivalent to ML, their coherence implies its coherence, and that in turn implies the consistency of ML and of arithmetic. Proof of such consistency, though much sought, is still lacking. Further, and most important, this inference-consistency relationship suggests the pos- sibility that suitably weakened varieties of these subsystems may be provably consistent, yet usefully strong foundations for mathe- matics. 2. General argument. ML and other foundational systems for mathematics can be developed by natural deduction, in the same manner as SF. ML conveniently displays the inference-consistency property under examination, which emerges typically in such de- velopments.4 Presented to the Society, August 29, 1963; received by the editors February 4, 1964.
    [Show full text]