A Rewrite System for Strongly Normalizable Terms

Size: px
Start display at page:

Download "A Rewrite System for Strongly Normalizable Terms"

Transcription

1 A Rewrite System for Strongly Normalizable Terms IRIF Seminar Olivier Hermant & Ronan Saillard CRI, MINES ParisTech, PSL University June 28, 2018 O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

2 Intersection Types (x : F) Γ (Axiom) Γ x : F Γ X : F G Γ Y : F ( E ) Γ X Y : G Γ, x : F X : G ( I ) Γ λx.x : F G Γ X : F G ( E1 ) Γ X : F Γ X : F G ( E2 ) Γ X : G Γ X : F Γ X : G ( I Γ X : F G λx.(x x) : (A (A A)) A if X is typable, it is SN if X is SN, it is typable O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

3 Statman s System [2012] higher-order predicate/new connective D : ι o o o, a discriminator D v F G properties : D 0 F G is F and D 1 F G is G intuition D is an if...then...else... operator v DvFG encodes F G meaning given by rewrite rules D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dt( xf)g x(dtfg) ( 1 ) DtF( xg) x(dtfg) ( 2 ) xf F ($ ) X yf y xf ($$) ( ) no variable is captured (including those of t) ( ) x does not appear in F O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

4 Typing Rules (x : F) Γ (Axiom) Γ x : F Γ X : F F G (Conv) Γ X : G Γ X : F G Γ Y : F ( E ) Γ X Y : G Γ, x : F X : G ( I ) Γ λx.x : F G Γ X : F v : ι v fv(γ) Γ X : v.f ( I ) Γ X : v.f t : ι t free for v in F ( E ) Γ X : F[v/t] Figure Typing Rules of Minimal Natural Deduction with Conversion if X is typable, it is SN if X is SN, it is typable O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

5 Example Give a type to λx.(x x) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

6 Goals 1 down to first-order intuitionistic logic 2 prove with rewrite rules suitable framework : Deduction Modulo Theory if X is typable, it is SN if X is SN, it is typable 3 (further work) the superconsistency conjecture (G. Dowek) : a type system is superconsistent iff it is SN ( ) : proof by Dowek ( ) :? this system is a candidate to disprove the conjecture O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

7 Method a type system with conversion is totally acceptable conversion is now defined otherwise remind Statman s system D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dt( xf)g x(dtfg) ( ) DtF( xg) x(dtfg) ( ) xf F ($ ) X yf y xf ($$) we need to get rid of D at least at the propositional level what can we save from this system in Deduction Modulo Theory? O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

8 term rewrite rule : A A Deduction Modulo Theory Rewrite Rule A term (resp. proposition) rewrite rule is a pair of terms (resp. formulæ) l r, where F V(l) F V(r) and, in the propositiona case, l is atomic. Examples : proposition rewrite rule : A B x x A x B Conversion modulo a Rewrite System We consider the congruence generated by a set of proposition rewrite rules R and a set of term rewrite rules E (often implicit) Example : A A x x A x A O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

9 Typing Rules (x : F) Γ (Axiom) Γ x : F Γ X : F F G (Conv) Γ X : G Γ X : F G Γ Y : F ( E ) Γ X Y : G Γ, x : F X : G ( I ) Γ λx.x : F G Γ X : F v : ι v fv(γ) Γ X : v.f ( I ) Γ X : v.f t : ι t free for v in F ( E ) Γ X : F[v/t] Figure Typing Rules of Minimal Natural Deduction Modulo Theory O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

10 Proof of A A with and without DM without (Γ := z : A A x(x A x A)) : (ax) E2 Γ z : A A x(x A x A) Γ z 2 : x(x A x A) A A Γ (z 2 (λy.y)) : A A. Γ λy.y : x(x A x A) A A with (ax) y : x A y : x A λy.y : x A x A I λy.y : x(x A x A) (Conv) λy.y : A A as if we replaced z1 and z 2 with λα.α (see also Polarized Deduction Modulo Theory) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

11 Statman s System in First-Order Minimal DMT Analysis D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dt( xf)g x(dtfg) ( ) DtF( xg) x(dtfg) ( ) xf F ($ ) X yf y xf ($$) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

12 Statman s System in First-Order Minimal DMT Analysis D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dt( xf)g x(dtfg) ( ) DtF( xg) x(dtfg) ( ) xf F ($ ) X yf y xf ($$) get rid of D reflect it as a term (techniques to embed HOL) introduce the following terms :,, D, 0, 1 and a unique unary predicate ε O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

13 Statman s System in First-Order Minimal DMT Analysis D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dt( xf)g x(dtfg) ( ) DtF( xg) x(dtfg) ( ) xf F ($ ) X yf y xf ($$) get rid of D reflect it as a term (techniques to embed HOL) introduce the following terms :,, D, 0, 1 and a unique unary predicate ε combine terms properly (e.g. forbid ) simple types, with ι (0 and 1) and o (propositional terms) 0, 1 : ι D : ι o o o : (ι o) o : o o o add one propositional symbol ṗ : o propositional rewriting : ε(a B) ε(a) ε(b) ε( A) x.ε(a x) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

14 Statman s System in First-Order Minimalist Deduction Modulo Theory Statman s System : D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dt( xf)g x(dtfg) ( ) DtF( xg) x(dtfg) ( ) xf F ($ ) X yf y xf ($$) we can readily define three rewrite rules : D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) still to be defined Dt( F)G? ( 1 ) DtF( G)? ( 2 ) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

15 How to Abstract Need an equivalent of Dt( xf)g x(dtfg) at term level Dv( F)G no free variable x hence no freshness constraint (good) nevertheless need to define something like for some fresh x Dv( F)G (λx.(dv(fx)g)) two solutions exist in Deduction modulo theory 1 allow λ-abstraction in the simply-typed term language 2 replace this by a combinatorial calculus choice : Solution 1 cumbersome : explicit substitutions interfere with D Solution 2 cumbersome too could we have dropped explicit substitutions? O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

16 Combinatorial Calculus SKI we introduce and application symbols : I : ι ι K : τ ι τ S : (ι τ α) (ι τ) ι α denote in those slides as white space usual reduction rules I x x (I) K x y x (K) S x y z x z (y z) (S) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

17 Combinatorial Calculus SKI defining abstraction it is possible (see textbooks) we only need Dv( F)G (λx.(dv(fx)g)) with x fresh. so, define λx.(dv(fx)g) as S (K DvF) (S (KG) I) similarly for DvF( G) (λx.(dvf(gx))) note : no new (rewriting) redex is created some redex might be destroyed (take 0 or 1 for v) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

18 The Final Rewriting System encoding the logic : ε(a B) ε(a) ε(b) (ε ) I x x (I) ε( A) x.ε(a x) (ε ) K x y x (K) S x y z x z (yz) (S) encoding Statman s rules : D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dv( F)G (λx.(dv(fx)g)) ( 1 ) DvF( G) (λx.(dvf(gx))) ( 2 ) no way to encode ($) - pruning unnecessary quantifiers, ($$) - permuting quantifiers nonterminating rules but we need confluence! 7 critical pairs : Dv( F)( G) (needs ($$)) D0( F)G (reducing by 1 freezes the (0)) impossible for terms, weak confluence at the ε-level (sweat) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

19 Termination First encoding the logic : ε(a B) ε(a) ε(b) (ε ) I x x (I) ε( A) x.ε(a x) (ε ) K x y x (K) S x y z x z (yz) (S) encoding Statman s rules : D0FG F (0) D1FG G (1) Dt(F G)(H K) (DtFH) (DtGK) ( ) Dv( F)G (λx.(dv(fx)g)) ( 1 ) DvF( G) (λx.(dvf(gx))) ( 2 ) termination 1 ε reduces the number of, 2 typed-restricted S and K imply no duplication of and 3 goes up in terms 4 goes up and decreases 5 simply-typed SKI terminates automatically prove termination? O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

20 Confluence impossible at the term level D0( F)G (λx.(d0(f x)g) F fixed at the proposition level ε(d0( F)G) ε( (λx.(d0(f x)g)) ε( F) x.ε(f x) still problematic for D0F( G) : and Dv( F)( G) : yε(f) ε(f) x yε(dv(fx)(gy)) y xε(dv(fx)(gy)) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

21 Confluence up to equivalence but we can have confluence up to : variable renaming, pruning and inversion of quantifiers does not fit in a term equational theory E Definition A B : if A and B normal, and either A = x.ε(ta ), B = y.ε(t B ) and ε(t A ) ε(t B ) or A = x.(a1 A 2 ), B = y.(b 1 B 2 ) and A 1 B 1 and A 2 B 2. Lemma B A A0 B0 (in NF) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

22 Proof of the Lemma : Strategy B A (prove) B A (IH) C0 B 0 (NF) A 0 get rid of no rewrite step from B to A or to B0 prove the existence of C0 induction on : the height of the reduction tree of B, noted B easy if A B B does not involve a critical pair let us see the F D0( F)G λx.(d0(f x)g) case O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

23 we have B = K[D0( F)G] One Critical Pair A = K[ F] B = K[ λx.(d0(f x)g)] B 0 (NF) long time to wait before joining at the ε level introduce the inductive invariant t 1 t 2 if there exist a context K and two terms θ 1, θ 2 such that : A t 1 = K[ θ 1 ], B t 2 = K[ θ 2 ] B 0, P(θ 1, θ 2 ) where P(u 1, u 2 ) is : u 2 x u 1 x and if u 2 u 2 then for some u 1 u 1, P(u, 1 u ) 2 P( F, λx.(d0(f x)g)) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

24 Critical Pair : Interesting Subcases t 1 t 2 if there exist a context K and two terms θ 1, θ 2 such that : A t 1 = K[ θ 1 ], B t 2 = K[ θ 2 ] B 0, P(θ1, θ 2 ) where P(u 1, u 2 ) is : u 2 x u 1 x and if u 2 u 2 then for some u 1 u 1, P(u, 1 u ) 2 proof the existence of C0 by induction on t 2 B 0 t2 = L[ε( θ 2 )] L[ x.ε(θ 2 x)] Confluence case. Saved! (big IH as t 2 < B ) t2 = L[Dv( θ 2 )Z] L[ λ x (Dv(θ 2 x)z)] IH, since P(λx.(Dv(θ 1 x)z), λx.(dv(θ 2 x)z)) t2 = K[ θ 2 ] K [ θ 2 ] : fits t2 = K[ θ 2 ] K[ θ 2 ] : fits O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

25 Digging Terms confluence up to at the proposition level! with intersection types, merging derivations : Γ X : F Γ X : G ( I ) Γ X : F G derivation transformations in Statman s system Derivation Merge (Statman) If Γ 1 X : F and Γ 2 X : G then DvΓ 1 Γ 2 X : DvFG we must prove the result perform this on terms (D is a term) Proposition Reification γ(ε(t)) := t γ(f G) := γ(f) γ(g) γ( x.f) := (λx.(γ(f))) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

26 Reification Proposition Reification γ(f) noted Ḟ. γ(ε(t)) := t γ(f G) := γ(f) γ(g) γ( x.f) := (λx.(γ(f))) ε(γ(f)) F we need (for conversions) if F F, G G then DvḞĠ DvḞ Ġ problem : not preserved by γ! Counter-example : F = x.ε(d0ab) and F = x.ε(a) Ḟ is not convertible with F When F contains quantifiers : redexes frozen by λ O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

27 Reification Proposition Reification γ(f) noted Ḟ. We actually need Merges are Convertible γ(ε(t)) := t γ(f G) := γ(f) γ(g) γ( x.f) := (λx.(γ(f))) if F F, G G then ε(dvḟġ) ε(dvḟ Ġ ) Works separately for F1 G 1 and F 2 G 2, but not for deeper combinations : ε(dv(ḟ 1 Ḟ 2 )ṗ) not convertible with ε(dv(ġ1 Ġ2)ṗ) ṗ is not implicational : ε cannot expose the structure O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

28 Digging Proposition Reification γ(f) noted Ḟ. γ(ε(t)) := t γ(f G) := γ(f) γ(g) γ( x.f) := (λx.(γ(f))) ε(dv(ḟ1 Ḟ 2 )ṗ) not convertible with ε(dv(ġ1 Ġ2)ṗ) idea : dig out the implicational structure replace all ṗ with ṗ ṗ potentially, n times notation t{n} Merge Conversion If F 1 F 2 and G 1 G 2 then, for some n, ε(dvf 1 {n} G 1 {n}) ε(dvf 2 {n} G 2 {n}). O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

29 All SN terms are Typable finally able to follow Statman s line derivations are organized in segments Γ X : F ( I ),(Conv),( E ) Γ X : G that we can organize as Γ X : F ( E ) Γ X : G (Conv) Γ X : G ( I ) Γ X : H we can merge two segments : Γ 1 X : F Γ 2 X : G (seg) Γ 1 X : F Γ 2 X : G with some digging into Γ X : ε(dvḟ{n}ġ{n}) (seg) we can also merge two derivations of the same term X O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

30 All SN terms are Typable, and conversely SN typable : 1 follow more or less Statman s way (with more explanations) 2 All terms in NF are typable 3 if a reduct of a head β-redex is typable, so is the redex 4 if X is SN, it is typable typable SN find the worse reduction strategy, F (M) (Barendregt) prove that it terminates or use Reducibility Candidates? (cf. plain intersection types) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

31 Conclusion we have intersection types in Deduction Modulo Theory no new connectives, etc rewrite rules instead interesting confluence property regain nice properties and some extensionality : lot of plumbing further work do we have a model with values on the reducibility candidates? one technical detail to fix (variable renaming) O. Hermant (MINES ParisTech) Intersection Types in DMT June 28, / 29

From pre-models to models

From pre-models to models From pre-models to models normalization by Heyting algebras Olivier HERMANT 18 Mars 2008 Deduction System : natural deduction (NJ) first-order logic: function and predicate symbols, logical connectors:,,,,

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

A General Type for Storage Operators

A General Type for Storage Operators A General Type for Storage Operators Karim NOUR LAMA - Equipe de Logique, Université de Chambéry 73376 Le Bourget du Lac e-mail nour@univ-savoie.fr Abstract In 1990, J.L. Krivine introduced the notion

More information

Typage et déduction dans le calcul de

Typage et déduction dans le calcul de Typage et déduction dans le calcul de réécriture Benjamin Wack Encadrants : C. Kirchner, L. Liquori Deduction and computation λ-calculus [Church 40] is a simple and powerful computational model Explicit

More information

A simple proof that super-consistency implies cut elimination

A simple proof that super-consistency implies cut elimination A simple proof that super-consistency implies cut elimination Gilles Dowek 1 and Olivier Hermant 2 1 École polytechnique and INRIA, LIX, École polytechnique, 91128 Palaiseau Cedex, France gilles.dowek@polytechnique.edu

More information

Truth values algebras and proof normalization

Truth values algebras and proof normalization Truth values algebras and proof normalization Gilles Dowek École polytechnique and INRIA, LIX, École polytechnique, 91128 Palaiseau Cedex, France http://lix.polytechnique.fr/ dowek/ Gilles.Dowek@polytechnique.edu

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

Clausal Presentation of Theories in Deduction Modulo

Clausal Presentation of Theories in Deduction Modulo Gao JH. Clausal presentation of theories in deduction modulo. JOURNAL OF COMPUTER SCIENCE AND TECHNOL- OGY 28(6): 1085 1096 Nov. 2013. DOI 10.1007/s11390-013-1399-0 Clausal Presentation of Theories in

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

PROOF NORMALIZATION MODULO

PROOF NORMALIZATION MODULO PROOF NORMALIZATION MODULO GILLES DOWEK AND BENJAMIN WERNER Abstract. We define a generic notion of cut that applies to many first-order theories. We prove a generic cut elimination theorem showing that

More information

A Formalised Proof of Craig s Interpolation Theorem in Nominal Isabelle

A Formalised Proof of Craig s Interpolation Theorem in Nominal Isabelle A Formalised Proof of Craig s Interpolation Theorem in Nominal Isabelle Overview We intend to: give a reminder of Craig s theorem, and the salient points of the proof introduce the proof assistant Isabelle,

More information

Orthogonality and Boolean Algebras for Deduction Modulo

Orthogonality and Boolean Algebras for Deduction Modulo Orthogonality and Boolean Algebras for Deduction Modulo Aloïs Brunel 1, Olivier Hermant 2, and Clément Houtmann 3 1 ENS de Lyon, Alois.Brunel@ens-lyon.org 2 ISEP, Olivier.Hermant@isep.fr 3 INRIA Saclay,

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

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

Intersection Synchronous Logic

Intersection Synchronous Logic UnB 2007 p. 1/2 Intersection Synchronous Logic Elaine Gouvêa Pimentel Simona Ronchi della Rocca Luca Roversi UFMG/UNITO, 2007 UnB 2007 p. 2/2 Outline Motivation UnB 2007 p. 2/2 Outline Motivation Intuitionistic

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

Kleene realizability and negative translations

Kleene realizability and negative translations Q E I U G I C Kleene realizability and negative translations Alexandre Miquel O P. D E. L Ō A U D E L A R April 21th, IMERL Plan 1 Kleene realizability 2 Gödel-Gentzen negative translation 3 Lafont-Reus-Streicher

More information

Γ is usually left implicit: ϕ

Γ is usually left implicit: ϕ Types Summer School Gothenburg Sweden August 2005 Type Systems Herman Geuvers Radboud University Nijmegen, NL Lecture 2: Higher Order Logic and Type Theory The original motivation of Church to introduce

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

The Suspension Notation as a Calculus of Explicit Substitutions

The Suspension Notation as a Calculus of Explicit Substitutions The Suspension Notation as a Calculus of Explicit Substitutions Gopalan Nadathur Digital Technology Center and Department of Computer Science University of Minnesota [Joint work with D.S. Wilson and A.

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

Non-Idempotent Typing Operators, beyond the λ-calculus

Non-Idempotent Typing Operators, beyond the λ-calculus Non-Idempotent Typing Operators, beyond the λ-calculus Soutenance de thèse Pierre VIAL IRIF (Univ. Paris Diderot and CNRS) December 7, 2017 Non-idempotent typing operators P. Vial 0 1 /46 Certification

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

First-Order Logic First-Order Theories. Roopsha Samanta. Partly based on slides by Aaron Bradley and Isil Dillig

First-Order Logic First-Order Theories. Roopsha Samanta. Partly based on slides by Aaron Bradley and Isil Dillig First-Order Logic First-Order Theories Roopsha Samanta Partly based on slides by Aaron Bradley and Isil Dillig Roadmap Review: propositional logic Syntax and semantics of first-order logic (FOL) Semantic

More information

The faithfulness of atomic polymorphism

The faithfulness of atomic polymorphism F Ferreira G Ferreira The faithfulness of atomic polymorphism Abstract It is known that the full intuitionistic propositional calculus can be embedded into the atomic polymorphic system F at, a calculus

More information

First Order Logic vs Propositional Logic CS477 Formal Software Dev Methods

First Order Logic vs Propositional Logic CS477 Formal Software Dev Methods First Order Logic vs Propositional Logic CS477 Formal Software Dev Methods Elsa L Gunter 2112 SC, UIUC egunter@illinois.edu http://courses.engr.illinois.edu/cs477 Slides based in part on previous lectures

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

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

Introduction to dependent type theory. CIRM, May 30

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

More information

Structuring Logic with Sequent Calculus

Structuring Logic with Sequent Calculus Structuring Logic with Sequent Calculus Alexis Saurin ENS Paris & École Polytechnique & CMI Seminar at IIT Delhi 17th September 2004 Outline of the talk Proofs via Natural Deduction LK Sequent Calculus

More information

Notation for Logical Operators:

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

More information

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

3.17 Semantic Tableaux for First-Order Logic

3.17 Semantic Tableaux for First-Order Logic 3.17 Semantic Tableaux for First-Order Logic There are two ways to extend the tableau calculus to quantified formulas: using ground instantiation using free variables Tableaux with Ground Instantiation

More information

Discrete Mathematics. Instructor: Sourav Chakraborty. Lecture 4: Propositional Logic and Predicate Lo

Discrete Mathematics. Instructor: Sourav Chakraborty. Lecture 4: Propositional Logic and Predicate Lo gic Instructor: Sourav Chakraborty Propositional logic and Predicate Logic Propositional logic and Predicate Logic Every statement (or proposition) is either TRUE or FALSE. Propositional logic and Predicate

More information

Non- -overlappings TRSs are UN. Stefan Kahrs and Connor Smith University of Kent

Non- -overlappings TRSs are UN. Stefan Kahrs and Connor Smith University of Kent Non- -overlappings TRSs are UN Stefan Kahrs and Connor Smith University of Kent This is about: When is the equational theory of a TRS consistent (CON), when does it have unique normal forms (UN), How can

More information

Chapter 11: Automated Proof Systems

Chapter 11: Automated Proof Systems Chapter 11: Automated Proof Systems SYSTEM RS OVERVIEW Hilbert style systems are easy to define and admit a simple proof of the Completeness Theorem but they are difficult to use. Automated systems are

More information

Realizing the axiom of dependent choice

Realizing the axiom of dependent choice Realizing the axiom of dependent choice Jean-Louis Krivine PPS Group, University Paris 7, CNRS krivine@pps.jussieu.fr Edinburgh, March 26, 2003 1 The extended Curry-Howard correspondence We want to get

More information

Propositional Logic Language

Propositional Logic Language Propositional Logic Language A logic consists of: an alphabet A, a language L, i.e., a set of formulas, and a binary relation = between a set of formulas and a formula. An alphabet A consists of a finite

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

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

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

More information

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

Chapter 3. Formal Number Theory

Chapter 3. Formal Number Theory Chapter 3. Formal Number Theory 1. An Axiom System for Peano Arithmetic (S) The language L A of Peano arithmetic has a constant 0, a unary function symbol, a binary function symbol +, binary function symbol,

More information

Propositional Logic: Syntax

Propositional Logic: Syntax Logic Logic is a tool for formalizing reasoning. There are lots of different logics: probabilistic logic: for reasoning about probability temporal logic: for reasoning about time (and programs) epistemic

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

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

URL: 13 pages Eigenvariables, bracketing and the decidability of positive minimal intuitionistic log

URL:   13 pages Eigenvariables, bracketing and the decidability of positive minimal intuitionistic log URL: http://www.elsevier.nl/locate/entcs/volume85.html 13 pages Eigenvariables, bracketing and the decidability of positive minimal intuitionistic logic Gilles Dowek 1 École polytechnique and INRIA, LIX,

More information

Quandles and the Towers of Hanoi

Quandles and the Towers of Hanoi The the Bob Laboratory for Algebraic and Symbolic Computation Reem-Kayden Center for Science and Computation Bard College Annandale-on-Hudson, NY 12504 August 8, 2011 The 1 2 3 4 The The Figure Eight (4

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

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

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

More information

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

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

Provably Total Functions of Arithmetic with Basic Terms

Provably Total Functions of Arithmetic with Basic Terms Provably Total Functions of Arithmetic with Basic Terms Evgeny Makarov INRIA Orsay, France emakarov@gmail.com A new characterization of provably recursive functions of first-order arithmetic is described.

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

A Cut-Free Calculus for Second-Order Gödel Logic

A Cut-Free Calculus for Second-Order Gödel Logic Fuzzy Sets and Systems 00 (2014) 1 30 Fuzzy Sets and Systems A Cut-Free Calculus for Second-Order Gödel Logic Ori Lahav, Arnon Avron School of Computer Science, Tel Aviv University Abstract We prove that

More information

model called a pre-model. For instance, simple type theory can be expressed in deduction modulo [5, 6] and it has a pre-model [7, 6] and hence it has

model called a pre-model. For instance, simple type theory can be expressed in deduction modulo [5, 6] and it has a pre-model [7, 6] and hence it has The Stratied Foundations as a theory modulo Gilles Dowek Abstract The Stratied Foundations are a restriction of naive set theory where the comprehension scheme is restricted to stratiable propositions.

More information

Non deterministic classical logic: the λµ ++ -calculus

Non deterministic classical logic: the λµ ++ -calculus Paru dans : Mathematical Logic Quarterly, 48, pp. 357-366, 2002 Non deterministic classical logic: the λµ ++ -calculus Karim NOUR LAMA - Equipe de Logique, Université de Savoie 73376 Le Bourget du Lac

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

A call-by-name lambda-calculus machine

A call-by-name lambda-calculus machine A call-by-name lambda-calculus machine Jean-Louis Krivine University Paris VII, C.N.R.S. 2 place Jussieu 75251 Paris cedex 05 (krivine@pps.jussieu.fr) Introduction We present, in this paper, a particularly

More information

The Vectorial Lambda-Calculus

The Vectorial Lambda-Calculus The Vectorial Lambda-Calculus Pablo Arrighi a,b, Alejandro Díaz-Caro c,e, Benoît Valiron d,e a ENS-Lyon, Laboratoire LIP, France b Université de Grenoble, Laboratoire LIG, France c Université Paris-Ouest

More information

First-Order Predicate Logic. Basics

First-Order Predicate Logic. Basics First-Order Predicate Logic Basics 1 Syntax of predicate logic: terms A variable is a symbol of the form x i where i = 1, 2, 3.... A function symbol is of the form fi k where i = 1, 2, 3... und k = 0,

More information

Applied Logic for Computer Scientists. Answers to Some Exercises

Applied Logic for Computer Scientists. Answers to Some Exercises Applied Logic for Computer Scientists Computational Deduction and Formal Proofs Springer, 2017 doi: http://link.springer.com/book/10.1007%2f978-3-319-51653-0 Answers to Some Exercises Mauricio Ayala-Rincón

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

Mathematical Logic. Helmut Schwichtenberg

Mathematical Logic. Helmut Schwichtenberg Mathematical Logic Helmut Schwichtenberg Mathematisches Institut der Universität München Wintersemester 2009/2010 Contents Chapter 1. Logic 1 1.1. Natural Deduction 1 1.2. Normalization 15 1.3. Soundness

More information

Herbrand Theorem, Equality, and Compactness

Herbrand Theorem, Equality, and Compactness CSC 438F/2404F Notes (S. Cook and T. Pitassi) Fall, 2014 Herbrand Theorem, Equality, and Compactness The Herbrand Theorem We now consider a complete method for proving the unsatisfiability of sets of first-order

More information

Between proof theory and model theory Three traditions in logic: Syntactic (formal deduction)

Between proof theory and model theory Three traditions in logic: Syntactic (formal deduction) Overview Between proof theory and model theory Three traditions in logic: Syntactic (formal deduction) Jeremy Avigad Department of Philosophy Carnegie Mellon University avigad@cmu.edu http://andrew.cmu.edu/

More information

MATH 1090 Problem Set #3 Solutions March York University

MATH 1090 Problem Set #3 Solutions March York University York University Faculties of Science and Engineering, Arts, Atkinson MATH 1090. Problem Set #3 Solutions Section M 1. Use Resolution (possibly in combination with the Deduction Theorem, Implication as

More information

Command = Value Context. Hans-Dieter Hiep. 15th of June, /17

Command = Value Context. Hans-Dieter Hiep. 15th of June, /17 1/17 Command = Value Context Hans-Dieter Hiep 15th of June, 2018 2/17 Example Consider a total functional programming language. swap :: A B B A swap (a, b) = (b, a) paws :: A B B A paws a = a paws b =

More information

Jacques Fleuriot. Automated Reasoning Rewrite Rules

Jacques Fleuriot. Automated Reasoning Rewrite Rules Automated Reasoning Rewrite Rules Jacques Fleuriot Lecture 8, page 1 Term Rewriting Rewriting is a technique for replacing terms in an expression with equivalent terms useful for simplification, e.g. given

More information

Chapter 11: Automated Proof Systems (1)

Chapter 11: Automated Proof Systems (1) Chapter 11: Automated Proof Systems (1) SYSTEM RS OVERVIEW Hilbert style systems are easy to define and admit a simple proof of the Completeness Theorem but they are difficult to use. Automated systems

More information

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

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

More information

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

Intelligent Agents. First Order Logic. Ute Schmid. Cognitive Systems, Applied Computer Science, Bamberg University. last change: 19.

Intelligent Agents. First Order Logic. Ute Schmid. Cognitive Systems, Applied Computer Science, Bamberg University. last change: 19. Intelligent Agents First Order Logic Ute Schmid Cognitive Systems, Applied Computer Science, Bamberg University last change: 19. Mai 2015 U. Schmid (CogSys) Intelligent Agents last change: 19. Mai 2015

More information

185.A09 Advanced Mathematical Logic

185.A09 Advanced Mathematical Logic 185.A09 Advanced Mathematical Logic www.volny.cz/behounek/logic/teaching/mathlog13 Libor Běhounek, behounek@cs.cas.cz Lecture #1, October 15, 2013 Organizational matters Study materials will be posted

More information

Some Applications of MATH 1090 Techniques

Some Applications of MATH 1090 Techniques 1 Some Applications of MATH 1090 Techniques 0.1 A simple problem about Nand gates in relation to And gates and inversion (Not) Gates. In this subsection the notation A means that A is proved from the axioms

More information

From Operational Semantics to Abstract Machines

From Operational Semantics to Abstract Machines From Operational Semantics to Abstract Machines John Hannan Department of Computer Science, University of Copenhagen, Universitetsparken 1, DK-2100 Copenhagen East, Denmark. hannan@diku.dk Dale Miller

More information

Equational Theory of Kleene Algebra

Equational Theory of Kleene Algebra Introduction to Kleene Algebra Lecture 7 CS786 Spring 2004 February 16, 2004 Equational Theory of Kleene Algebra We now turn to the equational theory of Kleene algebra. This and the next lecture will be

More information

Discrete Mathematics

Discrete Mathematics Slides for Part IA CST 2015/16 Discrete Mathematics Prof Marcelo Fiore Marcelo.Fiore@cl.cam.ac.uk What are we up to? Learn to read and write, and also work with,

More information

PREDICATE LOGIC: UNDECIDABILITY AND INCOMPLETENESS HUTH AND RYAN 2.5, SUPPLEMENTARY NOTES 2

PREDICATE LOGIC: UNDECIDABILITY AND INCOMPLETENESS HUTH AND RYAN 2.5, SUPPLEMENTARY NOTES 2 PREDICATE LOGIC: UNDECIDABILITY AND INCOMPLETENESS HUTH AND RYAN 2.5, SUPPLEMENTARY NOTES 2 Neil D. Jones DIKU 2005 14 September, 2005 Some slides today new, some based on logic 2004 (Nils Andersen) OUTLINE,

More information

COMP 409: Logic Homework 5

COMP 409: Logic Homework 5 COMP 409: Logic Homework 5 Note: The pages below refer to the text from the book by Enderton. 1. Exercises 1-6 on p. 78. 1. Translate into this language the English sentences listed below. If the English

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

CS156: The Calculus of Computation

CS156: The Calculus of Computation Page 1 of 31 CS156: The Calculus of Computation Zohar Manna Winter 2010 Chapter 3: First-Order Theories Page 2 of 31 First-Order Theories I First-order theory T consists of Signature Σ T - set of constant,

More information

The Permutative λ-calculus

The Permutative λ-calculus The Permutative λ-calculus Beniamino Accattoli 1 Delia Kesner 2 INRIA and LIX (École Polytechnique) PPS (CNRS and Université Paris-Diderot) 1 / 34 Outline 1 λ-calculus 2 Permutative extension 3 Confluence

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

HORSes: format, termination and confluence

HORSes: format, termination and confluence HORSes: format, termination and confluence Jean-Pierre Jouannaud INRIA-LIAMA and singhua Software Chair Joint on-going work with Jianqi Li School of Software, singhua University Project CoqLF NList Cross-discipline

More information

UNITARY UNIFICATION OF S5 MODAL LOGIC AND ITS EXTENSIONS

UNITARY UNIFICATION OF S5 MODAL LOGIC AND ITS EXTENSIONS Bulletin of the Section of Logic Volume 32:1/2 (2003), pp. 19 26 Wojciech Dzik UNITARY UNIFICATION OF S5 MODAL LOGIC AND ITS EXTENSIONS Abstract It is shown that all extensions of S5 modal logic, both

More information

Normal Forms for First-Order Logic

Normal Forms for First-Order Logic Logic and Proof Hilary 2016 James Worrell Normal Forms for First-Order Logic In this lecture we show how to transform an arbitrary formula of first-order logic to an equisatisfiable formula in Skolem form.

More information

CHAPTER 10. Gentzen Style Proof Systems for Classical Logic

CHAPTER 10. Gentzen Style Proof Systems for Classical Logic CHAPTER 10 Gentzen Style Proof Systems for Classical Logic Hilbert style systems are easy to define and admit a simple proof of the Completeness Theorem but they are difficult to use. By humans, not mentioning

More information

Axioms of Kleene Algebra

Axioms of Kleene Algebra Introduction to Kleene Algebra Lecture 2 CS786 Spring 2004 January 28, 2004 Axioms of Kleene Algebra In this lecture we give the formal definition of a Kleene algebra and derive some basic consequences.

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

GÖDEL S COMPLETENESS AND INCOMPLETENESS THEOREMS. Contents 1. Introduction Gödel s Completeness Theorem

GÖDEL S COMPLETENESS AND INCOMPLETENESS THEOREMS. Contents 1. Introduction Gödel s Completeness Theorem GÖDEL S COMPLETENESS AND INCOMPLETENESS THEOREMS BEN CHAIKEN Abstract. This paper will discuss the completeness and incompleteness theorems of Kurt Gödel. These theorems have a profound impact on the philosophical

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

Conservativity of Embeddings in the λπ Calculus Modulo Rewriting

Conservativity of Embeddings in the λπ Calculus Modulo Rewriting Conservativity of Embeddings in the λπ Calculus Modulo Rewriting Ali Assaf 1,2 1 Inria, Paris, France 2 École polytechnique, Palaiseau, France Abstract The λπ calculus can be extended with rewrite rules

More information

CSC 7101: Programming Language Structures 1. Axiomatic Semantics. Stansifer Ch 2.4, Ch. 9 Winskel Ch.6 Slonneger and Kurtz Ch. 11.

CSC 7101: Programming Language Structures 1. Axiomatic Semantics. Stansifer Ch 2.4, Ch. 9 Winskel Ch.6 Slonneger and Kurtz Ch. 11. Axiomatic Semantics Stansifer Ch 2.4, Ch. 9 Winskel Ch.6 Slonneger and Kurtz Ch. 11 1 Overview We ll develop proof rules, such as: { I b } S { I } { I } while b do S end { I b } That allow us to verify

More information

Logic: The Big Picture

Logic: The Big Picture Logic: The Big Picture A typical logic is described in terms of syntax: what are the legitimate formulas semantics: under what circumstances is a formula true proof theory/ axiomatization: rules for proving

More information

Meta-Reasoning in a Concurrent Logical Framework

Meta-Reasoning in a Concurrent Logical Framework Meta-Reasoning in a Concurrent Logical Framework Iliano Cervesato and Jorge Luis Sacchini Carnegie Mellon University Chalmers University, 16 Oct 2013 Iliano Cervesato and Jorge Luis Sacchini Meta-Reasoning

More information

Automated Synthesis of Tableau Calculi

Automated Synthesis of Tableau Calculi Automated Synthesis of Tableau Calculi Renate A. Schmidt 1 and Dmitry Tishkovsky 1 School of Computer Science, The University of Manchester Abstract This paper presents a method for synthesising sound

More information

arxiv:math/ v1 [math.lo] 27 Jan 2003

arxiv:math/ v1 [math.lo] 27 Jan 2003 Locality for Classical Logic arxiv:math/0301317v1 [mathlo] 27 Jan 2003 Kai Brünnler Technische Universität Dresden Fakultät Informatik - 01062 Dresden - Germany kaibruennler@inftu-dresdende Abstract In

More information

Homotopy Type Theory

Homotopy Type Theory Homotopy Type Theory Jeremy Avigad Department of Philosophy and Department of Mathematical Sciences Carnegie Mellon University February 2016 Homotopy Type Theory HoTT relies on a novel homotopy-theoretic

More information

Truth values algebras and proof normalization

Truth values algebras and proof normalization Truth values algebras and proof normalization Gilles Dowek École polytechnique and INRIA, LIX, École polytechnique, 91128 Palaiseau Cedex, France http://lix.polytechnique.fr/ dowek/ Gilles.Dowek@polytechnique.edu

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