On the Standardization Theorem for λβη-calculus

Size: px
Start display at page:

Download "On the Standardization Theorem for λβη-calculus"

Transcription

1 On the Standardization Theorem for λβη-calculus Ryo Kashima Department of Mathematical and Computing Sciences Tokyo Institute of Technology Ookayama, Meguro, Tokyo , Japan. September 2001 Abstract We present a new proof of the standardization theorem for λβη-calculus, which is performed by inductions based on an inductive definition of βηreducibility with a standard sequence. 1 Introduction The standardization theorem is a fundamental theorem in reduction theory of λ- calculus, which states that if a λ-term M β-(or βη-)reduces to a λ-term N, then there is a standard β-(or βη-)reduction sequence from M to N. In [3], the author gave a simple proof of the theorem for β-reduction. This paper extends the result to βη-reduction: we give a simple proof of the (weak) standardization theorem for βη-reduction. There have been some proofs of the standardization theorem in literature (e.g., [1, 2, 4, 5, 6, 7]). Compared with these, a feature of the presented proof is that we use an inductive definition (formal theory) of βη-reducibility with a standard sequence. In virtue of this definition, all the proof can be performed by easy inductions. Applications of this method to proofs of other theorems (e.g., the leftmost reduction theorem for βη-reduction) and other calculi (e.g., term rewriting systems) are future studies. 2 Preliminaries λ-terms are constructed by application and abstraction from variables (λ-terms of the form (MN) and (λx.m) are called an application and an abstraction respectively). Capital letters A, B,... denote arbitrary λ-terms, and small letters x, y,... denote arbitrary variables. M[x := N] denotes the result of substituting N for all the free occurrences of x in M with adequate renaming of bound variables. The set 1

2 of free variables in M is written by FV(M). We identify λ-terms that are mutually obtained by renaming of bound variables. In successive abstractions or applications, parentheses are omitted as follows: for example, λxyz.a = λx.(λy.(λz.a)), and ABCD = ((AB)C)D. (See, e.g., [1] for the basic notion and terminology.) The binary relation βη (one-step βη-reducibility) on the set of λ-terms are defined as usual: ( ((λx.a)b) ) βη ( (A[x := B]) ) and ( (λx.(cx)) ) βη ( C ) where x FV(C). The subterms (λx.a)b and λx.(cx) are called βη-redexes where the former and the latter are also called a β-redex and an η-redex respectively. Let R be an occurrence of a βη-redex in a λ-term M. We write M R βη N if and only if N is obtained from M by contracting the redex R. The relation l βη (one-step leftmost βη-reducibility) is defined as usual: M l βη N if and only if M R βη N for the leftmost βη-redex R in M, where a redex occurrence R 1 in M is said to be to the left of another redex occurence R 2 in M if they occur as follows. M = ( R 1 R 2 ) or M = ( ( R 2 ) ) }{{} R 1 The binary relations βη and l βη are the reflexive transitive closures of βη and l βη respectively. Suppose that M R βη N and that P and Q are subterm occurrences of M and N respectively. We write P Q if Q is a one step residual of P. For example, if ( ( {}} ) { ) M = P 1 (λx. ( P 3 )) ( P }{{} 4 ) P }{{} 5 A B P 2 Q 2 ( ( {}} ) { ) N = P 1 ( P 3 )[x := ( P }{{} 4 )] P }{{} 5 A B where R = (λx.a)b P 2 and P 3 x, then P 1 P 1, P 2 Q 2, P 3 P 3 [x := B], P 4 each copy of P 4 in A[x := B], and P 5 P 5. (Note that the redex (λx.a)b has no residual.) Suppose that ( X ) βη βη ( Y ). We say that Y is a residual of X if X Z 1 Z n Y for some Z 1,..., Z n (n 0). A βη-reduction sequence R M 1 R 1 βη M 2 2 βη Rn 1 βη M n is called weakly standard if the following condition is satisfied. 2

3 i [ R i+1 is not a residual of a βη-redex occurrence P in M i such that P is to the left of R i ] Moreover, the sequence is called strongly standard if the following condition is satisfied. i, j > i [ R j is not a residual of a βη-redex occurrence P in M i such that P is to the left of R i ] (The distinction between weak and strong appeared in [2]. Note that these two conditions are equivalent if η-reduction does not exist.) For example, the sequence λx.(iy(ix)) Iy βη λx.(y(ix)) Ix βη λx.(yx) λx.(yx) βη y is weakly and strongly standard; the sequence λx.(iy(ix)) Ix βη λx.(iyx) λx.(iyx) βη Iy Iy βη y is not strongly standard but weakly standard; and the sequence λx.(iyx) Iy βη λx.(yx) λx.(yx) βη y is neither strongly nor weakly standard, where I = λz.z. In this paper, we present a simple proof of the theorem: Theorem 2.1 (Weak Standardization Theorem) If M βη N, then there is a weakly standard βη-reduction sequence from M to N. Other important theorems, which have been proved in the literature (e.g., [4, 6]), are there: (Strong Standardization Theorem) If M βη N, then there is a strongly standard βη-reduction sequence from M to N. (Leftmost Reduction Theorem) If M βη N and N is a βη-normal form, then M l βη N. We will discuss them in Section 4. 3 Proof We define a formal theory which proves formulas of the forms A hap B and A st B. Axioms (Id) A hap A. (β) (λx.a)bc 1 C n hap A[x:=B]C 1 C n, where n 0. 3

4 Rules A hap B B hap C A hap C (Tr) L hap x L st x (Var) L hap AB A st C B st D L st CD L hap λx.a A st B L st λx.b L hap λx.a A st Bx with the proviso: L st B x FV(B) and B is not an abstraction. We write A hap B (or A st B) if and only if the formula A hap B (or A st B, respectively) is provable in this system. ( hap and st stand for head reduction in application and standard.) Theorem 3.1 If M hap N, then M l βη N. If M st N, then there is a weakly standard βη-reduction sequence from M to N. Proof By induction on the proof of M hap N or M st N. Here we show the only nontrivial case: The proof is.. M hap λx.a A st Nx M st N where x FV(N) and N is not an abstraction. By the induction hypotheses, there are a leftmost reduction sequence L from M to λx.a, and a weakly standard reduction sequence S from A to Nx. We will show that there is a weakly standard reduction sequence S + from λx.a to N; then the concatenation of L and S + is the required standard sequence from M to N. We will explain, based on an example, the definition of the sequence S +. If a λ-term P is of the form P x and x FV(P ), then we say that P is an η-body for x. Suppose that the weakly standard reduction sequence S is where A R 1 βη A R 2 βη Bx R 3 βη (λy.(cy))x (λy.(cy))x βη Cx R 5 βη Nx Bx, (λy.(cy))x, Cx, and Nx are η-bodies for x; 4

5 A is not an η-body for x; B R 3 βη λy.(cy); and C R 5 βη N. Note that R 3 = B; otherwise, reduction of R 3 cannot make λy.(cy) if B is an application, and S is not weakly standard if B is an abstraction. Then, the weakly standard sequence S + is defined as follows. λx.a R 1 βη λx.a R 2 βη λx.(bx) λx.(bx) βη B R 3 βη λy.(cy) λy.(cy) βη C R 5 βη N. Lemma 3.2 (1) If M hap N, then MP hap NP. (2) If L hap M st N, then L st N. (3) If M hap N, then M[z := P ] hap N[z := P ]. Proof (1) By induction on the proof of M hap N. (2) If M st N is proved, then there must be a premise M hap P for certain P. From this and the assumption L hap M, we can infer L hap P by the rule (Tr). Then L st N is proved by the rule that infers M st N. (3) By induction on the proof of M hap N. Lemma 3.3 If M st N and P st y, then M[z := P ] st N[z := y]. Proof By induction on the proof of M st N. We divide cases according to the last inference of the proof. The substitution [z := P ] and [z := y] will be represented by [P ] and [y] for short. (Case 1): The last inference is where N = x z. In this case, we have (Case 2): The last inference is M hap x M st x (Var) and Lemma 3.2(3) M[P ] hap x (Var) M[P ] st x. M hap z M st z 5 (Var)

6 where N = z. In this case, we have and Lemma 3.2(3) M[P ] hap P M[P ] st y.. assumption of the lemma P st y Lemma 3.2(2) (Case 3): The last inference is. σ M hap AB A st C M st CD B st D where N = CD. In this case, we have and Lem.3.2(3). i.h. for σ M[P ] hap (AB)[P ] A[P ] st C[y] M[P ] st (CD)[y].. i.h. for τ B[P ] st D[y] (Case 4): The last inference is where N = λx.b. If x z, then we have. σ M hap λx.a A st B M st λx.b and Lem.3.2(3). i.h. for σ M[P ] hap (λx.a)[p ] A[P ] st B[y] M[P ] st (λx.b)[y] where we assume that x FV(P, y) (otherwise we rename x). If x = z, then (λx.x)[z := Z] = λx.x, and the induction hypothesis is not necessary. (Case 5): The last inference is. σ M hap λx.a A st Nx M st N where x FV(N) and N is not an abstraction. If x z, then we have and Lem.3.2(3). i.h. for σ M[P ] hap (λx.a)[p ] A[P ] st (Nx)[y] M[P ] st N[y] where we assume that x FV(P, y) (otherwise we rename x). Note that (Nx)[y] = (N[y])x and the proviso for N[y] is satisfied. If x = z, then the induction hypothesis is not necessary. 6

7 Lemma 3.4 If L st (λx 1 x m.m)y 1 y m F 1 F n, then L st M[x 1 :=y 1,..., x m := y m ]F 1 F n, where m 1, n 0 and x 1,..., x m are distinct. (Note that [x 1 := y 1,..., x m := y m ] is a simultaneous substitution, and this will be represented by [ y] for short.) Proof By induction on the proof of L st (λx 1 x m.m)y 1 y m F 1 F n. We divide cases according to the last inference of the proof. (Case 1): n = 0, and the proof is L hap AB. σ A st (λx 1 x m.m)y 1 y m 1 L st (λx 1 x m.m)y 1 y m. B st y m If m 2, then by the induction hypothesis for σ, there is a proof. σ A st (λx m.m)[ y ] where [ y ] = [x 1 := y 1,..., x m 1 := y m 1 ]. If m = 1, then we define σ = σ. In any case, the proof σ must be of the form. φ A hap λx m.c. ψ C st M[ y ] A st λx m.(m[ y ]). (Note that x m {y 1,..., y m 1 }; otherwise we rename x m.) Then we have where ( ) is. ( ). ( ) L hap C[x m :=B] C[x m :=B] st M[ y] Lem. 3.2(2) L st M[ y] L hap AB. φ A hap λx m.c AB hap (λx m.c)b Lem.3.2(1) (axiom β) (λx m.c)b hap C[x m :=B] L hap C[x m :=B] (Tr) 2 and ( ) is obtained by ψ, τ and Lemma 3.3. (Case 2): n 1, and the proof is L hap AB. σ A st (λx 1 x m.m)y 1 y m F 1 F n 1 L st (λx 1 x m.m)y 1 y m F 1 F n. 7 B st F n

8 In this case, we have L hap AB (Case 3): The proof is. i.h. for σ A st M[ y]f 1 F n 1 L st M[ y]f 1 F n. B st F n. σ L hap λz.a A st (λx 1 x m.m)y 1 y m F 1 F n z L st (λx 1 x m.m)y 1 y m F 1 F n where z FV((λx 1 x m.m)y 1 y m F 1 F n ). If M[ y]f 1 F n is not an abstraction, then we have. i.h. for σ L hap λz.a A st M[ y]f 1 F n z L st M[ y]f 1 F n. Note that z FV(M[ y]f 1 F n ) FV((λx 1 x m.m)y 1 y m F 1 F n ). If M[ y]f 1 F n is an abstraction, then n = 0, M = λv.b, and σ is. σ A st (λx 1 x m v.b)y 1 y m z. where v {x 1,..., x m, y 1,..., y m } (otherwise, we rename v). Then we have. i.h. for σ L hap λz.a A st B[ y, z] L st λz.(b[ y, z]) = (λv.b)[ y] where [ y, z] = [x 1 :=y 1,..., x m :=y m, v :=z]. We consider an inference rule: L hap λx.a A st Bx L st B (η + ) with the proviso: x FV(B). This is an extension of rule (B may be an abstraction). Lemma 3.5 The rule (η + ) is admissible; that is, if L hap λx.a, A st Bx, and x FV(B), then L st B. Proof If B is not an abstraction, then (η + ) is just the rule. If B = λy.c, then we have A st (λy.c)x L hap λx.a A st C[y := x] Lem.3.4 L st λx.(c[y := x]) = λy.c. Note that x FV(C). 8

9 Lemma 3.6 If M st N and P st Q, then M[z := P ] st N[z := Q]. Proof Similar to the proof of Lemma 3.3 (y = Q). The only difference is that N[z := Q] may be an abstraction, in Case 5, that is in contravention of the proviso of rule. In such a case, we use the rule (η + ) (Lemma 3.5) to infer M[P ] st N[Q]. Lemma 3.7 If L st (λx.m)nf 1 F n, then L st M[x := N]F 1 F n, where n 0. Proof Similar to the proof of Lemma 3.4. (m = 1 and y m = N. In Case 1, we use Lemma 3.6 instead of 3.3. In Case 3, we use (η + ) rule (Lemma 3.5).) Lemma 3.8 If L st M βη N, then L st N. Proof By induction on the proof of L st M. We divide cases according to the last inference of the proof. Let R be the occurrence of the βη-redex such that M R βη N. (Case 1): The proof is. σ L hap AB A st C L st CD B st D where M = CD. (Subcase 1-1): R = CD; that is, C = λx.e, M = (λx.e)d and N = E[x := D]. This is a special case of Lemma 3.7. (Subcase 1-2): R is in C; that is, C R βη C and N = C D. In this case, we have L hap AB. i.h. for σ A st C L st C D. B st D (Subcase 1-3): R is in D. This is similar to Subcase 1-2. (Case 2): The proof is. σ L hap λx.a A st B L st λx.b where M = λx.b. (Subcase 2-1): R = λx.b; that is, B = Nx, M = λx.(nx), and x FV(N). This is just the rule (η + ) (Lemma 3.5). 9

10 (Subcase 2-2): R is in B; that is, B R βη B, and N = λx.b. Then we have (Case 3): The proof is. i.h. for σ L hap λx.a A st B L st λx.b.. σ L hap λx.a A st Mx L st M where x FV(M) and M is not an abstraction. In this case, we have. i.h. for σ (because Mx βη Nx) L hap λx.a A st Nx (η L st N. + ) (Lem. 3.5) Note that x FV(N) FV(M). Lemma 3.9 M st M. Proof By induction on the structure of M. Theorem 3.10 If M βη N, then M st N. Proof Suppose M = M 1 βη M 2 βη βη M k = N. We can show M st M i for i = 1,..., k, by Lemmas 3.9 and 3.8. Now the Weak Standardization Theorem 2.1 is obvious by Theorems 3.1 and Remarks (1) It seems that we can prove, by the similar proof of Theorem 3.1, the strong version of it: If M st N, then there is a strongly standard βη-reduction sequence from M to N. Then the Strong Standardization Theorem for βη-reduction is proved. (2) In the case of β-reduction, the Leftmost Reduction Theorem is an easy corollary to the Standardization Theorem because we have the following: If M R 1 β Rn β N is a standard β-reduction sequence and N is a β-normal form, then R 1,..., R n are all the leftmost occurrences of β-redexes. However, this does not hold for βηreduction: there are counterexamples ( ) ( ) Ix λx.((λy.(yy))x) λx. (λy.(yy))(ix) βη λx. (λy.(yy))x βη λy.(yy) 10

11 and ( ) I(λy.(yy)) ( ) (λy.(yy))x λx. I(λy.(yy))x βη λx. (λy.(yy))x βη λx.(xx) which are strongly standard and end with βη-normal forms, but neither of them is a leftmost reduction sequence. Note that these can be regarded as the sequences ( ) ( ) Ix (λy.(yy))x λx. (λy.(yy))(ix) βη λx. (λy.(yy))x βη λx.(xx) and ( ) I(λy.(yy)) ( ) λx.((λy.(yy))x) λx. I(λy.(yy))x βη λx. (λy.(yy))x βη λy.(yy), neither of which is weakly ( standard; ) then these are not counterexamples. overlap of redexes λx. (λy.(yy))x causes a problem. The References [1] H.P. Barendregt, The Lambda Calculus (North-Holland, 1984). [2] R. Hindley, Standard and normal reductions, Trans. Amer. Math. Soc. 241 (1978) [3] R. Kashima, A proof of the standardization theorem in λ-calculus, Research Reports on Mathematical and Computing Sciences C-145, (Tokyo Institute of Technology, 2000). [4] J.W. Klop, Combinatory Reduction Systems, Mathematical Center Tracts 127, Amsterdam (1980). [5] G. Mitschke, The standardization theorem for λ-calculus, Zeitshr. Math. Logik Grundlag. Math. 25 (1979) [6] M. Takahashi, Parallel reductions in λ-calculus, Information and Computation 118 (1995) [7] H. Xi, Upper bounds for standardizations and an application, J. Symbolic Logic 64 (1999)

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

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

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

Proof Theoretical Studies on Semilattice Relevant Logics

Proof Theoretical Studies on Semilattice Relevant Logics Proof Theoretical Studies on Semilattice Relevant Logics 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

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

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

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

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

Traditional and Non Traditional lambda calculi

Traditional and Non Traditional lambda calculi Strategies July 2009 Strategies Syntax Semantics Manipulating Expressions Variables and substitutions Free and bound variables Subterms and substitution Grafting and substitution Ordered list of variables

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

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

Lambda Calculus and Types

Lambda Calculus and Types Lambda Calculus and Types (complete) Andrew D. Ker 16 Lectures, Hilary Term 2009 Oxford University Computing Laboratory ii Contents Introduction To The Lecture Notes vii 1 Terms, Equational Theory 1 1.1

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

Infinite λ-calculus and non-sensible models

Infinite λ-calculus and non-sensible models Infinite λ-calculus and non-sensible models Alessandro Berarducci Dipartimento di Matematica, Università di Pisa Via Buonarroti 2, 56127 Pisa, Italy berardu@dm.unipi.it July 7, 1994, Revised Nov. 13, 1994

More information

Computational Soundness of a Call by Name Calculus of Recursively-scoped Records. UMM Working Papers Series, Volume 2, Num. 3.

Computational Soundness of a Call by Name Calculus of Recursively-scoped Records. UMM Working Papers Series, Volume 2, Num. 3. Computational Soundness of a Call by Name Calculus of Recursively-scoped Records. UMM Working Papers Series, Volume 2, Num. 3. Elena Machkasova Contents 1 Introduction and Related Work 1 1.1 Introduction..............................

More information

Rewriting, Explicit Substitutions and Normalisation

Rewriting, Explicit Substitutions and Normalisation Rewriting, Explicit Substitutions and Normalisation XXXVI Escola de Verão do MAT Universidade de Brasilia Part 1/3 Eduardo Bonelli LIFIA (Fac. de Informática, UNLP, Arg.) and CONICET eduardo@lifia.info.unlp.edu.ar

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

AN ALTERNATIVE NATURAL DEDUCTION FOR THE INTUITIONISTIC PROPOSITIONAL LOGIC

AN ALTERNATIVE NATURAL DEDUCTION FOR THE INTUITIONISTIC PROPOSITIONAL LOGIC Bulletin of the Section of Logic Volume 45/1 (2016), pp 33 51 http://dxdoiorg/1018778/0138-068045103 Mirjana Ilić 1 AN ALTERNATIVE NATURAL DEDUCTION FOR THE INTUITIONISTIC PROPOSITIONAL LOGIC Abstract

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

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

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

SHARING IN THE WEAK LAMBDA-CALCULUS REVISITED

SHARING IN THE WEAK LAMBDA-CALCULUS REVISITED SHARING IN THE WEAK LAMBDA-CALCULUS REVISITED TOMASZ BLANC, JEAN-JACQUES LÉVY, AND LUC MARANGET INRIA e-mail address: tomasz.blanc@inria.fr INRIA, Microsoft Research-INRIA Joint Centre e-mail address:

More information

arxiv: v1 [cs.lo] 29 May 2014

arxiv: v1 [cs.lo] 29 May 2014 An Introduction to the Clocked Lambda Calculus Jörg Endrullis, Dimitri Hendriks, Jan Willem Klop, and Andrew Polonsky VU University Amsterdam, The Netherlands Abstract We give a brief introduction to the

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

Beyond First-Order Logic

Beyond First-Order Logic Beyond First-Order Logic Software Formal Verification Maria João Frade Departmento de Informática Universidade do Minho 2008/2009 Maria João Frade (DI-UM) Beyond First-Order Logic MFES 2008/09 1 / 37 FOL

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

THE A-CALCULUS IS c-incomplete

THE A-CALCULUS IS c-incomplete THE JOURNAL OF SYSTOLIc LoGIc Volume 39, Number 2, June 1974 THE A-CALCULUS IS c-incomplete G. D. PLOTKIN?1. Introduction. The w-rule in the A-calculus (or, more exactly, the AK-fg, 7 calculus) is MZ =

More information

Computation Theory, L 9 116/171

Computation Theory, L 9 116/171 Definition. A partial function f is partial recursive ( f PR) ifitcanbebuiltupinfinitelymanysteps from the basic functions by use of the operations of composition, primitive recursion and minimization.

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

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

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

On the Complexity of the Reflected Logic of Proofs

On the Complexity of the Reflected Logic of Proofs On the Complexity of the Reflected Logic of Proofs Nikolai V. Krupski Department of Math. Logic and the Theory of Algorithms, Faculty of Mechanics and Mathematics, Moscow State University, Moscow 119899,

More information

Abstract A new proof is given of the analogue of Böhm s Theorem in the typed lambda calculus with functional types.

Abstract A new proof is given of the analogue of Böhm s Theorem in the typed lambda calculus with functional types. The Typed Böhm Theorem Kosta Došen University of Toulouse III, IRIT 31062 Toulouse cedex, France and Mathematical Institute Knez Mihailova 35, PO Box 367 11001 Belgrade, Yugoslavia email: kosta@misanuacyu

More information

EXTENDED ABSTRACT. 2;4 fax: , 3;5 fax: Abstract

EXTENDED ABSTRACT. 2;4 fax: , 3;5 fax: Abstract 1 Syntactic denitions of undened: EXTENDED ABSTRACT on dening the undened Zena Ariola 1, Richard Kennaway 2, Jan Willem Klop 3, Ronan Sleep 4 and Fer-Jan de Vries 5 1 Computer and Information Science Department,

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

Consequence Relations and Natural Deduction

Consequence Relations and Natural Deduction Consequence Relations and Natural Deduction Joshua D. Guttman Worcester Polytechnic Institute September 9, 2010 Contents 1 Consequence Relations 1 2 A Derivation System for Natural Deduction 3 3 Derivations

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

1. each λ-variable is a λρ-term, called atom or atomic term, 2. if M and N are λρ-term then (MN) is a λρ-term called application,

1. each λ-variable is a λρ-term, called atom or atomic term, 2. if M and N are λρ-term then (MN) is a λρ-term called application, Yuichi Komori Arato Cho λρ-calculus abstract. In [K02], one of the authors introduced the system λρ-calculus and stated without proof that the strong normalization theorem hold. We have discovered an elegant

More information

An Implicit Characterization of PSPACE

An Implicit Characterization of PSPACE An Implicit Characterization of PSPACE Marco Gaboardi Dipartimento di Scienze dell Informazione, Università degli Studi di Bologna - Mura Anteo Zamboni 7, 40127 Bologna, Italy, gaboardi@cs.unibo.it and

More information

SOME REMARKS ON MAEHARA S METHOD. Abstract

SOME REMARKS ON MAEHARA S METHOD. Abstract Bulletin of the Section of Logic Volume 30/3 (2001), pp. 147 154 Takahiro Seki SOME REMARKS ON MAEHARA S METHOD Abstract In proving the interpolation theorem in terms of sequent calculus, Maehara s method

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

Classical Combinatory Logic

Classical Combinatory Logic Computational Logic and Applications, CLA 05 DMTCS proc. AF, 2006, 87 96 Classical Combinatory Logic Karim Nour 1 1 LAMA - Equipe de logique, Université de Savoie, F-73376 Le Bourget du Lac, France Combinatory

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

Parallel Reduction in Type Free λµ-calculus

Parallel Reduction in Type Free λµ-calculus Electronic Notes in Theoretical Computer Science 42 (2001) URL: http://www.elsevier.nl/locate/entcs/volume42.html 15 pages Parallel Reduction in Type Free λµ-calculus Kensuke Baba 1 Graduate School of

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

TR : Binding Modalities

TR : Binding Modalities City University of New York (CUNY) CUNY Academic Works Computer Science Technical Reports Graduate Center 2012 TR-2012011: Binding Modalities Sergei N. Artemov Tatiana Yavorskaya (Sidon) Follow this and

More information

Modularity of Confluence: A Simplified Proof

Modularity of Confluence: A Simplified Proof 1 Modularity of Confluence: A Simplified Proof Jan Willem Klop 1,2,5,6 Aart Middeldorp 3,5 Yoshihito Toyama 4,7 Roel de Vrijer 2 1 Department of Software Technology CWI, Kruislaan 413, 1098 SJ Amsterdam

More information

A general method to prove the normalization theorem for first and second order typed λ-calculi

A general method to prove the normalization theorem for first and second order typed λ-calculi Under consideration for publication in Math. Struct. in Comp. Science A general method to prove the normalization theorem for first and second order typed λ-calculi Venanzio Capretta and Silvio Valentini

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

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

Parallel Reduction in Type Free Lambda-mu- Calculus

Parallel Reduction in Type Free Lambda-mu- Calculus 九州大学学術情報リポジトリ Kyushu University Institutional Repository Parallel Reduction in Type Free Lambda-mu- Calculus Baba, Kensuke Graduate School of Information Science and Electrical Engineering, Kyushu University

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

Computer Science at Kent

Computer Science at Kent Computer Science at Kent New eta-reduction and Church-Rosser Yong Luo Technical Report No. 7-05 October 2005 Copyright c 2005 University of Kent Published by the Computing Laboratory, University of Kent,

More information

Silvia Ghilezan and Jelena Ivetić

Silvia Ghilezan and Jelena Ivetić PUBLICATIONS DE L INSTITUT MATHÉMATIQUE Nouvelle série, tome 82(96) (2007), 85 91 DOI 102298/PIM0796085G INTERSECTION TYPES FOR λ Gtz -CALCULUS Silvia Ghilezan and Jelena Ivetić Abstract. We introduce

More information

An Introduction to the Lambda Calculus

An Introduction to the Lambda Calculus An Introduction to the Lambda Calculus Mayer Goldberg February 20, 2000 1 Notation and Conventions It is surprising that despite the simplicity of its syntax, the λ-calculus hosts a large body of notation,

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

Informal Statement Calculus

Informal Statement Calculus FOUNDATIONS OF MATHEMATICS Branches of Logic 1. Theory of Computations (i.e. Recursion Theory). 2. Proof Theory. 3. Model Theory. 4. Set Theory. Informal Statement Calculus STATEMENTS AND CONNECTIVES Example

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

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

A Behavioural Model for Klop s Calculus

A Behavioural Model for Klop s Calculus Replace this file with prentcsmacro.sty for your meeting, or with entcsmacro.sty for your meeting. Both can be found at the ENTCS Macro Home Page. A Behavioural Model for Klop s Calculus Mariangiola Dezani-Ciancaglini

More information

Partially commutative linear logic: sequent calculus and phase semantics

Partially commutative linear logic: sequent calculus and phase semantics Partially commutative linear logic: sequent calculus and phase semantics Philippe de Groote Projet Calligramme INRIA-Lorraine & CRIN CNRS 615 rue du Jardin Botanique - B.P. 101 F 54602 Villers-lès-Nancy

More information

FIXED POINTS AND EXTENSIONALITY IN TYPED FUNCTIONAL PROGRAMMING LANGUAGES

FIXED POINTS AND EXTENSIONALITY IN TYPED FUNCTIONAL PROGRAMMING LANGUAGES FIXED POINTS AND EXTENSIONALITY IN TYPED FUNCTIONAL PROGRAMMING LANGUAGES a dissertation submitted to the department of computer science and the committee on graduate studies of stanford university in

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

Strong normalization of a symmetric lambda calculus for second order classical logic

Strong normalization of a symmetric lambda calculus for second order classical logic Archive for Mathematical Logic manuscript No. (will be inserted by the editor) Strong normalization of a symmetric lambda calculus for second order classical logic YAMAGATA, yoriyuki e-mail: yoriyuki@ms.u-tokyo.ac.jp

More information

A syntactical proof of the operational equivalence of two λ-terms

A syntactical proof of the operational equivalence of two λ-terms A syntactical proof of the operational equivalence of two λ-terms René DAVID and Karim NOUR Abstract In this paper we present a purely syntactical proof of the operational equivalence of I = λxx and the

More information

Lecture Notes on Sequent Calculus

Lecture Notes on Sequent Calculus Lecture Notes on Sequent Calculus 15-816: Modal Logic Frank Pfenning Lecture 8 February 9, 2010 1 Introduction In this lecture we present the sequent calculus and its theory. The sequent calculus was originally

More information

Rewriting for Fitch style natural deductions

Rewriting for Fitch style natural deductions Rewriting for Fitch style natural deductions Herman Geuvers, Rob Nederpelt Nijmegen University, The Netherlands Eindhoven University of Technology, The Netherlands bstract Logical systems in natural deduction

More information

Parametric λ-theories

Parametric λ-theories Parametric λ-theories Luca Paolini 1 Dipartimento di Informatica Università degli Studi di Torino Corso Svizzera, 185 10149 Torino - Italy e-mail: paolini@di.unito.it Abstract The parametric lambda calculus

More information

Solutions to Exercises. Solution to Exercise 2.4. Solution to Exercise 2.5. D. Sabel and M. Schmidt-Schauß 1

Solutions to Exercises. Solution to Exercise 2.4. Solution to Exercise 2.5. D. Sabel and M. Schmidt-Schauß 1 D. Sabel and M. Schmidt-Schauß 1 A Solutions to Exercises Solution to Exercise 2.4 We calculate the sets of free and bound variables: FV ((λy.(y x)) (λx.(x y)) (λz.(z x y))) = FV ((λy.(y x)) (λx.(x y)))

More information

The Greek Alphabet. (a) The Untyped λ-calculus

The Greek Alphabet. (a) The Untyped λ-calculus 3. The λ-calculus and Implication Greek Letters (a) The untyped λ-calculus. (b) The typed λ-calculus. (c) The λ-calculus in Agda. (d) Logic with Implication (e) Implicational Logic in Agda. (f) More on

More information

M, N ::= x λp : A.M MN (M, N) () c A. x : b p x : b

M, N ::= x λp : A.M MN (M, N) () c A. x : b p x : b A PATTERN-MATCHING CALCULUS FOR -AUTONOMOUS CATEGORIES ABSTRACT. This article sums up the details of a linear λ-calculus that can be used as an internal language of -autonomous categories. The coherent

More information

Equivalent Types in Lambek Calculus and Linear Logic

Equivalent Types in Lambek Calculus and Linear Logic Equivalent Types in Lambek Calculus and Linear Logic Mati Pentus Steklov Mathematical Institute, Vavilov str. 42, Russia 117966, Moscow GSP-1 MIAN Prepublication Series for Logic and Computer Science LCS-92-02

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

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

a 11 x 1 + a 12 x a 1n x n = b 1 a 21 x 1 + a 22 x a 2n x n = b 2.

a 11 x 1 + a 12 x a 1n x n = b 1 a 21 x 1 + a 22 x a 2n x n = b 2. Chapter 1 LINEAR EQUATIONS 11 Introduction to linear equations A linear equation in n unknowns x 1, x,, x n is an equation of the form a 1 x 1 + a x + + a n x n = b, where a 1, a,, a n, b are given real

More information

The Syntax of First-Order Logic. Marc Hoyois

The Syntax of First-Order Logic. Marc Hoyois The Syntax of First-Order Logic Marc Hoyois Table of Contents Introduction 3 I First-Order Theories 5 1 Formal systems............................................. 5 2 First-order languages and theories..................................

More information

Lambda calculus L9 103

Lambda calculus L9 103 Lambda calculus L9 103 Notions of computability L9 104 Church (1936): λ-calculus Turing (1936): Turing machines. Turing showed that the two very different approaches determine the same class of computable

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

Sub-λ-calculi, Classified

Sub-λ-calculi, Classified Electronic Notes in Theoretical Computer Science 203 (2008) 123 133 www.elsevier.com/locate/entcs Sub-λ-calculi, Classified François-Régis Sinot Universidade do Porto (DCC & LIACC) Rua do Campo Alegre

More information

Formulas for which Contraction is Admissible

Formulas for which Contraction is Admissible Formulas for which Contraction is Admissible ARNON AVRON, Department of Computer Science, School of Mathematical Sciences, Tel Aviv University, Tel Aviv 69978, Israel. E-mail: aa@math.tau.ac.il Abstract

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

Typed Lambda Calculi. Nikos Tzeveλekos Queen Mary, University of London 1 / 23

Typed Lambda Calculi. Nikos Tzeveλekos Queen Mary, University of London 1 / 23 Typed Lambda Calculi Nikos Tzeveλekos Queen Mary, University of London 1 / 23 What is the Lambda Calculus A minimal formalism expressing computation with functionals s ::= x λx.s ss All you need is lambda.

More information

5. The Logical Framework

5. The Logical Framework 5. The Logical Framework (a) Judgements. (b) Basic form of rules. (c) The non-dependent function type and product. (d) Structural rules. (Omitted 2008). (e) The dependent function set and -quantification.

More information

Annals of Pure and Applied Logic 130 (2004) On the λy calculus. Rick Statman

Annals of Pure and Applied Logic 130 (2004) On the λy calculus. Rick Statman Annals of Pure and Applied Logic 130 (2004) 325 337 www.elsevier.com/locate/apal On the λy calculus Rick Statman Department of Mathematical Sciences, Carnegie Mellon University, Pittsburgh, PA 15213, USA

More information

hal , version 1-21 Oct 2009

hal , version 1-21 Oct 2009 ON SKOLEMISING ZERMELO S SET THEORY ALEXANDRE MIQUEL Abstract. We give a Skolemised presentation of Zermelo s set theory (with notations for comprehension, powerset, etc.) and show that this presentation

More information

3. The λ-calculus and Implication

3. The λ-calculus and Implication 3. The λ-calculus and Implication (a) (b) (c) (d) (e) (f) The untyped λ-calculus. The typed λ-calculus. The λ-calculus in Agda. Logic with Implication Implicational Logic in Agda. More on the typed λ-calculus.

More information

Handout: Proof of the completeness theorem

Handout: Proof of the completeness theorem MATH 457 Introduction to Mathematical Logic Spring 2016 Dr. Jason Rute Handout: Proof of the completeness theorem Gödel s Compactness Theorem 1930. For a set Γ of wffs and a wff ϕ, we have the following.

More information

Standardization of a call-by-value calculus

Standardization of a call-by-value calculus Standardization of a call-by-value calculus Giulio Guerrieri 1, Luca Paolini 2, and Simona Ronchi Della Rocca 2 1 Laboratoire PPS, UMR 7126, Université Paris Diderot, Sorbonne Paris Cité F-75205 Paris,

More information

ELEMENTARY LINEAR ALGEBRA

ELEMENTARY LINEAR ALGEBRA ELEMENTARY LINEAR ALGEBRA K R MATTHEWS DEPARTMENT OF MATHEMATICS UNIVERSITY OF QUEENSLAND First Printing, 99 Chapter LINEAR EQUATIONS Introduction to linear equations A linear equation in n unknowns x,

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

Call-by-value non-determinism in a linear logic type discipline

Call-by-value non-determinism in a linear logic type discipline Call-by-value non-determinism in a linear logic type discipline Alejandro Díaz-Caro? Giulio Manzonetto Université Paris-Ouest & INRIA LIPN, Université Paris 13 Michele Pagani LIPN, Université Paris 13

More information

A general method for proving the normalization theorem for first and second order typed λ-calculi

A general method for proving the normalization theorem for first and second order typed λ-calculi Math. Struct. in Comp. Science (1999), vol. 9, pp. 719 739. c 1999 Cambridge University Press Printed in the United Kingdom A general method for proving the normalization theorem for first and second order

More information

A Fully Labelled Lambda Calculus: Towards Closed Reduction in the Geometry of Interaction Machine

A Fully Labelled Lambda Calculus: Towards Closed Reduction in the Geometry of Interaction Machine Electronic Notes in Theoretical Computer Science 171 (2007) 111 126 www.elsevier.com/locate/entcs A Fully Labelled Lambda Calculus: Towards Closed Reduction in the Geometry of Interaction Machine Nikolaos

More information

Five Basic Concepts of. Axiomatic Rewriting Theory

Five Basic Concepts of. Axiomatic Rewriting Theory Five Basic Concepts of Axiomatic Rewriting Theory Paul-André Melliès Institut de Recherche en Informatique Fondamentale (IRIF) CNRS & Université Paris Denis Diderot 5th International Workshop on Confluence

More information

Sequent Combinators: A Hilbert System for the Lambda Calculus

Sequent Combinators: A Hilbert System for the Lambda Calculus Sequent Combinators: A Hilbert System for the Lambda Calculus Healfdene Goguen Department of Computer Science, University of Edinburgh The King s Buildings, Edinburgh, EH9 3JZ, United Kingdom Fax: (+44)

More information

Consequence Relations and Natural Deduction

Consequence Relations and Natural Deduction Consequence Relations and Natural Deduction Joshua D Guttman Worcester Polytechnic Institute September 16, 2010 Contents 1 Consequence Relations 1 2 A Derivation System for Natural Deduction 3 3 Derivations

More information

Extensional Equivalence and Singleton Types

Extensional Equivalence and Singleton Types Extensional Equivalence and Singleton Types CHRISTOPHER A. STONE Harvey Mudd College and ROBERT HARPER Carnegie Mellon University In this paper we study a λ-calculus enriched with singleton types, where

More information

Coinductive big-step operational semantics

Coinductive big-step operational semantics Coinductive big-step operational semantics Xavier Leroy a, Hervé Grall b a INRIA Paris-Rocquencourt Domaine de Voluceau, B.P. 105, 78153 Le Chesnay, France b École des Mines de Nantes La Chantrerie, 4,

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

Optimizing Optimal Reduction: A Type Inference Algorithm for Elementary Affine Logic

Optimizing Optimal Reduction: A Type Inference Algorithm for Elementary Affine Logic Optimizing Optimal Reduction: A Type Inference Algorithm for Elementary Affine Logic Paolo Coppola Università di Udine Dip. di Matematica e Informatica Simone Martini Università di Bologna Dip. di Scienze

More information