Combinators & Lambda Calculus

Size: px
Start display at page:

Download "Combinators & Lambda Calculus"

Transcription

1 Combinators & Lambda Calculus

2 Abstracting 1/16 three apples plus two pears = five fruits concrete 3+2 = 5 abstract objects a+b = b+a a (b c) = (a b) c abstract quantities abstract operations a, b[r(a, b) R(b, a)] a[ R(a, a)] abstract relation Sxyz = xz(yz) abstract meaning

3 Words, language, theory 2/16 Remember that for a language L over an alphabet Σ one has L Σ Σ consists of all strings, possibly nonsensical L Σ chooses in some way meaningful strings called sentences often such a language is given by a grammar With a theory T we go one step further: A theory in a language L is just a subset T L selecting a set of correct sentences often such a theory is given by an axiomatic system

4 Words, language, theory 3/16 3)( 2 + meaningless = 7 2 meaningful, incorrect = 5 2 meaningful, correct T L Σ Σ Σ L T

5 Combinators 4/16 Σ CL = {I,K,S,x,,),(,=} We introduce several simple regular grammars over Σ CL. (i) constant := I K S (ii) variable := x variable (iii) term := constant variable (term term) (iv) formula := term = term Intuition: in (FA) the term F stands for a function and A for an argument

6 Combinatory Logic (Schönfinkel 1920 [1924]) 5/16 Axioms IP = P (I) KPQ = P (K) SPQR = PR(QR) (S) Deduction rules P = P P = Q Q = P P = Q,Q = R P = R P = Q PR = QR P = Q RP = RQ Here P,Q,R denote arbitrary terms IP stands for (IP), KPQ for ((KP)Q) and SPQR for (((SP)Q)R) In general PQ 1...Q n (..((PQ 1 )Q 2 )...Q n ) (association to the left)

7 Some magic with combinators 6/16 Proposition. (i) Let D SII. Then (doubling) Dx = CL xx. (ii) Let B S(KS)K. Then (composition) Bfgx = CL f(gx). (iii) Let L D(BDD). Then (self-doubling, life!) L = CL LL. Proof. (i) Dx SIIx = Ix(Ix) = xx. (ii) Bf gx S(KS)Kf gx = KSf(Kf)gx = S(Kf)gx = Kf x(gx) = f(gx). We want to understand and preferably also to control this! (iii) L D(BDD) = BDD(BDD) = D(D(BDD)) DL = LL.

8 First insight 7/16 Lemma. For every term P and every variable x, there is a term Q such that x does not occur in Q and Qx = CL P. We denote this term Q constructed in the proof as [x]p. Proof. Induction on the complexity of P. Case 1. P is a constant or a variable. Subcase 1.1 P C with C {I,K,S}. Take [x]c KC. Then indeed Subcase 1.2 P x. Take [x]x I. Then ([x]c)x = CL KCx = CL C. ([x]x)x Ix = CL x. Subcase 1.3 P y x. Take [x]y Kx. Then indeed ([x]y)x Kyx = CL y. Case 2. P UV. Take [x](uv) S([x]U)([x]V). Then indeed ([x](uv))x S([x]U)([x]V)x = CL (([x]u)x)(([x]v)x) = CL UV.

9 Algorithms 8/16 The previous proof gave P [x]p ([x]p)x = P? C KC KCx = C x I Ix = x y x Ky Kyx = y UV S([x]U)([x]V) S([x]U)([x]V)x = (([x]u)x)(([x]v)x) = UV More efficient algorithm P x P with x / P UV [x]p I KP S([x]U)([x]V)

10 Lambda Calculus: intended meaning 9/16 The meaning of λx.3x is the function x 3x that assigns to x the value 3x (3 times x) So according to this intended meaning we have (λx.3x)(6) = 18. The parentheses around the 6 are usually not written: Principal axiom So λx.m intends to capture [x]m (λx.3x)6 = 18 (λx.m)n = β M[x: = N]

11 Language and Theory (Church [1932]) 10/16 Alphabet Σ = {x,,(,),λ,=} Language variable : = x variable Theory term : = variable (term term) (λvariable term) formula : = term = term Axioms (λxm)n = M[x: = N] M = M Rules M = N N = M M = N,N = L M = N M = N ML = NL M = N LM = LN M = N λxm = λxn

12 Bureaucracy 11/16 Substitution M M[x: = N] x N y y PQ (P[x: = N])(Q[x: = N]) λxp λxp λyp λy(p[x: = N]) where y x Association to the left Associating to the right PQ 1...Q n (..((PQ 1 )Q 2 )...Q n ). λx 1...x n.m (λx 1 (λx 2 (..(λx n (M))..)))). Outer parentheses are often omitted. For example (λx.x)y ((λxx)y)

13 Examples 12/16 I (λx.x) IX = β X K (λxy.x) KXY = β X S (λxyz.xz(yz)) SXYZ = β XZ(YZ) D (λx.xx) DX = β XX B (λxyz.x(yz) BXYZ = β X(YZ) Set of lambda terms: Λ

14 Fixed point theorem 13/16 Theorem. For all F Λ there is an M Λ such that FM = β M Proof. Defines W λx.f(xx) and M WW. Then M WW (λx.f(xx))w = F(WW) FM. Corollary. For any context C[ x,m] there exists a M such that M X = C[ X,M]. Proof. M can be taken the fixed point of λm x.c[ x,m]. Then M X = (λm x.c[ x,m])m X = C[ X,M].

15 From Russell Paradox to Fixed point Theorem 14/16 The axiom of (unlimited) comprehension (essentially in Frege [1993]) is A = {x P(x)} exists, i.e. a.[a A P(a)] But then we can derive the Russell Paradox. Define then so R = {x x / x} a.[a R a / a] R R R / R, a contradiction. Haskell Curry found the fixed point theorem analyzing the Russell paradox: Writing x A as Ax (identifying sets and predicates) one obtains a.[ra (aa)] RR (RR) the meaning of R is λx. (xx), as Rx (xx) Now RR is the fixed point of, leading to the proof of the fixed point theorem

16 Consequences 15/16 We can construct terms Y,L,O,P such that Yf = f(yf) L = LL Ox = O Q = QI; Px = xp. producing fixed points; take L YD; take O YK;

17 References 16/16 A Church [1936] An unsolvable problem of elementary number theory, Am. J. Math., 58, HB Curry [1930] Grundlagen der Kombinatorischen Logik, American J. Mathematics, 52 (3), HB Curry [1934] Functionality in combinatory logic. Proc. Nat. Ac. Sc. USA, 20, G Frege [1893, 1903/1966] Grundgesetze der Arithmetik. Hildesheim: Georg Olms Verlag. M Schönfinkel [1924] On the building blocks of mathematical logic. In: van Heijenoort, Ed., 1967, From Frege to Gödel: A Source Book in Mathematical Logic, Cambridge, MA: Harvard University Press,

Origin in Mathematical Logic

Origin in Mathematical Logic Lambda Calculus Origin in Mathematical Logic Foundation of mathematics was very much an issue in the early decades of 20th century. Cantor, Frege, Russel s Paradox, Principia Mathematica, NBG/ZF Origin

More information

Origin in Mathematical Logic

Origin in Mathematical Logic Lambda Calculus Origin in Mathematical Logic Foundation of mathematics was very much an issue in the early decades of 20th century. Cantor, Frege, Russel s Paradox, Principia Mathematica, NBG/ZF The Combinatory

More information

FORMAL SYSTEMS: COMBINATORY LOGIC

FORMAL SYSTEMS: COMBINATORY LOGIC FORMAL SYSTEMS: COMBINATORY LOGIC AND λ-calculus Andrew R. Plummer Department of Linguistics The Ohio State University 30 Sept., 2009 OUTLINE 1 INTRODUCTION 2 APPLICATIVE SYSTEMS 3 USEFUL INFORMATION COMBINATORY

More information

The Lambda-Calculus Reduction System

The Lambda-Calculus Reduction System 2 The Lambda-Calculus Reduction System 2.1 Reduction Systems In this section we present basic notions on reduction systems. For a more detailed study see [Klop, 1992, Dershowitz and Jouannaud, 1990]. Definition

More information

Lambda Calculus. Andrés Sicard-Ramírez. Semester Universidad EAFIT

Lambda Calculus. Andrés Sicard-Ramírez. Semester Universidad EAFIT Lambda Calculus Andrés Sicard-Ramírez Universidad EAFIT Semester 2010-2 Bibliography Textbook: Hindley, J. R. and Seldin, J. (2008). Lambda-Calculus and Combinators. An Introduction. Cambridge University

More information

Proofs in classical logic as programs: a generalization of lambda calculus. A. Salibra. Università Ca Foscari Venezia

Proofs in classical logic as programs: a generalization of lambda calculus. A. Salibra. Università Ca Foscari Venezia Proofs in classical logic as programs: a generalization of lambda calculus A. Salibra Università Ca Foscari Venezia Curry Howard correspondence, in general Direct relationship between systems of logic

More information

Advanced Lambda Calculus Lecture 5

Advanced Lambda Calculus Lecture 5 Advanced Lambda Calculus Lecture 5 The fathers Alonzo Church (1903-1995) as mathematics student at Princeton University (1922 or 1924) Haskell B. Curry (1900-1982) as BA in mathematics at Harvard (1920)

More information

Mathematical Logic IV

Mathematical Logic IV 1 Introduction Mathematical Logic IV The Lambda Calculus; by H.P. Barendregt(1984) Part One: Chapters 1-5 The λ-calculus (a theory denoted λ) is a type free theory about functions as rules, rather that

More information

Set Theory History. Martin Bunder. September 2015

Set Theory History. Martin Bunder. September 2015 Set Theory History Martin Bunder September 2015 What is a set? Possible Definition A set is a collection of elements having a common property Abstraction Axiom If a(x) is a property ( y)( x)(x y a(x))

More information

Intersection and Singleton Type Assignment Characterizing Finite Böhm-Trees

Intersection and Singleton Type Assignment Characterizing Finite Böhm-Trees Information and Computation 178, 1 11 (2002) doi:101006/inco20022907 Intersection and Singleton Type Assignment Characterizing Finite Böhm-Trees Toshihiko Kurata 1 Department of Mathematics, Tokyo Metropolitan

More information

Termherschrijfsystemen 2003

Termherschrijfsystemen 2003 Termherschrijfsystemen 2003 Docent: Op basis van het boek Term Rewriting Systems van Terese voorjaar 2003 1 School arithmetic (3 + 5) (1 + 2) 8 (1 + 2) 8 3 24 Elementary steps: 3 + 5 8 1 + 2 3 8 3 24 Elementary

More information

The λ-calculus and Curry s Paradox Drew McDermott , revised

The λ-calculus and Curry s Paradox Drew McDermott , revised The λ-calculus and Curry s Paradox Drew McDermott drew.mcdermott@yale.edu 2015-09-23, revised 2015-10-24 The λ-calculus was invented by Alonzo Church, building on earlier work by Gottlob Frege and Moses

More information

Part I: Propositional Calculus

Part I: Propositional Calculus Logic Part I: Propositional Calculus Statements Undefined Terms True, T, #t, 1 False, F, #f, 0 Statement, Proposition Statement/Proposition -- Informal Definition Statement = anything that can meaningfully

More information

Higher Portfolio Quadratics and Polynomials

Higher Portfolio Quadratics and Polynomials Higher Portfolio Quadratics and Polynomials Higher 5. Quadratics and Polynomials Section A - Revision Section This section will help you revise previous learning which is required in this topic R1 I have

More information

Victoria Gitman and Thomas Johnstone. New York City College of Technology, CUNY

Victoria Gitman and Thomas Johnstone. New York City College of Technology, CUNY Gödel s Proof Victoria Gitman and Thomas Johnstone New York City College of Technology, CUNY vgitman@nylogic.org http://websupport1.citytech.cuny.edu/faculty/vgitman tjohnstone@citytech.cuny.edu March

More information

A NOTE ON ARITHMETIC IN FINITE TYPES. 1. Introduction

A NOTE ON ARITHMETIC IN FINITE TYPES. 1. Introduction A NOTE ON ARITHMETIC IN FINITE TYPES BENNO VAN DEN BERG 1 Abstract. We show that one can a notion of equality at higher types inside the system called HA ω on page 46 of [8] for which all congruence laws

More information

arxiv:math/ v1 [math.lo] 16 Feb 1998

arxiv:math/ v1 [math.lo] 16 Feb 1998 SOME RESULTS ON COMBINATORS IN THE SYSTEM TRC arxiv:math/9802075v1 [math.lo] 16 Feb 1998 Thomas Jech The Pennsylvania State University Abstract. We investigate the system TRC of untyped illative combinatory

More information

Lambda-Calculus (I) 2nd Asian-Pacific Summer School on Formal Methods Tsinghua University, August 23, 2010

Lambda-Calculus (I) 2nd Asian-Pacific Summer School on Formal Methods Tsinghua University, August 23, 2010 Lambda-Calculus (I) jean-jacques.levy@inria.fr 2nd Asian-Pacific Summer School on Formal Methods Tsinghua University, August 23, 2010 Plan computation models lambda-notation bound variables conversion

More information

Type Theory and Constructive Mathematics. Type Theory and Constructive Mathematics Thierry Coquand. University of Gothenburg

Type Theory and Constructive Mathematics. Type Theory and Constructive Mathematics Thierry Coquand. University of Gothenburg Type Theory and Constructive Mathematics Type Theory and Constructive Mathematics Thierry Coquand University of Gothenburg Content An introduction to Voevodsky s Univalent Foundations of Mathematics The

More information

MAGIC Set theory. lecture 1

MAGIC Set theory. lecture 1 MAGIC Set theory lecture 1 David Asperó University of East Anglia 15 October 2014 Welcome Welcome to this set theory course. This will be a 10 hour introduction to set theory. The only prerequisite is

More information

Advanced Lambda Calculus. Henk Barendregt & Giulio Manzonetto ICIS Faculty of Science Radboud University Nijmegen, The Netherlands

Advanced Lambda Calculus. Henk Barendregt & Giulio Manzonetto ICIS Faculty of Science Radboud University Nijmegen, The Netherlands Advanced Lambda Calculus Henk Barendregt & Giulio Manzonetto ICIS Faculty of Science Radboud University Nijmegen, The Netherlands Form of the course Ordinary lecture Seminar form Exam: working out an exercise

More information

Alonzo Church ( ) Lambda Calculus. λ-calculus : syntax. Grammar for terms : Inductive denition for λ-terms

Alonzo Church ( ) Lambda Calculus. λ-calculus : syntax. Grammar for terms : Inductive denition for λ-terms Alonzo Church (1903-1995) Lambda Calculus 2 λ-calculus : syntax Grammar for terms : t, u ::= x (variable) t u (application) λx.t (abstraction) Notation : Application is left-associative so that t 1 t 2...

More information

Přednáška 12. Důkazové kalkuly Kalkul Hilbertova typu. 11/29/2006 Hilbertův kalkul 1

Přednáška 12. Důkazové kalkuly Kalkul Hilbertova typu. 11/29/2006 Hilbertův kalkul 1 Přednáška 12 Důkazové kalkuly Kalkul Hilbertova typu 11/29/2006 Hilbertův kalkul 1 Formal systems, Proof calculi A proof calculus (of a theory) is given by: A. a language B. a set of axioms C. a set of

More information

Philosophy 240 Symbolic Logic Russell Marcus Hamilton College Fall 2014

Philosophy 240 Symbolic Logic Russell Marcus Hamilton College Fall 2014 Philosophy 240 Symbolic Logic Russell Marcus Hamilton College Fall 2014 Class #23 - Translation into Predicate Logic II ( 3.2) Only as a Quantifier P Only Ps are Qs is logically equivalent to all Qs are

More information

Mathematical Logic. Reasoning in First Order Logic. Chiara Ghidini. FBK-IRST, Trento, Italy

Mathematical Logic. Reasoning in First Order Logic. Chiara Ghidini. FBK-IRST, Trento, Italy Reasoning in First Order Logic FBK-IRST, Trento, Italy April 12, 2013 Reasoning tasks in FOL Model checking Question: Is φ true in the interpretation I with the assignment a? Answer: Yes if I = φ[a]. No

More information

Example. Lemma. Proof Sketch. 1 let A be a formula that expresses that node t is reachable from s

Example. Lemma. Proof Sketch. 1 let A be a formula that expresses that node t is reachable from s Summary Summary Last Lecture Computational Logic Π 1 Γ, x : σ M : τ Γ λxm : σ τ Γ (λxm)n : τ Π 2 Γ N : τ = Π 1 [x\π 2 ] Γ M[x := N] Georg Moser Institute of Computer Science @ UIBK Winter 2012 the proof

More information

Lazy Strong Normalization

Lazy Strong Normalization Lazy Strong Normalization Luca Paolini 1,2 Dipartimento di Informatica Università di Torino (ITALIA) Elaine Pimentel 1,2 Departamento de Matemática Universidade Federal de Minas Gerais (BRASIL) Dipartimento

More information

Henk Barendregt and Freek Wiedijk assisted by Andrew Polonsky. Radboud University Nijmegen. March 5, 2012

Henk Barendregt and Freek Wiedijk assisted by Andrew Polonsky. Radboud University Nijmegen. March 5, 2012 1 λ Henk Barendregt and Freek Wiedijk assisted by Andrew Polonsky Radboud University Nijmegen March 5, 2012 2 reading Femke van Raamsdonk Logical Verification Course Notes Herman Geuvers Introduction to

More information

l-calculus and Decidability

l-calculus and Decidability U.U.D.M. Project Report 2017:34 l-calculus and Decidability Erik Larsson Examensarbete i matematik, 15 hp Handledare: Vera Koponen Examinator: Jörgen Östensson Augusti 2017 Department of Mathematics Uppsala

More information

On the Standardization Theorem for λβη-calculus

On the Standardization Theorem for λβη-calculus On the Standardization Theorem for λβη-calculus Ryo Kashima Department of Mathematical and Computing Sciences Tokyo Institute of Technology Ookayama, Meguro, Tokyo 152-8552, Japan. e-mail: kashima@is.titech.ac.jp

More information

Lambda Calculus with Types. Henk Barendregt ICIS Radboud University Nijmegen The Netherlands

Lambda Calculus with Types. Henk Barendregt ICIS Radboud University Nijmegen The Netherlands Lambda Calculus with Types Henk Barendregt ICIS Radboud University Nijmegen The Netherlands New book Cambridge University Press / ASL Perspectives in Logic, 2011 Lambda Calculus with Types (698 pp) Authors:

More information

Selected Math 553 Homework Solutions

Selected Math 553 Homework Solutions Selected Math 553 Homework Solutions HW6, 1. Let α and β be rational numbers, with α 1/2, and let m > 0 be an integer such that α 2 mβ 2 = 1 δ where 0 δ < 1. Set ǫ:= 1 if α 0 and 1 if α < 0. Show that

More information

Simply Typed λ-calculus

Simply Typed λ-calculus Simply Typed λ-calculus Lecture 2 Jeremy Dawson The Australian National University Semester 2, 2017 Jeremy Dawson (ANU) COMP4630,Lecture 2 Semester 2, 2017 1 / 19 Outline Properties of Curry type system:

More information

Predicate Logic: Sematics Part 1

Predicate Logic: Sematics Part 1 Predicate Logic: Sematics Part 1 CS402, Spring 2018 Shin Yoo Predicate Calculus Propositional logic is also called sentential logic, i.e. a logical system that deals with whole sentences connected with

More information

Algebraic Expressions

Algebraic Expressions Algebraic Expressions 1. Expressions are formed from variables and constants. 2. Terms are added to form expressions. Terms themselves are formed as product of factors. 3. Expressions that contain exactly

More information

Frege s Proofs of the Axioms of Arithmetic

Frege s Proofs of the Axioms of Arithmetic Frege s Proofs of the Axioms of Arithmetic Richard G. Heck, Jr. 1 The Dedekind-Peano Axioms for Arithmetic 1. N0 2. x(nx y.p xy) 3(a). x y z(nx P xy P xy y = z) 3(b). x y z(nx Ny P xz P yz x = y) 4. z(nz

More information

The Lambda Calculus is Algebraic

The Lambda Calculus is Algebraic Under consideration for publication in J. Functional Programming 1 The Lambda Calculus is Algebraic PETER SELINGER Department of Mathematics and Statistics University of Ottawa, Ottawa, Ontario K1N 6N5,

More information

Introduction to λ-calculus

Introduction to λ-calculus p.1/65 Introduction to λ-calculus Ken-etsu FUJITA fujita@cs.gunma-u.ac.jp http://www.comp.cs.gunma-u.ac.jp/ fujita/ Department of Computer Science Gunma University :Church 32, 36, 40; Curry 34 1. Universal

More information

Löwnheim Skolem Theorem

Löwnheim Skolem Theorem Löwnheim Skolem Theorem David Pierce September 17, 2014 Mimar Sinan Fine Arts University http://mat.msgsu.edu.tr/~dpierce/ These notes are part of a general investigation of the Compactness Theorem. They

More information

Chapter 6. Properties of Regular Languages

Chapter 6. Properties of Regular Languages Chapter 6 Properties of Regular Languages Regular Sets and Languages Claim(1). The family of languages accepted by FSAs consists of precisely the regular sets over a given alphabet. Every regular set is

More information

Peano Arithmetic. CSC 438F/2404F Notes (S. Cook) Fall, Goals Now

Peano Arithmetic. CSC 438F/2404F Notes (S. Cook) Fall, Goals Now CSC 438F/2404F Notes (S. Cook) Fall, 2008 Peano Arithmetic Goals Now 1) We will introduce a standard set of axioms for the language L A. The theory generated by these axioms is denoted PA and called Peano

More information

Simply Typed λ-calculus

Simply Typed λ-calculus Simply Typed λ-calculus Lecture 1 Jeremy Dawson The Australian National University Semester 2, 2017 Jeremy Dawson (ANU) COMP4630,Lecture 1 Semester 2, 2017 1 / 23 A Brief History of Type Theory First developed

More information

Church s undecidability result

Church s undecidability result Church s undecidability result Alan Turing Birth Centennial Talk at IIT Bombay, Mumbai Joachim Breitner April 21, 2011 Welcome, and thank you for the invitation to speak about Church s lambda calculus

More information

First-Order Logic. 1 Syntax. Domain of Discourse. FO Vocabulary. Terms

First-Order Logic. 1 Syntax. Domain of Discourse. FO Vocabulary. Terms First-Order Logic 1 Syntax Domain of Discourse The domain of discourse for first order logic is FO structures or models. A FO structure contains Relations Functions Constants (functions of arity 0) FO

More information

MAGIC Set theory. lecture 2

MAGIC Set theory. lecture 2 MAGIC Set theory lecture 2 David Asperó University of East Anglia 22 October 2014 Recall from last time: Syntactical vs. semantical logical consequence Given a set T of formulas and a formula ', we write

More information

Large Numbers, Busy Beavers, Noncomputability and Incompleteness

Large Numbers, Busy Beavers, Noncomputability and Incompleteness Large Numbers, Busy Beavers, Noncomputability and Incompleteness Food For Thought November 1, 2007 Sam Buss Department of Mathematics U.C. San Diego PART I Large Numbers, Busy Beavers, and Undecidability

More information

Chapter 1. Logic and Proof

Chapter 1. Logic and Proof Chapter 1. Logic and Proof 1.1 Remark: A little over 100 years ago, it was found that some mathematical proofs contained paradoxes, and these paradoxes could be used to prove statements that were known

More information

Logic Michælmas 2003

Logic Michælmas 2003 Logic Michælmas 2003 ii Contents 1 Introduction 1 2 Propositional logic 3 3 Syntactic implication 5 3.0.1 Two consequences of completeness.............. 7 4 Posets and Zorn s lemma 9 5 Predicate logic

More information

COMP 182 Algorithmic Thinking. Proofs. Luay Nakhleh Computer Science Rice University

COMP 182 Algorithmic Thinking. Proofs. Luay Nakhleh Computer Science Rice University COMP 182 Algorithmic Thinking Proofs Luay Nakhleh Computer Science Rice University 1 Reading Material Chapter 1, Section 3, 6, 7, 8 Propositional Equivalences The compound propositions p and q are called

More information

All psychiatrists are doctors All doctors are college graduates All psychiatrists are college graduates

All psychiatrists are doctors All doctors are college graduates All psychiatrists are college graduates Predicate Logic In what we ve discussed thus far, we haven t addressed other kinds of valid inferences: those involving quantification and predication. For example: All philosophers are wise Socrates is

More information

Computability via the Lambda Calculus with Patterns

Computability via the Lambda Calculus with Patterns Computability via the Lambda Calculus with Patterns Bodin Skulkiat (Corresponding author) Department of Mathematics, Faculty of Science Chulalongkorn University, Bangkok, Thailand Tel: 66-89-666-5804 E-mail:

More information

Algebra I. Book 2. Powered by...

Algebra I. Book 2. Powered by... Algebra I Book 2 Powered by... ALGEBRA I Units 4-7 by The Algebra I Development Team ALGEBRA I UNIT 4 POWERS AND POLYNOMIALS......... 1 4.0 Review................ 2 4.1 Properties of Exponents..........

More information

How to Think of Intersection Types as Cartesian Products

How to Think of Intersection Types as Cartesian Products Available online at www.sciencedirect.com Electronic Notes in Theoretical Computer Science 325 (2016) 305 312 www.elsevier.com/locate/entcs How to Think of Intersection Types as Cartesian Products Rick

More information

Theory of Languages and Automata

Theory of Languages and Automata Theory of Languages and Automata Chapter 0 - Introduction Sharif University of Technology References Main Reference M. Sipser, Introduction to the Theory of Computation, 3 nd Ed., Cengage Learning, 2013.

More information

Factorization in Integral Domains II

Factorization in Integral Domains II Factorization in Integral Domains II 1 Statement of the main theorem Throughout these notes, unless otherwise specified, R is a UFD with field of quotients F. The main examples will be R = Z, F = Q, and

More information

Dr. Bob s Axiom of Choice Centennial Lecture Fall A Century Ago

Dr. Bob s Axiom of Choice Centennial Lecture Fall A Century Ago Dr. Bob s Axiom of Choice Centennial Lecture Fall 2008 Ernst Zermelo, 1871 1953 A Century Ago Note. This year (2008) marks the 100 year anniversary of Ernst Zermelo s first statement of the currently accepted

More information

EXAMPLES OF PROOFS BY INDUCTION

EXAMPLES OF PROOFS BY INDUCTION EXAMPLES OF PROOFS BY INDUCTION KEITH CONRAD 1. Introduction In this handout we illustrate proofs by induction from several areas of mathematics: linear algebra, polynomial algebra, and calculus. Becoming

More information

1. Propositional Calculus

1. Propositional Calculus 1. Propositional Calculus Some notes for Math 601, Fall 2010 based on Elliott Mendelson, Introduction to Mathematical Logic, Fifth edition, 2010, Chapman & Hall. 2. Syntax ( grammar ). 1.1, p. 1. Given:

More information

Axiomatic set theory. Chapter Why axiomatic set theory?

Axiomatic set theory. Chapter Why axiomatic set theory? Chapter 1 Axiomatic set theory 1.1 Why axiomatic set theory? Essentially all mathematical theories deal with sets in one way or another. In most cases, however, the use of set theory is limited to its

More information

Logic and Probability Lecture 3: Beyond Boolean Logic

Logic and Probability Lecture 3: Beyond Boolean Logic Logic and Probability Lecture 3: Beyond Boolean Logic Wesley Holliday & Thomas Icard UC Berkeley & Stanford August 13, 2014 ESSLLI, Tübingen Wesley Holliday & Thomas Icard: Logic and Probability, Lecture

More information

Syntax. Notation Throughout, and when not otherwise said, we assume a vocabulary V = C F P.

Syntax. Notation Throughout, and when not otherwise said, we assume a vocabulary V = C F P. First-Order Logic Syntax The alphabet of a first-order language is organised into the following categories. Logical connectives:,,,,, and. Auxiliary symbols:.,,, ( and ). Variables: we assume a countable

More information

Introduction to dependent type theory. CIRM, May 30

Introduction to dependent type theory. CIRM, May 30 CIRM, May 30 Goals of this presentation Some history and motivations Notations used in type theory Main goal: the statement of main properties of equality type and the univalence axiom First talk P ropositions

More information

This section will take the very naive point of view that a set is a collection of objects, the collection being regarded as a single object.

This section will take the very naive point of view that a set is a collection of objects, the collection being regarded as a single object. 1.10. BASICS CONCEPTS OF SET THEORY 193 1.10 Basics Concepts of Set Theory Having learned some fundamental notions of logic, it is now a good place before proceeding to more interesting things, such as

More information

Handbook of Logic and Proof Techniques for Computer Science

Handbook of Logic and Proof Techniques for Computer Science Steven G. Krantz Handbook of Logic and Proof Techniques for Computer Science With 16 Figures BIRKHAUSER SPRINGER BOSTON * NEW YORK Preface xvii 1 Notation and First-Order Logic 1 1.1 The Use of Connectives

More information

Predicate Calculus - Semantics 1/4

Predicate Calculus - Semantics 1/4 Predicate Calculus - Semantics 1/4 Moonzoo Kim CS Dept. KAIST moonzoo@cs.kaist.ac.kr 1 Introduction to predicate calculus (1/2) Propositional logic (sentence logic) dealt quite satisfactorily with sentences

More information

Denote John by j and Smith by s, is a bachelor by predicate letter B. The statements (1) and (2) may be written as B(j) and B(s).

Denote John by j and Smith by s, is a bachelor by predicate letter B. The statements (1) and (2) may be written as B(j) and B(s). PREDICATE CALCULUS Predicates Statement function Variables Free and bound variables Quantifiers Universe of discourse Logical equivalences and implications for quantified statements Theory of inference

More information

CHAPTER 2. FIRST ORDER LOGIC

CHAPTER 2. FIRST ORDER LOGIC CHAPTER 2. FIRST ORDER LOGIC 1. Introduction First order logic is a much richer system than sentential logic. Its interpretations include the usual structures of mathematics, and its sentences enable us

More information

Minimal logic for computable functionals

Minimal logic for computable functionals Minimal logic for computable functionals Helmut Schwichtenberg Mathematisches Institut der Universität München Contents 1. Partial continuous functionals 2. Total and structure-total functionals 3. Terms;

More information

Roots and Coefficients Polynomials Preliminary Maths Extension 1

Roots and Coefficients Polynomials Preliminary Maths Extension 1 Preliminary Maths Extension Question If, and are the roots of x 5x x 0, find the following. (d) (e) Question If p, q and r are the roots of x x x 4 0, evaluate the following. pq r pq qr rp p q q r r p

More information

Class 29 - November 3 Semantics for Predicate Logic

Class 29 - November 3 Semantics for Predicate Logic Philosophy 240: Symbolic Logic Fall 2010 Mondays, Wednesdays, Fridays: 9am - 9:50am Hamilton College Russell Marcus rmarcus1@hamilton.edu Class 29 - November 3 Semantics for Predicate Logic I. Proof Theory

More information

Paradox Machines. Christian Skalka The University of Vermont

Paradox Machines. Christian Skalka The University of Vermont Paradox Machines Christian Skalka The University of Vermont Source of Mathematics Where do the laws of mathematics come from? The set of known mathematical laws has evolved over time (has a history), due

More information

Lecture Notes on Combinatory Modal Logic

Lecture Notes on Combinatory Modal Logic Lecture Notes on Combinatory Modal Logic 15-816: Modal Logic Frank Pfenning Lecture 9 February 16, 2010 1 Introduction The connection between proofs and program so far has been through a proof term assignment

More information

LECTURE NOTES DISCRETE MATHEMATICS. Eusebius Doedel

LECTURE NOTES DISCRETE MATHEMATICS. Eusebius Doedel LECTURE NOTES on DISCRETE MATHEMATICS Eusebius Doedel 1 LOGIC Introduction. First we introduce some basic concepts needed in our discussion of logic. These will be covered in more detail later. A set is

More information

COMMON FIXED POINT THEOREM OF THREE MAPPINGS IN COMPLETE METRIC SPACE

COMMON FIXED POINT THEOREM OF THREE MAPPINGS IN COMPLETE METRIC SPACE COMMON FIXED POINT THEOREM OF THREE MAPPINGS IN COMPLETE METRIC SPACE Latpate V.V. and Dolhare U.P. ACS College Gangakhed DSM College Jintur Abstract:-In this paper we prove common fixed point theorem

More information

Decidability: Church-Turing Thesis

Decidability: Church-Turing Thesis Decidability: Church-Turing Thesis While there are a countably infinite number of languages that are described by TMs over some alphabet Σ, there are an uncountably infinite number that are not Are there

More information

1 Introduction to Predicate Resolution

1 Introduction to Predicate Resolution 1 Introduction to Predicate Resolution The resolution proof system for Predicate Logic operates, as in propositional case on sets of clauses and uses a resolution rule as the only rule of inference. The

More information

Charles Wells 1. February 25, 1999

Charles Wells 1. February 25, 1999 NOTES ON THE λ-calculus Charles Wells 1 February 25, 1999 Department of Mathematics Case Western Reserve University 10900 Euclid Ave. Cleveland, OH 44106-7058 USA charles@freude.com http://www.cwru.edu/artsci/math/wells/home.html

More information

Propositional Calculus

Propositional Calculus CHAPTER - 1 Propositional Calculus Introduction Logic means reasoning. One of the important aims of logic is to provide rules through which one can determine the validity of any particular argument. Logic

More information

Categories, Proofs and Programs

Categories, Proofs and Programs Categories, Proofs and Programs Samson Abramsky and Nikos Tzevelekos Lecture 4: Curry-Howard Correspondence and Cartesian Closed Categories In A Nutshell Logic Computation 555555555555555555 5 Categories

More information

Lecture Notes 1 Basic Concepts of Mathematics MATH 352

Lecture Notes 1 Basic Concepts of Mathematics MATH 352 Lecture Notes 1 Basic Concepts of Mathematics MATH 352 Ivan Avramidi New Mexico Institute of Mining and Technology Socorro, NM 87801 June 3, 2004 Author: Ivan Avramidi; File: absmath.tex; Date: June 11,

More information

Gödel s Incompleteness Theorem. Overview. Computability and Logic

Gödel s Incompleteness Theorem. Overview. Computability and Logic Gödel s Incompleteness Theorem Overview Computability and Logic Recap Remember what we set out to do in this course: Trying to find a systematic method (algorithm, procedure) which we can use to decide,

More information

Section 8.3 Higher-Order Logic A logic is higher-order if it allows predicate names or function names to be quantified or to be arguments of a

Section 8.3 Higher-Order Logic A logic is higher-order if it allows predicate names or function names to be quantified or to be arguments of a Section 8.3 Higher-Order Logic A logic is higher-order if it allows predicate names or function names to be quantified or to be arguments of a predicate. Example. The sentence, There is a function with

More information

258 Handbook of Discrete and Combinatorial Mathematics

258 Handbook of Discrete and Combinatorial Mathematics 258 Handbook of Discrete and Combinatorial Mathematics 16.3 COMPUTABILITY Most of the material presented here is presented in far more detail in the texts of Rogers [R], Odifreddi [O], and Soare [S]. In

More information

CA320 - Computability & Complexity

CA320 - Computability & Complexity CA320 - Computability & Complexity David Sinclair Overview In this module we are going to answer 2 important questions: Can all problems be solved by a computer? What problems be efficiently solved by

More information

Computational Logic. Recall of First-Order Logic. Damiano Zanardini

Computational Logic. Recall of First-Order Logic. Damiano Zanardini Computational Logic Recall of First-Order Logic Damiano Zanardini UPM European Master in Computational Logic (EMCL) School of Computer Science Technical University of Madrid damiano@fi.upm.es Academic

More information

Eighth Homework Solutions

Eighth Homework Solutions Math 4124 Wednesday, April 20 Eighth Homework Solutions 1. Exercise 5.2.1(e). Determine the number of nonisomorphic abelian groups of order 2704. First we write 2704 as a product of prime powers, namely

More information

Notes on generating functions in automata theory

Notes on generating functions in automata theory Notes on generating functions in automata theory Benjamin Steinberg December 5, 2009 Contents Introduction: Calculus can count 2 Formal power series 5 3 Rational power series 9 3. Rational power series

More information

Additional Practice Lessons 2.02 and 2.03

Additional Practice Lessons 2.02 and 2.03 Additional Practice Lessons 2.02 and 2.03 1. There are two numbers n that satisfy the following equations. Find both numbers. a. n(n 1) 306 b. n(n 1) 462 c. (n 1)(n) 182 2. The following function is defined

More information

1. Propositional Calculus

1. Propositional Calculus 1. Propositional Calculus Some notes for Math 601, Fall 2010 based on Elliott Mendelson, Introduction to Mathematical Logic, Fifth edition, 2010, Chapman & Hall. 2. Syntax ( grammar ). 1.1, p. 1. Given:

More information

Reflection: a powerfull and ubiquitous logical mechanism

Reflection: a powerfull and ubiquitous logical mechanism Reflection: a powerfull and ubiquitous logical mechanism Henk Barendregt Faculty of Science Radboud University Nijmegen, The Netherlands Huygens Lecture Fall 2009 Contents 1 Overview 3 2 Languages 12 3

More information

Solution/Correction standard, second Test Mathematics A + B1; November 7, 2014.

Solution/Correction standard, second Test Mathematics A + B1; November 7, 2014. Solution/Correction standard, second Test Mathematics A + B1; November 7, 014. Kenmerk : Leibniz/toetsen/Re-Exam-Math-A-B1-141-Solutions Course : Mathematics A + B1 (Leibniz) Vakcode : 1911010 Date : November

More information

Lambda Calculus. Yuxi Fu. 31 May, 2013

Lambda Calculus. Yuxi Fu. 31 May, 2013 Lambda Calculus Yuxi Fu 31 May, 2013 Origin in Mathematical Logic Foundation of mathematics was very much an issue in the early decades of 20th century. Cantor, Frege, Russel s Paradox, Principia Mathematica,

More information

Notation for Logical Operators:

Notation for Logical Operators: Notation for Logical Operators: always true always false... and...... or... if... then...... if-and-only-if... x:x p(x) x:x p(x) for all x of type X, p(x) there exists an x of type X, s.t. p(x) = is equal

More information

Introduction to Metalogic

Introduction to Metalogic Philosophy 135 Spring 2008 Tony Martin Introduction to Metalogic 1 The semantics of sentential logic. The language L of sentential logic. Symbols of L: Remarks: (i) sentence letters p 0, p 1, p 2,... (ii)

More information

Midterm 1 Solutions Thursday, February 26

Midterm 1 Solutions Thursday, February 26 Math 59 Dr. DeTurck Midterm 1 Solutions Thursday, February 26 1. First note that since f() = f( + ) = f()f(), we have either f() = (in which case f(x) = f(x + ) = f(x)f() = for all x, so c = ) or else

More information

Principles of Programming Languages

Principles of Programming Languages Principles of Programming Languages Lecture 03 Theoretical Foundations 1 Domains Semantic model of a data type: semantic domain! Examples: Integer, Natural, Truth-Value Domains D are more than a set of

More information

Foundations of Mathematics MATH 220 FALL 2017 Lecture Notes

Foundations of Mathematics MATH 220 FALL 2017 Lecture Notes Foundations of Mathematics MATH 220 FALL 2017 Lecture Notes These notes form a brief summary of what has been covered during the lectures. All the definitions must be memorized and understood. Statements

More information

Great Theoretical Ideas in Computer Science. Lecture 4: Deterministic Finite Automaton (DFA), Part 2

Great Theoretical Ideas in Computer Science. Lecture 4: Deterministic Finite Automaton (DFA), Part 2 5-25 Great Theoretical Ideas in Computer Science Lecture 4: Deterministic Finite Automaton (DFA), Part 2 January 26th, 27 Formal definition: DFA A deterministic finite automaton (DFA) M =(Q,,,q,F) M is

More information

From Constructibility and Absoluteness to Computability and Domain Independence

From Constructibility and Absoluteness to Computability and Domain Independence From Constructibility and Absoluteness to Computability and Domain Independence Arnon Avron School of Computer Science Tel Aviv University, Tel Aviv 69978, Israel aa@math.tau.ac.il Abstract. Gödel s main

More information

Introduction to Metalogic

Introduction to Metalogic Introduction to Metalogic Hans Halvorson September 21, 2016 Logical grammar Definition. A propositional signature Σ is a collection of items, which we call propositional constants. Sometimes these propositional

More information