Advanced Lambda Calculus Lecture 5

Size: px
Start display at page:

Download "Advanced Lambda Calculus Lecture 5"

Transcription

1 Advanced Lambda Calculus Lecture 5

2 The fathers Alonzo Church ( ) as mathematics student at Princeton University (1922 or 1924) Haskell B. Curry ( ) as BA in mathematics at Harvard (1920)

3 Untyped lambda terms λ Λ, Simple types Free type algebras λ A A, Recursive types Type algebras λ A = A,, = Subtyping Type structures λ S S,, Intersection types Intersection type structures λ S S,,,,

4 Curry s contributions Curry: Russell paradox as fixed point of the operator Not Idea: For a A write Aa Then as {x P[x]} we can take λx.p[x] Indeed, we get the intended interpretation a {x P[x]} becomes (λx.p[x])a = P[a] Taking R = {x x / x} = λx. (xx) we get hence RR (RR) r.[rr (rr)] Note that RR (λx. (xx))(λx. (xx)) = Y( ) Typing of Whitehead-Russell was transformed into functionality Γ FABM Γ B(MN) Γ AN Γ,Ax BM Γ FAB(λx.M)

5 Curry s contributions Curry: Russell paradox as fixed point of the operator Not Idea: For a A write Aa Then as {x P[x]} we can take λx.p[x] Indeed, we get the intended interpretation a {x P[x]} becomes (λx.p[x])a = P[a] Taking R = {x x / x} = λx. (xx) we get hence RR (RR) r.[rr (rr)] Note that RR (λx. (xx))(λx. (xx)) = Y( ) Typing of Whitehead-Russell was transformed into functionality Γ M : A B Γ MN : B Γ N : A Γ,x : A M : B Γ λx.m : (A B)

6 An increasing chain of systems λ A λ A = λ S λ S Γ,x : A x : A λ A Γ M : (A B) Γ (MN) : B Γ N : A Γ,x : A M : B Γ (λx.m) : (A B) λ A = λ S Γ M : A A = B Γ M : B Γ M : A A B Γ M : B Γ M : A B Γ M : A B Γ M : A Γ M : B λ S Γ M : A Γ M : B Γ M : A B Γ M :

7 An increasing chain of systems λ A λ A = λ S λ S λ S 8 λ S 8 >< >< >: λ A = 8 >< >: λ A 8 >< >: Γ, x : A x : A Γ M : (A B) Γ N : A Γ, x : A M : B Γ (MN) : B Γ (λx.m) : (A B) Γ M : A A = B Γ M : B Γ M : A A B Γ M : B Γ M : A B Γ M : A B Γ M : A Γ M : B >: Γ M : A Γ M : Γ M : B Γ M : A B

8 Examples λ A λxy.xyy : (A A B) A B λ A = λx.xx : A if A = A B in A (λx.xx)(λx.xx) : B λ S λx.xx : A B only; if A A B in S λx.xx : (A B) B if A B A λ S λx.xx : A (A B) B KIΩ : A A where Ω (λx.xx)(λx.xx) as Ω :

9 Simply typed λ-calculus: λ o Simple types from ground type 0 T = 0 T T Λ(A): λ-terms of type A. Write Λ = A T Λ(A) x A Λ(A) M Λ(A B),N Λ(A) (MN) Λ(B) M Λ(B) (λx A.M) Λ(A B) Default equality = βη preserves types (λx A.M)N = M[x A := N] β-conversion λx A.Mx A = M η-conversion

10 Standard terms I A λx A.x Λ(A A) K A,B λx A y B.x Λ(A B A) S A,B,C λx A B C y A B z A.xz(yz) Λ((A B C) (A B) A C) Curry: Hey, these are tautologies Curry-Howard correspondence From these ( many) terms all others can be defined applicatively Prop. (i) For M Λ (A) one has M : A (ii) For M Λ in β-nf such that M : A there is a unique M A Λ(A) such that M A M (iii) For open M not in β-nf (ii) fails: KIy : A A (iv) Even for closed M not in β-nf (ii) fails: (λx.xi)(λy.i) : A A The counter-examples in (iii), (iv) are due to the presence or creation of a K-redex For normal M one can identify M : A and M A Λ(A)

11 Type structures Def. Let M = {M(A)} A T be a family of non-empty sets (i) M is called a type structure for λ o if M(A B) M(B) M(A) Here Y X denotes the collection of set-theoretic functions {f f : X Y } (ii) Let M be provided with application operators (M, ) = ({M(A)} A T, { A,B } A,B T ) A,B : M(A B) M(A) M(B). A typed applicative structure is such an (M, ) satisfying extensionality: f,g M(A B) [[ a M(A) f A,B a = g A,B a] f = g]. Prop. The notions type structure and typed applicative structure are equivalent

12 Full type structures Def. Given a set X. The full type structure over X M X = {X(A)} A T where X(A) is defined inductively as follows X(0) X; X(A B) X(B) X(A), the set of functions from X(A) into X(B) Def. M n M {1,,n} M(A B) M(A) M(B) M(2) M(1) = X X M(0) = X F M FM Partial view of M = M X F, M Λ ch finite at each level A if X is finite

13 Full type structures Def. Given a set X. The full type structure over X M X = {X(A)} A T where X(A) is defined inductively as follows X(0) X; X(A B) X(B) X(A), the set of functions from X(A) into X(B) Def. M n M {1,,n} M(A B) [F ] M(A) [M ] M(B) [FM ] M(2) M(1) = X X M(0) = X Partial view of M = M X F, M Λ ch finite at each level A if X is finite

14 Semantics in full type structures Let ρ : Var T M(A) be a valuation in M X : we require ρ(x A ) M(A) For M Λ (A) we define [M ] ρ M(A) [x A ] ρ ρ(x A ) [MN ] ρ [λx A.M ] ρ [M ] ρ [N ] ρ λd X(A).[M ] ρ(x A :=d) where ρ(x A : = d) = ρ with ρ (x A ) d ρ (y B ) ρ(y B ) if y B x A Define M X = M = N ρ [M ] ρ = [N ] ρ [M ] = [N ] if M,N Λ

15 Application We know that N = N, +,, 0, 1 can be λ-defined This is not so for the rational numbers Q = Q, +,,, :, 0, 1 1. Formulate this precisely. 2. Prove this. [Hint. Use that the homomorphic image of a field is the field itself; each M X (A) is finite for X finite.]

16 M 1, M 2 Def. Th(M)= {M = N M,N Λ & M = M = N} Th(M 1 ) is inconsistent: all terms of the same type are equated M 2 = c 1 = c 3 : M 2 = c 1 = c 2 : Exercises M 5 = c 4 = c 64 M 6 = c 4 = c 64 M 6 = c 5 = c 65 [Hint. Show that for i, j N one has M n = c i = c j i = j [i, j n 1 & i j(mod lcm{1,, n})]. For a M n (0), f M n (1) define the trace of a under f as {f i (a) i N}, directed by G f = {(a, b) f(a) = b}, which by the pigeonhole principle is lasso-shaped. Consider the traces of 1 under the functions f n, g m with 1 m n, where f n (k) = k + 1, if k < n, = n, if k = n, and g m (k) = k + 1, if k < m, = 1, if k = m, = k, else.]

17 Partial semantics (Friedman [1975]) Let M be a typed applicative structure A partial valuation in M is a family ρ = {ρ A } A T of partial maps ρ A : Var(A) M(A) The partial semantics [ ] M ρ : Λ (A) M(A) under ρ is [x A ] M ρ ρ A (x) [PQ] M ρ [λx A.P ] M ρ [P ] M ρ [Q]M ρ λd M(A).[P ] M ρ[x:=d] Often we write [M ] ρ for [M ] M ρ The expression [M ] ρ may not always be defined, even if ρ is total The problem arises with [λx.p ] ρ when λd M(A).[P ] M ρ[x:=d] M(B)M(A) M(A B) If [λx.p ] ρ exists it is uniquely defined

18 Typed λ-models A typed λ-model is a type structure M such that [M ] ρ is defined for all A T, M Λ(A), and ρ such that FV(M) dom(ρ) Examples of typed λ-models M X M βη : full type structures : open typed terms modulo βη-equality M[C] : closed typed term models modulo extensionality where C is a set of typed constants such that M[C](0) In M[C] one can define and show it works [M ] ρ = [M[ x := ρ( x)]]

19 Five Easy Pieces (Statman) There are only five Th(M[C]) coming from C 1 = {c 0,d 0 } C 2 = {c 0,f 1 } C 3 = {c 0,f 1,g 1 } C 4 = {c 0,Φ } C 5 = {c 0,b } There is a sixth, the inconsistent theory, coming from C 0 = {c 0 } One has Th(M[C 5 ]) Th(M[C 4 ]) Th(M[C 3 ]) Th(M[C 2 ]) Th(M[C 1 ]) Th(M[C 0 ]) Th(M[C 5 ]) = {M = N M = βη N} minimal theory Th(M[C 1 ]) is the unique maximally consistent theory consisting of all consistent equations together M[C 1 ] is the minimal model, with decidable equality (Loader)

20 M[C] Let C be a set of typed constants Examples C 0 = {c 0 }, C 1 = {c 0,d 0 } Define Λ [C] as the set of closed typed λ-terms built up from C Now Λ [C] modulo extensionality will be considered as a term model For M,N M[C](A) define M ext C N M = βη N if A = 0 P M[C](B).[MP ext C NP] if A = B C Then M ext C N P M[C].[M P = βη N P] Thm. M[C] = Λ [C]/ ext C is an extensional λ-model not trivial at all, we need M[C] = M = N M[C] = FM = FN & M[C] = λx.m = λx.n Exercises 1. M(c 0 ) = M 1, where M[c 0 ] = M[{c 0 }] 2. M[c 0, d 0 ] = c 1 = c 2 3. M[c 0, d 0 ] = M 2

21 Observational equality For M,N Λ [C](A) define M obs C N F : (A 0).FM = βη FN Remark M obs C N FM obs C FN M obs M ext Thm. M,N.[M obs C C N M ext C N C N Z.MZ ext C NZ N M ext Cor. M[C] is an (extensional) λ-model C N] non-trivial

22 Logical relations on M[C] A relation on M[C] is a family R = {R A } A T with R A M[C](A) n A relation is logical if for all A,B T and all M M[C](A B) n R A B (M 1,,M n ) N 1 M[C](A) N n M[C](A) Thus a logical relation is fully determined by R 0 [R A (N 1,,N n ) R B (M 1 N 1,,M n N n ) Prop. Suppose ext C is logical on M[C]. Then for all M,N M[C] M ext C Proof. Only ( ) is interesting N M C obs N Assume M C extn and F M[C](A 0) towards FM = βη FN Trivially F ext C F FM C ext FN, as ext C is logical FM = βη FN, as the type is 0

23 Analysis of ext C i (1) It remains to show that the ext C i are logical Def. BE is the logical relation on M[C] determined by BE 0 (M,N) M = βη N Lemma 1. Suppose BE(c, c) for c C. Then M Λ[C].BE(M, M) Proof. By the usual arguments for logical relations.

24 Analysis of C ext i (2) Lemma 2. Suppose BE(c, c) for all c C. Then ext C Proof. By Lemma 1 one has for all M M[C] is BE and hence logical BE(M, M) (0) It follows that BE is an equivalence relation on M[C]. We claim that for all F, G M[C](A) BE A (F, G) F ext C G, By induction on the structure of A. Case A = 0. By definition. Case A = B C, then ( ) BE B C (F, G) BE C (FP, GP), for all P M[C](B), ( ) since P ext C P and hence by the IH BE B (P, P) FP ext C GP, for all P M[C] by the IH F ext C G, by definition. F ext C G FP ext C GP, for all P M[C], BE C (FP, GP) (1) by the induction hypothesis. In order to prove BE B C (F, G), assume BE B (P, Q) towards BE C (FP, GQ). Well, since also BE B C (G, G), by (0), we have BE C (GP, GQ). (2) It follows from (1) and (2) and the transitivity of BE (which on this type is the same as by the IH) that BE C (FP, GQ) indeed. ext C By the claim ext is BE and therefore ext is logical. C C

25 Analysis of ext C i (3) Lemma 3. BE(M, M) holds for M M[C] of types 0, 1, Proof. Easy. Lemma 4. Let c = c 3 M[C]. Suppose Then BE A 0 (c, c) F, G M[C](2)[F ext C G F = βη G] Proof. Let c be given. Then for F, G M[C](2), P M[C](1) one has BE(F, G) FP = βη GP by Lemma 3 F ext C G F = βη G by assumption Therefore we have by definition BE(c, c) Last morgage For every F, G M[C](2) one has cf = βη cg F ext C 4 G F = βη G. We must show [ h M[C](1).Fh = βη Gh] F = βη G. (1)

26 Analysis of terms of given type λφx.x, λφx.φ(λf.x), λφx.φ(λf.f x), λφx.φ(λf.f(φ(λg.g(f x)))), λφx.φ(λf 1.w {f1 }x), λφx.φ(λf 1.w {f1 }Φ(λf 2.w {f1,f 2 }x)), ; λφx.φ(λf 1.w {f1 }Φ(λf 2.w {f1,f 2 } Φ(λf n.w {f1,,f n }x) )) w {f1 }, w {f1,f 2 },, w {f1,,f n } 3 o o f λφ 3 λx o o Φ λf 1 2 x Let h m λx.φ(λf.f m x) = f m : M[C](1) Claim F,G M[C](2) m N.[Fh m = Gh m F = βη G] See book p

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

Lambda Calculus. Week 12 The canonical term models for λ. Henk Barendregt, Freek Wiedijk assisted by Andrew Polonsky

Lambda Calculus. Week 12 The canonical term models for λ. Henk Barendregt, Freek Wiedijk assisted by Andrew Polonsky Lambda Calculus Week 12 The canonical term models for λ Henk Barendregt, Freek Wiedijk assisted by Andrew Polonsky Two version of λ Curry version (type assignment). Λ Γ (A) {M Λ Γ M : A} with (axiom) Γ

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

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

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

COMP6463: λ-calculus

COMP6463: λ-calculus COMP6463: λ-calculus 1. Basics Michael Norrish Michael.Norrish@nicta.com.au Canberra Research Lab., NICTA Semester 2, 2015 Outline Introduction Lambda Calculus Terms Alpha Equivalence Substitution Dynamics

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

Reducibility proofs in λ-calculi with intersection types

Reducibility proofs in λ-calculi with intersection types Reducibility proofs in λ-calculi with intersection types Fairouz Kamareddine, Vincent Rahli, and J. B. Wells ULTRA group, Heriot-Watt University, http://www.macs.hw.ac.uk/ultra/ March 14, 2008 Abstract

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

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

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

Combinators & Lambda Calculus

Combinators & Lambda Calculus Combinators & Lambda Calculus 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,

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

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

Realisability methods of proof and semantics with application to expansion

Realisability methods of proof and semantics with application to expansion Realisability methods of proof and semantics with application to expansion First Year Examination Supervisors : Professor Fairouz Kamareddine and Doctor Joe B. Wells Student : Vincent Rahli ULTRA group,

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

Graph lambda theories

Graph lambda theories Under consideration for publication in Math. Struct. in Comp. Science Graph lambda theories A N T O N I O B U C C I A R E L L I 1 and A N T O N I N O S A L I B R A 2 1 Equipe PPS (case 7014), Université

More information

λ Slide 1 Content Exercises from last time λ-calculus COMP 4161 NICTA Advanced Course Advanced Topics in Software Verification

λ Slide 1 Content Exercises from last time λ-calculus COMP 4161 NICTA Advanced Course Advanced Topics in Software Verification Content COMP 4161 NICTA Advanced Course Advanced Topics in Software Verification Toby Murray, June Andronick, Gerwin Klein λ Slide 1 Intro & motivation, getting started [1] Foundations & Principles Lambda

More information

Komponenten- und Service-orientierte Softwarekonstruktion

Komponenten- und Service-orientierte Softwarekonstruktion Komponenten- und Service-orientierte Softwarekonstruktion Vorlesung 5: Combinatory Logic Synthesis Jakob Rehof LS XIV Software Engineering TU Dortmund Sommersemester 2015 SS 2015 J. Rehof (TU Dortmund)

More information

Parameterizations and Fixed-Point Operators on Control Categories

Parameterizations and Fixed-Point Operators on Control Categories Parameterizations and Fixed-Point Operators on Control Categories oshihiko Kakutani 1 and Masahito Hasegawa 12 1 Research Institute for Mathematical Sciences, Kyoto University {kakutani,hassei}@kurims.kyoto-u.ac.jp

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

CS522 - Programming Language Semantics

CS522 - Programming Language Semantics 1 CS522 - Programming Language Semantics Simply Typed Lambda Calculus Grigore Roşu Department of Computer Science University of Illinois at Urbana-Champaign 2 We now discuss a non-trivial extension of

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

Functional Programming with Coq. Yuxin Deng East China Normal University

Functional Programming with Coq. Yuxin Deng East China Normal University Functional Programming with Coq Yuxin Deng East China Normal University http://basics.sjtu.edu.cn/ yuxin/ September 10, 2017 Functional Programming Y. Deng@ECNU 1 Reading materials 1. The Coq proof assistant.

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

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

Programming Language Concepts: Lecture 18

Programming Language Concepts: Lecture 18 Programming Language Concepts: Lecture 18 Madhavan Mukund Chennai Mathematical Institute madhavan@cmi.ac.in http://www.cmi.ac.in/~madhavan/courses/pl2009 PLC 2009, Lecture 18, 30 March 2009 One step reduction

More information

The Lambda Calculus. Stephen A. Edwards. Fall Columbia University

The Lambda Calculus. Stephen A. Edwards. Fall Columbia University The Lambda Calculus Stephen A. Edwards Columbia University Fall 2014 Lambda Expressions Function application written in prefix form. Add four and five is (+ 4 5) Evaluation: select a redex and evaluate

More information

Part 1. For any A-module, let M[x] denote the set of all polynomials in x with coefficients in M, that is to say expressions of the form

Part 1. For any A-module, let M[x] denote the set of all polynomials in x with coefficients in M, that is to say expressions of the form Commutative Algebra Homework 3 David Nichols Part 1 Exercise 2.6 For any A-module, let M[x] denote the set of all polynomials in x with coefficients in M, that is to say expressions of the form m 0 + m

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

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

Completeness Theorems and λ-calculus

Completeness Theorems and λ-calculus Thierry Coquand Apr. 23, 2005 Content of the talk We explain how to discover some variants of Hindley s completeness theorem (1983) via analysing proof theory of impredicative systems We present some remarks

More information

Graph models for the untyped λ-calculus

Graph models for the untyped λ-calculus Graph models for the untyped λ-calculus Kelley Philip van Evert On the cover: a picture I drew of Dana Scott. Graph models for the untyped λ-calculus Kelley Philip van Evert 4046854 Bachelor s thesis in

More information

The Curry-Howard Isomorphism

The Curry-Howard Isomorphism The Curry-Howard Isomorphism Software Formal Verification Maria João Frade Departmento de Informática Universidade do Minho 2008/2009 Maria João Frade (DI-UM) The Curry-Howard Isomorphism MFES 2008/09

More information

The following techniques for methods of proofs are discussed in our text: - Vacuous proof - Trivial proof

The following techniques for methods of proofs are discussed in our text: - Vacuous proof - Trivial proof Ch. 1.6 Introduction to Proofs The following techniques for methods of proofs are discussed in our text - Vacuous proof - Trivial proof - Direct proof - Indirect proof (our book calls this by contraposition)

More information

NICTA Advanced Course. Theorem Proving Principles, Techniques, Applications

NICTA Advanced Course. Theorem Proving Principles, Techniques, Applications NICTA Advanced Course Theorem Proving Principles, Techniques, Applications λ 1 CONTENT Intro & motivation, getting started with Isabelle Foundations & Principles Lambda Calculus Higher Order Logic, natural

More information

Constructive approach to relevant and affine term calculi

Constructive approach to relevant and affine term calculi Constructive approach to relevant and affine term calculi Jelena Ivetić, University of Novi Sad, Serbia Silvia Ghilezan,University of Novi Sad, Serbia Pierre Lescanne, University of Lyon, France Silvia

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

On Upper Bounds on the Church-Rosser Theorem

On Upper Bounds on the Church-Rosser Theorem On Upper Bounds on the Church-Rosser Theorem Ken-etsu Fujita Department of Computer Science Gunma University Kiryu, Japan fujita@cs.gunma-u.ac.jp The Church-Rosser theorem in the type-free λ-calculus is

More information

Part II Logic and Set Theory

Part II Logic and Set Theory Part II Logic and Set Theory Theorems Based on lectures by I. B. Leader Notes taken by Dexter Chua Lent 2015 These notes are not endorsed by the lecturers, and I have modified them (often significantly)

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

Semantics with Intersection Types

Semantics with Intersection Types Semantics with Intersection Types Steffen van Bakel Department of Computing, Imperial College of Science, Technology and Medicine, 180 Queen s Gate, London SW7 2BZ, U.K., E-mail: svb@doc.ic.ac.uk (Sections

More information

1 Completeness Theorem for First Order Logic

1 Completeness Theorem for First Order Logic 1 Completeness Theorem for First Order Logic There are many proofs of the Completeness Theorem for First Order Logic. We follow here a version of Henkin s proof, as presented in the Handbook of Mathematical

More information

TYPED LAMBDA CALCULI. Andrzej S. Murawski University of λeicester.

TYPED LAMBDA CALCULI. Andrzej S. Murawski University of λeicester. TYPED LAMBDA CALCULI Andrzej S. Murawski University of λeicester http://www.cs.le.ac.uk/people/amurawski/mgs2011-tlc.pdf THE COURSE The aim of the course is to provide an introduction to the lambda calculus

More information

NUMBER SYSTEMS. Number theory is the study of the integers. We denote the set of integers by Z:

NUMBER SYSTEMS. Number theory is the study of the integers. We denote the set of integers by Z: NUMBER SYSTEMS Number theory is the study of the integers. We denote the set of integers by Z: Z = {..., 3, 2, 1, 0, 1, 2, 3,... }. The integers have two operations defined on them, addition and multiplication,

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

Intensionality, Extensionality, and Proof Irrelevance in Modal Type Theory

Intensionality, Extensionality, and Proof Irrelevance in Modal Type Theory Intensionality, Extensionality, and Proof Irrelevance in Modal Type Theory Frank Pfenning LICS 01 Boston, Massachusetts June 17, 2001 Acknowledgments: Alberto Momigliano,... 1 Outline 1. Introduction 2.

More information

The Calculus of Inductive Constructions

The Calculus of Inductive Constructions The Calculus of Inductive Constructions Hugo Herbelin 10th Oregon Programming Languages Summer School Eugene, Oregon, June 16-July 1, 2011 1 Outline - A bit of history, leading to the Calculus of Inductive

More information

Linear Algebra M1 - FIB. Contents: 5. Matrices, systems of linear equations and determinants 6. Vector space 7. Linear maps 8.

Linear Algebra M1 - FIB. Contents: 5. Matrices, systems of linear equations and determinants 6. Vector space 7. Linear maps 8. Linear Algebra M1 - FIB Contents: 5 Matrices, systems of linear equations and determinants 6 Vector space 7 Linear maps 8 Diagonalization Anna de Mier Montserrat Maureso Dept Matemàtica Aplicada II Translation:

More information

Justifying Algorithms for βη-conversion

Justifying Algorithms for βη-conversion Justifying Algorithms for βη-conversion Healfdene Goguen AT&T Labs, 180 Park Ave., Florham Park NJ 07932 USA hhg@att.com. Abstract. Deciding the typing judgement of type theories with dependent types such

More information

Small families. (at INRIA with Gérard and in the historical λ-calculus) Jean-Jacques Lévy

Small families. (at INRIA with Gérard and in the historical λ-calculus) Jean-Jacques Lévy Small families (at INRIA with Gérard and in the historical λ-calculus) Jean-Jacques Lévy INRIA Rocquencourt and Microsoft Research-INRIA Joint Centre June 22, 2007 caml years coq sixty years is 31,557,600

More information

DEPARTMENT OF MATHEMATICS. MA1301 Discrete Mathematics

DEPARTMENT OF MATHEMATICS. MA1301 Discrete Mathematics SHRI ANGALAMMAN COLLEGE OF ENGINEERING AND TECHNOLOGY (An ISO 9001:2000 Certified Institution) SIRUGANOOR, TIRUCHIRAPPALLI 621 105 DEPARTMENT OF MATHEMATICS MA1301 Discrete Mathematics UNIT-I PART-A 1.Give

More information

Nominal Completion for Rewrite Systems with Binders

Nominal Completion for Rewrite Systems with Binders Nominal Completion for Rewrite Systems with Binders Maribel Fernández King s College London July 2012 Joint work with Albert Rubio Summary Motivations Nominal Rewriting Closed nominal rules Confluence

More information

Continuity. Chapter 4

Continuity. Chapter 4 Chapter 4 Continuity Throughout this chapter D is a nonempty subset of the real numbers. We recall the definition of a function. Definition 4.1. A function from D into R, denoted f : D R, is a subset of

More information

Chapter 2 Unbounded Operators and Abstract Functional Calculus

Chapter 2 Unbounded Operators and Abstract Functional Calculus Chapter 2 Unbounded Operators and Abstract Functional Calculus 2.1 Unbounded Operators We start with an introduction to unbounded operators and their spectral theory. This will be brief and cursory so

More information

Models of computation

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

More information

Baire category theorem and nowhere differentiable continuous functions

Baire category theorem and nowhere differentiable continuous functions Baire category theorem and nowhere differentiable continuous functions Takako Nemoto JAIST third CORE meeting 26 January 2018 Abstract In constructive mathematics, Baire Category Theorem has at least the

More information

TEST GROUPS FOR WHITEHEAD GROUPS

TEST GROUPS FOR WHITEHEAD GROUPS TEST GROUPS FOR WHITEHEAD GROUPS PAUL C. EKLOF, LÁSZLÓ FUCHS, AND SAHARON SHELAH Abstract. We consider the question of when the dual of a Whitehead group is a test group for Whitehead groups. This turns

More information

arxiv:cs/ v1 [cs.lo] 4 Jan 2007

arxiv:cs/ v1 [cs.lo] 4 Jan 2007 Definable Functions in the Simply Typed λ-calculus Mateusz Zakrzewski arxiv:cs/0701022v1 [cs.lo] 4 Jan 2007 Institute of Informatics, Warsaw University, Banacha 2, 02-097 Warsaw, Poland. mz201114@students.mimuw.edu.pl

More information

The Lifting Lemma. Ralf Hinze

The Lifting Lemma. Ralf Hinze The Lifting Lemma Ralf Hinze Computing Laboratory, University of Oxford Wolfson Building, Parks Road, Oxford, OX1 3QD, England ralf.hinze@comlab.ox.ac.uk http://www.comlab.ox.ac.uk/ralf.hinze/ June 2009

More information

Models of Computation,

Models of Computation, Models of Computation, 2010 1 The Lambda Calculus A brief history of mathematical notation. Our notation for numbers was introduced in the Western World in the Renaissance (around 1200) by people like

More information

Applied Logic. Lecture 1 - Propositional logic. Marcin Szczuka. Institute of Informatics, The University of Warsaw

Applied Logic. Lecture 1 - Propositional logic. Marcin Szczuka. Institute of Informatics, The University of Warsaw Applied Logic Lecture 1 - Propositional logic Marcin Szczuka Institute of Informatics, The University of Warsaw Monographic lecture, Spring semester 2017/2018 Marcin Szczuka (MIMUW) Applied Logic 2018

More information

Introduction to lambda calculus Part 2

Introduction to lambda calculus Part 2 Introduction to lambda calculus Part 2 Antti-Juhani Kaijanaho 2017-01-24... 1 Untyped lambda calculus 1.1 Syntax... x, y, z Var t, u Term t, u ::= x t u λx t... In this document, I will be using the following

More information

Probabilistic Applicative Bisimulation and Call-by-Value Lam

Probabilistic Applicative Bisimulation and Call-by-Value Lam Probabilistic Applicative and Call-by-Value Lambda Calculi Joint work with Ugo Dal Lago ENS Lyon February 9, 2014 Probabilistic Applicative and Call-by-Value Lam Introduction Fundamental question: when

More information

Typing λ-terms. Types. Typed λ-terms. Base Types. The Typing Relation. Advanced Formal Methods. Lecture 3: Simply Typed Lambda calculus

Typing λ-terms. Types. Typed λ-terms. Base Types. The Typing Relation. Advanced Formal Methods. Lecture 3: Simply Typed Lambda calculus Course 2D1453, 200607 Advanced Formal Methods Lecture 3: Simply Typed Lambda calculus Mads Dam KTH/CSC Some material from B. Pierce: TAPL + some from G. Klein, NICTA Typing λterms The uptyped λcalculus

More information

Chapter 8. P-adic numbers. 8.1 Absolute values

Chapter 8. P-adic numbers. 8.1 Absolute values Chapter 8 P-adic numbers Literature: N. Koblitz, p-adic Numbers, p-adic Analysis, and Zeta-Functions, 2nd edition, Graduate Texts in Mathematics 58, Springer Verlag 1984, corrected 2nd printing 1996, Chap.

More information

1.1. The Kleene Recursion Theorem

1.1. The Kleene Recursion Theorem 1.1. The Kleene Recursion Theorem This brief note covers Kleene s recursion Theorem and a few applications. 1.1.1 Theorem. Kleene s recursion theorem If λz x.fz, x n P, then for some e, Proof. Let φ n+1

More information

Investigation of Prawitz s completeness conjecture in phase semantic framework

Investigation of Prawitz s completeness conjecture in phase semantic framework Investigation of Prawitz s completeness conjecture in phase semantic framework Ryo Takemura Nihon University, Japan. takemura.ryo@nihon-u.ac.jp Abstract In contrast to the usual Tarskian set-theoretic

More information

1.5 The Nil and Jacobson Radicals

1.5 The Nil and Jacobson Radicals 1.5 The Nil and Jacobson Radicals The idea of a radical of a ring A is an ideal I comprising some nasty piece of A such that A/I is well-behaved or tractable. Two types considered here are the nil and

More information

Review 1. Andreas Klappenecker

Review 1. Andreas Klappenecker Review 1 Andreas Klappenecker Summary Propositional Logic, Chapter 1 Predicate Logic, Chapter 1 Proofs, Chapter 1 Sets, Chapter 2 Functions, Chapter 2 Sequences and Sums, Chapter 2 Asymptotic Notations,

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

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

summer school Logic and Computation Goettingen, July 24-30, 2016

summer school Logic and Computation Goettingen, July 24-30, 2016 Università degli Studi di Torino summer school Logic and Computation Goettingen, July 24-30, 2016 A bit of history Alonzo Church (1936) The as formal account of computation. Proof of the undecidability

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

Modèles des langages de programmation Domaines, catégories, jeux. Programme de cette seconde séance:

Modèles des langages de programmation Domaines, catégories, jeux. Programme de cette seconde séance: Modèles des langages de programmation Domaines, catégories, jeux Programme de cette seconde séance: Modèle ensembliste du lambda-calcul ; Catégories cartésiennes fermées 1 Synopsis 1 the simply-typed λ-calculus,

More information

Continuity. Chapter 4

Continuity. Chapter 4 Chapter 4 Continuity Throughout this chapter D is a nonempty subset of the real numbers. We recall the definition of a function. Definition 4.1. A function from D into R, denoted f : D R, is a subset of

More information

Notes for Math 601, Fall based on Introduction to Mathematical Logic by Elliott Mendelson Fifth edition, 2010, Chapman & Hall

Notes for Math 601, Fall based on Introduction to Mathematical Logic by Elliott Mendelson Fifth edition, 2010, Chapman & Hall Notes for Math 601, Fall 2010 based on Introduction to Mathematical Logic by Elliott Mendelson Fifth edition, 2010, Chapman & Hall All first-order languages contain the variables: v 0, v 1, v 2,... the

More information

A should be R-closed: R(A) A. We would like this to hold because we would like every element that the rules say should be in A to actually be in A.

A should be R-closed: R(A) A. We would like this to hold because we would like every element that the rules say should be in A to actually be in A. CS 6110 S18 Lecture 7 Inductive Definitions and Least Fixed Points 1 Set Operators Last time we considered a set of rule instances of the form X 1 X 2... X n, (1) X where X and the X i are members of some

More information

CS 6110 Lecture 35 Solving Domain Equations 19 April 2013 Lecturer: Andrew Myers

CS 6110 Lecture 35 Solving Domain Equations 19 April 2013 Lecturer: Andrew Myers CS 6110 Lecture 35 Solving Domain Equations 19 April 2013 Lecturer: Andrew Myers To develop a denotational semantics for a language with recursive types, or to give a denotational semantics for the untyped

More information

Programming Language Concepts: Lecture 16

Programming Language Concepts: Lecture 16 Programming Language Concepts: Lecture 16 Madhavan Mukund Chennai Mathematical Institute madhavan@cmi.ac.in http://www.cmi.ac.in/~madhavan/courses/pl2009 PLC 2009, Lecture 16, 23 March 2009 λ-calculus:

More information

Set Theory. CSE 215, Foundations of Computer Science Stony Brook University

Set Theory. CSE 215, Foundations of Computer Science Stony Brook University Set Theory CSE 215, Foundations of Computer Science Stony Brook University http://www.cs.stonybrook.edu/~cse215 Set theory Abstract set theory is one of the foundations of mathematical thought Most mathematical

More information

Chapter 1 Preliminaries

Chapter 1 Preliminaries Chapter 1 Preliminaries 1.1 Conventions and Notations Throughout the book we use the following notations for standard sets of numbers: N the set {1, 2,...} of natural numbers Z the set of integers Q the

More information

Part II. Logic and Set Theory. Year

Part II. Logic and Set Theory. Year Part II Year 2018 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2018 60 Paper 4, Section II 16G State and prove the ǫ-recursion Theorem. [You may assume the Principle of ǫ- Induction.]

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

Intersection Types and Lambda Theories

Intersection Types and Lambda Theories Intersection Types and Lambda Theories M.Dezani-Ciancaglini S.Lusin Abstract We illustrate the use of intersection types as a semantic tool for showing properties of the lattice of λ-theories. Relying

More information

TYPED LAMBDA CALCULUS. Volume I: λ A λ A = λ S. Henk Barendregt Wil Dekkers Richard Statman

TYPED LAMBDA CALCULUS. Volume I: λ A λ A = λ S. Henk Barendregt Wil Dekkers Richard Statman TYPED LAMBDA CALCULUS Volume I: λ A λ A = λ S Henk Barendregt Wil Dekkers Richard Statman Version: August 21, 2006 2 Preface DRAFT. DO NOT DISTRIBUTE. Bla bla. yghbkjhbkn. And we love our women. Nijmegen

More information

STATMAN S HIERARCHY THEOREM

STATMAN S HIERARCHY THEOREM Logical Methods in Computer Science Vol. 13(4:19)2017, pp. 1 39 https://lmcs.episciences.org/ Submitted Aug. 12, 2013 Published Nov. 27, 2017 STATMAN S HIERARCHY THEOREM BRAM WESTERBAAN, BAS WESTERBAAN,

More information

Extension theorems for homomorphisms

Extension theorems for homomorphisms Algebraic Geometry Fall 2009 Extension theorems for homomorphisms In this note, we prove some extension theorems for homomorphisms from rings to algebraically closed fields. The prototype is the following

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

Equational Reasoning in Algebraic Structures: a Complete Tactic

Equational Reasoning in Algebraic Structures: a Complete Tactic Equational Reasoning in Algebraic Structures: a Complete Tactic Luís Cruz-Filipe 1,2 and Freek Wiedijk 1 1 NIII, University of Nijmegen, Netherlands and 2 CLC, Lisbon, Portugal Abstract We present rational,

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

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

Alberto Carraro 1, 2 and Antonino Salibra 1

Alberto Carraro 1, 2 and Antonino Salibra 1 Theoretical Informatics and Applications Informatique Théorique et Applications Will be set by the publisher EASY LAMBDA-TERMS ARE NOT ALWAYS SIMPLE Alberto Carraro 1, 2 and Antonino Salibra 1 Abstract.

More information

The Minimal Graph Model of Lambda Calculus

The Minimal Graph Model of Lambda Calculus The Minimal Graph Model of Lambda Calculus Antonio Bucciarelli 1 and Antonino Salibra 2 1 Université Paris 7, Equipe PPS, 2 place Jussieu, 72251 Paris Cedex 05, France buccia@pps.jussieu.fr, 2 Università

More information

CSCI 490 problem set 6

CSCI 490 problem set 6 CSCI 490 problem set 6 Due Tuesday, March 1 Revision 1: compiled Tuesday 23 rd February, 2016 at 21:21 Rubric For full credit, your solutions should demonstrate a proficient understanding of the following

More information

Chapter 2 Axiomatic Set Theory

Chapter 2 Axiomatic Set Theory Chapter 2 Axiomatic Set Theory Ernst Zermelo (1871 1953) was the first to find an axiomatization of set theory, and it was later expanded by Abraham Fraenkel (1891 1965). 2.1 Zermelo Fraenkel Set Theory

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

Local Fields. Chapter Absolute Values and Discrete Valuations Definitions and Comments

Local Fields. Chapter Absolute Values and Discrete Valuations Definitions and Comments Chapter 9 Local Fields The definition of global field varies in the literature, but all definitions include our primary source of examples, number fields. The other fields that are of interest in algebraic

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

Elementary linear algebra

Elementary linear algebra Chapter 1 Elementary linear algebra 1.1 Vector spaces Vector spaces owe their importance to the fact that so many models arising in the solutions of specific problems turn out to be vector spaces. The

More information