Scuola Estiva di Logica Gargnano, August

Size: px
Start display at page:

Download "Scuola Estiva di Logica Gargnano, August"

Transcription

1 Linear Logic, Linear Logic, Università degli Studi di Torino Scuola Estiva di Logica 2015 Gargnano, August

2 Complexity theory Linear Logic, study of complexity classes and their relations define first a computational model and its associated cost model (for time, space,...). The standard choice: Turing machines measure of time: number of elementary steps measure of space: dimension of the tape the TM M works in bound f iff for any input u, M<u>terminates using less than f ( u ) resources example: PTIME (FPTIME) is the set of decision problems (functions) that can be solved (computed) in polynomial bound

3 Problems Linear Logic, the design of a program and the proof of its complexity are made in two different steps it is difficult to supply formal proofs of complexity, since the difficulty of dealing formally with TMs

4 Implicit Computational Complexity (ICC) Linear Logic, describes complexity classes without explicit reference to a machine model and its cost bound uses techniques and results from Mathematical : proof theory recursion theory model theory two aims: to implicitly characterize complexity classes to supply programming languages with a certified complexity bound

5 A case study Linear Logic, the idea: start from a given programming language L supply a type discipline for L in such a way that: if a term (program) is well typed then its complexity belongs to a given complexity class C all and only the functions belonging to C are computed by well typed terms the realization: language: λ-calculus (with some extension) types: inspired from Soft Linear Logic (one of the light versions of LL) The results characterizations of PTIME, FPTIME, PSPACE and NP

6 λ-calculus: the paradigm for functional programming languages syntax: M ::= x λx.m MM where x ranges over a countable set of variables. λxy.m stands for λx.(λy.m)) λx 1...x n.m stands forλx 1.(λx 2.(...(λx n.m)...)) M 1 M 2...M n stands for M 1 (M 2 (...M n )). Linear Logic, operational semantics: the β-reduction is the contextual closure of the rule: (λx.m)n M[N/x] β where M[N/x] denotes the (capture free) replacement of all occurrences of x in M by N.

7 Computing with λ-calculus Linear Logic, coding of natural numbers: n=λxy. x(...(x y)) } {{ } n coding of binary words: < i 1...i n >=λx 0 x 1 y.x i1 (x i2 (...(x in y)) where i j ranges over{0, 1}. Theorem In the λ-calculus, all and only the computable functions can be coded.

8 Linear Logic: a resource sensitive logic Linear Logic, Two kinds of formulae: A (linear resource, can be used once)!a (can be used as many times we want, also 0) The intuitionistic implication A B is decomposed in!a B ( is the linear implication) Equivalence!!A =!A

9 The rules of Intuitionistic Linear Logic (ILL) Linear Logic, A A (Id) Γ A, A B Γ, B (cut) Γ, A B Γ A B ( R) Γ A B, C A B,Γ, C ( L) Γ A α FV(Γ) Γ α.a ( R) Γ, B[C/α] A Γ, α.b A ( L) n times { }} { Γ, A,..., A C Γ,!A C (mpx) Γ A!Γ!A (sp) Γ,!!B A Γ,!B A (digging) whereγis a multiset of formulae, andγ, denotes multiset union.

10 Soft Linear Logic (SLL) A A (Id) Γ A, A B Γ, B (cut) Linear Logic, Γ, A B Γ A B ( R) Γ A B, C A B,Γ, C ( L) Γ A α FV(Γ) Γ α.a ( R) Γ, B[C/α] A Γ, α.b A ( L) n times { }} { Γ, A,..., A C Γ,!A C (mpx) Γ A!Γ!A (sp) all rules of ILL but Γ,!!B A Γ,!B A (digging)

11 Properties of SLL Linear Logic, The fact that the equation:!a=!!a allows to use the modality! for counting the number of duplications of proofs during the cut-elimination procedure. In SLL all the polynomial computations can be coded.

12 Linear Logic, STA is a natural deduction style type assignment system inspired by SLL, but: Terms are built in a linear way, and (mpx) rule is used for controlling variable duplication Technically this is realized by using as types a subset of the SLL formulae such that: is not allowed on modal formulae! is not allowed on the right of weakening and axiom introduce not modal formulae. are the following subset of SLL formulae: A ::= α σ A α.a (linear types) σ ::= A!σ

13 Rules of STA Linear Logic, x : A x : A (Ax) Γ M :σ Γ, x : A M :σ (w) Γ, x :σ M : A Γ λx.m :σ A ( I) Γ M :σ A N :σ Γ# Γ, MN : A ( E) Γ, x 1 :σ,..., x n :σ M :τ Γ, x :!σ M[x/x 1,..., x/x n ] :τ (mpx) Γ M :σ!γ M :!σ (sp) Γ A α FV(Γ) Γ M : α.a ( I) Γ M : α.a Γ M : A[B/α] ( E) where Γ# denotes that the two contexts have disjoint variables.

14 Properties of STA Linear Logic, subject reduction Γ M :σand M β M implyγ M :σ. strong normalization Γ M :σimplies M is strongly normalizing.

15 Example Let A= D D, C=A A A B. y : C y : A A A B (Ax) x 1 : A x 1 : A (Ax) ( E) y : C, x 1 : A yx 1 : A A B x 2 : A x 2 : A (Ax) ( E) y : C, x 1 : A, x 2 : A yx 1 x 2 : A B x 3 : A x 3 : A Π 3 y : C, x 1 : A, x 2 : A, x 3 : A yx 1 x 2 x 3 : B (mpx) Π y : C, x :!A yxxx : B (Ax) ( E) Linear Logic, the rank ofπ 3 counts the number of copies of an argument replacing x. Π ( I) y : C λx.yxxx :!A B y : C (λx.yxxx)i : B z : D z: D (Ax) ( I) Φ Id : A (sp) I :!A ( E) Π 3 [(Ax)/Φ] y : C yiii : B whereπ 3 [(Ax)/Φ] denotesπ 3, where all axiom with subject x has been replaced byφ. the rule (sp) is a witness that I will be copied (a number of times corresponding to the rank ofπ 3 ).

16 measures Linear Logic, Π 3 y : C, x 1 : A, x 2 : A, x 3 : A yx 1 x 2 x 3 : B y : C, x :!A, x 3 : A yxxx 3 : B Π y : C, x :!!A yxxx : B (mpx) (mpx) Π y : C, x :!!A yxxx : B ( I) y : C λx.yxxx :!!A B Ψ y : C (λx.yxxx)i : B Φ I : A I :!A (sp) I :!!A (sp) ( E) Π 3 [(Ax)/Φ] y : C yiii : B the rank ofψis the maximum between the ranks of the (mpx) rules in it (2) the depth ofψis the maximum nesting of the (sp) rules in it (2) In the example, I will be copied a number of times less than or equal to r d (2 2 = 4) NOTE: counting is possible since the equation!a=!!a is no more valid.

17 Quantitative properties of STA Linear Logic, Theorem (complexity bound) Π Γ M :σimplies M reduces to normal form in nβ-reduction steps, where n M d(π)+1 and this implies that it reduces in normal form on a TM in time: M 3 (d(π)+1) (where M is the number of symbol of M and d(π) is the maximal nesting of (sp) rule applications in Π) Remark M can be assigned an infinite number of types. Every typing for M gives an upper bound to its reduction time.

18 Coding data types Linear Logic, truth values: true=λxy.x : B f alse=λxy.y : B iterators: natural numbers (binary words): n=λxy. x(...x(x y))) : N } {{ } i n N i = α. }{{}!...! (α α) α α i [b 0, b 1,...,b n ]=λcz.cb 0 ( (cb n z)) : S i where B= α.α α α, i Nat Remark S i = α. }{{}!...! (B α α) α α i Every data type can be typed by a derivation of depth 0.

19 Coding functions Linear Logic, Letπ: N p B be a predicate of arity p. A closed term M=λx 1...x p.p codesπiff: Mn 1...n p =π(n 1...n p ) M : S i1 S i2... S ip B, (i j Nat) Letφ:N p N be a function of arity p. A closed term M=λx 1...x p.p codesφiff: Mn 1...n p =φ(n 1...n p ) M : S i1 S i2... S ip S, (i j Nat)

20 Polynomial soundness Linear Logic, Theorem (polynomial soundness) Let P be a term coding either a predicateπ: N p B or a function φ : N p N. Then Pn 1...n p reduces to normal form in a number of steps polynomial in n 1 + n n p. Proof. All n i are typed by derivations of depth 0. Let P be typed by a derivation of depth d, so the derivation for Pn 1...n p has depth d, and reduces to normal form in a number of steps which is Pn 1...n p d. Since the size of the program is a constant with respect to the computation, this time is polynomial in n 1 + n n p.

21 PTIME and FPTIME completeness Linear Logic, Theorem (PTIMEcharacterization) All decision problems that can be computed in by a TM can be coded in STA. Theorem (FPTIMEcharacterization) All functions that can be computed in by a TM can be coded in STA.

22 From PTIME to PSPACE PSPACE is the set of problems that can be solved by a TM in polynomial space. Problems: 1 How to measure the space of a reduction? (In the real programming languages substitution is not explicitly performed) 2 How to transfer our tools from time to space? Solution: 1 Use an (abstract) reduction machine for λ-calculus (performing linear substitution) 2 Use the following equivalence: Linear Logic, PSPACE = APTIME where APTIME is the set of problems solved by an Alternating Turing Machine (ATM) (i.e., computation that repeatedly fork into subcomputations and whose result is obtained by a backward computation from all the subcomputations results.)

23 Extensions of terms and types Linear Logic, Terms: Reduction rules: M ::= x 0 1 λx.m MM if Mthen Melse M (λx.m)n β M[N/x] if 0then Melse N δ M if 1then Melse N δ N βδ denotes the reflexive and transitive closure of βδ. : A ::=B α σ A α.a σ ::= A!σ (Linear )

24 The type system STAB Linear Logic, x : A x : A (Ax) 0 : B (B 0I) 1 : B (B 1I) Γ M :σ Γ, x : A M :σ (w) Γ, x :σ M : A Γ λx.m :σ A ( I) Γ M :σ A N :σ Γ# Γ, MN : A ( E) Γ, x 1 :σ,..., x n :σ M :µ Γ, x :!σ M[x/x 1,, x/x n ] :µ (mpx) Γ M :σ!γ M :!σ (sp) Γ M : A α FTV(Γ) Γ M : α.a ( I) Γ M : α.b Γ M : B[A/α] ( E) Γ M : B Γ N 0 :σ Γ N 1 :σ Γ if Mthen N 0 else N 1 :σ (BE)

25 Properties of STAB Linear Logic, subject reduction Γ M :σand M β M implyγ M :σ. strong normalization Γ M :σimplies M is strongly normalizing.

26 A leftmost outermost reduction machine Linear Logic, The machine is a set of rules of the shape: C,A = N b where: A is the store, and it allows to perform substitutions one occurrence at a time: A ::= A@{x := M} C is a context remembering the computation path, and it allows to avoid backtracking: C[ ] ::= (ifc[ ]then Lelse R )V 1 V n N is a program (a closed term of type B)

27 The rules of the machine Linear Logic, C,A =b b (Ax) C,A@{x := N} = M[x /x]v 1 V m b C,A = (λx.m)nv 1 V m b (β) {x := N} A C,A = NV 1 V m b C,A = xv 1 V m b (h) C[(if [ ]then N 0 else N 1 )V 1 V m ],A = M 0 C,A = N 0 V 1 V m b C,A = (if Mthen N 0 else N 1 )V 1 V m b (if0) C[(if [ ]then N 0 else N 1 )V 1 V m ],A = M 1 C,A = N 1 V 1 V m b C,A = (if Mthen N 0 else N 1 )V 1 V m b (if1) (*) x is a fresh variable.

28 Example Linear Logic, Let M=λx.if xthen Ixelse O(Ix)1 (where I=λx.x and O=λxy.y). Clearly M0 βδ 0 and M1 βδ 1 and both are programs. Let us evaluate M0. if [ ]then Iyelse O(Iy)1,{y := 0} = 0 0 (Ax) if [ ]then Iyelse O(Iy)1,{y := 0} = y 0 (h) [ ],{y := 0} = if ythen Iyelse O(Iy)1 0 [ ], = M0 0 [ ],{y := 0, z := y} = 0 0 (Ax) [ ],{y := 0, z := y} = y 0 (h) [ ],{y := 0, z := y} = z 0 (h) (β) [ ],{y := 0} = Iy 0 (if 0) (β)

29 PSPACE results Let the abstract machine compute:c,a = M b. Then the space used by the machine during this computation is: the maximal size of the store in the computation + the maximal size of the context in the computation Theorem (Polynomial Space Soundness) Let M be a program (a closed term of type B), and letπbe a derivation of M : B, and let d(π) be the depth ofπ(the maximal nesting of applications of (sp) rule in Π). Then M reduces to normal form (through the given abstract machine) in space Linear Logic, 3 M 3 d(π)+4 Theorem (Polynomial Space Completeness) Every decision problemd PSPACE can be coded in STAB.

30 From PSPACE to NP Linear Logic, NP is the set of problem that can be decided in by a non-deterministic TM. The language: M ::= x MM λx.m M+M The reduction rules: (λx.m)n β M[N/x] M+N γ M M+N γ N Remark The calculus is not confluent!

31 The type system STA+ x : A x : A (Ax) Γ M :σ Γ, x : A M :σ (w) Linear Logic, Γ, x :σ M : A Γ λx.m :σ A ( I) Γ M :σ A N : A Γ# Γ, MN : A ( E) Γ, x 1 :σ,..., x n :σ M : A Γ, x :!σ M[x/x 1,..., x/x n ] : A (mpx) Γ σ!γ!σ (sp) Γ A α FV(Γ) Γ M : α.a ( I) Γ M : α.a Γ M : A[B/α] ( E) Γ M : A Γ N : A (sum) Γ M+N : A

32 Properties of STA+ Linear Logic, Theorem (Subject Reduction) LetΓ M :σand M βγ N. ThenΓ N :σ. remark Terms with an exponential time behaviour can be typed: E.g.: M n((λx.zx+zx)i) where n is a Church numeral and I is the identity. Let M be the normal form of M. M N γ M in a number of steps exponential in n (β-reductions β according to an innermost strategy) M βγ M in a number of steps linear in n (a suitable outermost strategy)

33 A non-deterministic abstract machine Linear Logic, C[λx.[ ]],A = M N C,A =λx.m λx.n (λ) C,A@{x := P} = M[x /x]v 1 V m N x fresh C,A = (λx.m)pv 1 V m N (β) ( ) C[x[ ]V 2 V m ],A = V 1 N 1 C[xN 1 N m 1 [ ]],A = V m N m C,A = xv 1 V m xn 1 N m (h 1 ) {x := P} A C,A = PV 1 V m N C,A = xv 1 V m N (h) C,A = M 0 V 1 V m N C,A = (M 0 + M 1 )V 1 V m N (L) C,A = M 1 V 1 V m N C,A = (M 0 + M 1 )V 1 V m N (R) ( ) x dom(a) C ::= [ ] λx.c[ ] xm 1...M i [ ]M i+1...m n (1 i n)

34 NPTIME characterization Linear Logic, Theorem (NPTIMESoundness) LetΠ be a derivation provingγ M :σ, for someγ,σ. Then M reduces to each one of its normal forms (by the non-deterministic abstract machine) in time bounded by O( M O(d(Π)) ). Theorem (NPTIMECompleteness) Every decision problem D decidable by a non deterministic TM in can be coded by a term typable in STA+.

35 Bibliography Linear Logic, Girard, J.-Y., Linear Logic, Theoretical Computer Science 50, p , Elsevier (1987) Girard, J.-Y.,Light Linear Logic, Information and Computation 143(2), p , 1998 Lafont Y., Soft Linear Logic and Polynomial Time, Theoretical Computer Science 318, p , Elsevier (2004) Gaboardi M. and Ronchi Della S., A Soft Type Assignment System for λ-calculus, CSL 07, Lecture Notes in Computer Science, 4646, p , 2007, Springer. Gaboardi M. and Marion J.Y. and Ronchi Della S., An Implicit Characterization of PSPACE, ACM Transactions on Computational Logic, 13(2):18:1 18:36, 2012 Gaboardi M. and Ronchi Della S., From Light to Type Assignements: a case study, Logic Journal of the IGPL 17, p , 2009.

Soft Linear Logic and Polynomial Complexity Classes

Soft Linear Logic and Polynomial Complexity Classes Electronic Notes in Theoretical Computer Science 205 (2008) 67 87 www.elsevier.com/locate/entcs Soft Linear Logic and Polynomial Complexity Classes Marco Gaboardi 1 Dipartimento di Informatica, Università

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

On Elementary Linear Logic and polynomial time (Extended Abstract)

On Elementary Linear Logic and polynomial time (Extended Abstract) On Elementary Linear Logic and polynomial time (Extended Abstract) Patrick Baillot ENS Lyon, Université de Lyon, LIP (UMR 5668 CNRS-ENSL-INRIA-UCBL) 1 Introduction Linear logic (LL) [Gir87] has been used

More information

Soft Linear Logic and the Polynomial Hierarchy (Extended Abstract)

Soft Linear Logic and the Polynomial Hierarchy (Extended Abstract) Soft Linear Logic and the Polynomial Hierarchy (Extended Abstract) Brian F. Redmond Department of Computing, Mathematics and Statistical Sciences Grande Prairie Regional College 10726-106 Avenue, Grande

More information

From light logics to type assignments: a case study

From light logics to type assignments: a case study From light logics to type assignments: a case study MARCO GABOARDI, Dipartimento di Informatica, Università degli Studi di Torino. Corso Svizzera 185, 10149 Torino, Italy. E-mail: gaboardi@di.unito.it

More information

Characterizing Polynomial and Exponential Complexity Classes in Elementary Lambda-Calculus

Characterizing Polynomial and Exponential Complexity Classes in Elementary Lambda-Calculus Characterizing Polynomial and Exponential Complexity Classes in Elementary Lambda-Calculus Patric Baillot 1, Eria De Benedetti 1,2, and Simona Ronchi Della Rocca 2 1 CNRS, ENS de Lyon, INRIA, UCBL, Université

More information

Linear Logic Pages. Yves Lafont (last correction in 2017)

Linear Logic Pages. Yves Lafont (last correction in 2017) Linear Logic Pages Yves Lafont 1999 (last correction in 2017) http://iml.univ-mrs.fr/~lafont/linear/ Sequent calculus Proofs Formulas - Sequents and rules - Basic equivalences and second order definability

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

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

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

Handbook of Logic and Proof Techniques for Computer Science

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

More information

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

On the Computational Complexity of Cut-Elimination in Linear Logic

On the Computational Complexity of Cut-Elimination in Linear Logic 16/09/2003, IML p.1/40 On the Computational Complexity of Cut-Elimination in Linear Logic (Joint work with Harry Mairson) Kazushige Terui terui@nii.ac.jp National Institute of Informatics, Tokyo 16/09/2003,

More information

Constructive approach to relevant and affine term calculi

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

More information

Intersection 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

Dottorato di Ricerca in Informatica Ciclo XX. Linearity: an Analytic Tool in the Study of Complexity and Semantics of Programming Languages

Dottorato di Ricerca in Informatica Ciclo XX. Linearity: an Analytic Tool in the Study of Complexity and Semantics of Programming Languages Dipartimento di Informatica Università degli Studi di Torino Ecole doctorale IAEM Lorraine Institut National Polytechnique de Lorraine Dottorato di Ricerca in Informatica Ciclo XX Linearity: an Analytic

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

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

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

More information

Logic and Probability Lecture 3: Beyond Boolean Logic

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

More information

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

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

Most General computer?

Most General computer? Turing Machines Most General computer? DFAs are simple model of computation. Accept only the regular languages. Is there a kind of computer that can accept any language, or compute any function? Recall

More information

3 Propositional Logic

3 Propositional Logic 3 Propositional Logic 3.1 Syntax 3.2 Semantics 3.3 Equivalence and Normal Forms 3.4 Proof Procedures 3.5 Properties Propositional Logic (25th October 2007) 1 3.1 Syntax Definition 3.0 An alphabet Σ consists

More information

Preuves de logique linéaire sur machine, ENS-Lyon, Dec. 18, 2018

Preuves de logique linéaire sur machine, ENS-Lyon, Dec. 18, 2018 Université de Lorraine, LORIA, CNRS, Nancy, France Preuves de logique linéaire sur machine, ENS-Lyon, Dec. 18, 2018 Introduction Linear logic introduced by Girard both classical and intuitionistic separate

More information

if t 1,...,t k Terms and P k is a k-ary predicate, then P k (t 1,...,t k ) Formulas (atomic formulas)

if t 1,...,t k Terms and P k is a k-ary predicate, then P k (t 1,...,t k ) Formulas (atomic formulas) FOL Query Evaluation Giuseppe De Giacomo Università di Roma La Sapienza Corso di Seminari di Ingegneria del Software: Data and Service Integration Laurea Specialistica in Ingegneria Informatica Università

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

an efficient procedure for the decision problem. We illustrate this phenomenon for the Satisfiability problem.

an efficient procedure for the decision problem. We illustrate this phenomenon for the Satisfiability problem. 1 More on NP In this set of lecture notes, we examine the class NP in more detail. We give a characterization of NP which justifies the guess and verify paradigm, and study the complexity of solving search

More information

Polynomial Space. The classes PS and NPS Relationship to Other Classes Equivalence PS = NPS A PS-Complete Problem

Polynomial Space. The classes PS and NPS Relationship to Other Classes Equivalence PS = NPS A PS-Complete Problem Polynomial Space The classes PS and NPS Relationship to Other Classes Equivalence PS = NPS A PS-Complete Problem 1 Polynomial-Space-Bounded TM s A TM M is said to be polyspacebounded if there is a polynomial

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

On the satisfiability problem for a 4-level quantified syllogistic and some applications to modal logic

On the satisfiability problem for a 4-level quantified syllogistic and some applications to modal logic On the satisfiability problem for a 4-level quantified syllogistic and some applications to modal logic Domenico Cantone and Marianna Nicolosi Asmundo Dipartimento di Matematica e Informatica Università

More information

Attack of the Exponentials

Attack of the Exponentials Attack of the Exponentials Damiano Mazza LIPN, CNRS Université Paris 13, France LL2016, Lyon school: 7 and 8 November 2016 D. Mazza (LIPN) Attack of the Exponentials LL2016 1 / 26 Something is missing...

More information

Decidability: Church-Turing Thesis

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

More information

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

Lecture 4 : Quest for Structure in Counting Problems

Lecture 4 : Quest for Structure in Counting Problems CS6840: Advanced Complexity Theory Jan 10, 2012 Lecture 4 : Quest for Structure in Counting Problems Lecturer: Jayalal Sarma M.N. Scribe: Dinesh K. Theme: Between P and PSPACE. Lecture Plan:Counting problems

More information

Implicit Computational Complexity

Implicit Computational Complexity Implicit Computational Complexity Simone Martini Dipartimento di Scienze dell Informazione Università di Bologna Italy Bertinoro International Spring School for Graduate Studies in Computer Science, 6

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

Elementary Affine Logic and the Call by Value Lambda Calculus

Elementary Affine Logic and the Call by Value Lambda Calculus Elementary Affine Logic and the Call by Value Lambda Calculus Paolo Coppola 1, Ugo Dal Lago 2, and Simona Ronchi Della Rocca 3 1 Università di Udine 2 Università di Bologna 3 Università di Torino Abstract.

More information

Undecidable Problems. Z. Sawa (TU Ostrava) Introd. to Theoretical Computer Science May 12, / 65

Undecidable Problems. Z. Sawa (TU Ostrava) Introd. to Theoretical Computer Science May 12, / 65 Undecidable Problems Z. Sawa (TU Ostrava) Introd. to Theoretical Computer Science May 12, 2018 1/ 65 Algorithmically Solvable Problems Let us assume we have a problem P. If there is an algorithm solving

More information

Encoding Graph Transformation in Linear Logic

Encoding Graph Transformation in Linear Logic Encoding Graph Transformation in Linear Logic Paolo Torrini joint work with Reiko Heckel pt95@mcs.le.ac.uk University of Leicester GTLL p. 1 Graph Transformation Graph Transformation Systems (GTS) high-level

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

The Many Faces of Modal Logic Day 4: Structural Proof Theory

The Many Faces of Modal Logic Day 4: Structural Proof Theory The Many Faces of Modal Logic Day 4: Structural Proof Theory Dirk Pattinson Australian National University, Canberra (Slides based on a NASSLLI 2014 Tutorial and are joint work with Lutz Schröder) LAC

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

Programming Language Concepts: Lecture 18

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

More information

A Soft Type Assignment System for λ-calculus

A Soft Type Assignment System for λ-calculus A Soft Type Assignment System for λ-calculus Marco Gaboardi and Simona Ronchi Della Rocca Dipartimento di Informatica Università degli Studi di Torino Corso Svizzera 185, 10149 Torino, Italy gaboardi,ronchi@di.unito.it

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

A probabilistic lambda calculus - Some preliminary investigations

A probabilistic lambda calculus - Some preliminary investigations A probabilistic lambda calculus - Some preliminary investigations Ugo Dal Lago, Margherita Zorzi Università di Bologna, Università di Verona June, 9-11, 2010, Torino Introduction: Λ P We present some results

More information

Abstract model theory for extensions of modal logic

Abstract model theory for extensions of modal logic Abstract model theory for extensions of modal logic Balder ten Cate Stanford, May 13, 2008 Largely based on joint work with Johan van Benthem and Jouko Väänänen Balder ten Cate Abstract model theory for

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

Characterizing Polynomial and Exponential Complexity Classes in Elementary Lambda-Calculus

Characterizing Polynomial and Exponential Complexity Classes in Elementary Lambda-Calculus Characterizing Polynomial and Exponential Complexity Classes in Elementary Lambda-Calculus Patrick Baillot 1, Erika De Benedetti 2, and Simona Ronchi Della Rocca 2 1 CNRS, ENS de Lyon, INRIA, UCBL, Université

More information

Notes for Lecture 3... x 4

Notes for Lecture 3... x 4 Stanford University CS254: Computational Complexity Notes 3 Luca Trevisan January 14, 2014 Notes for Lecture 3 In this lecture we introduce the computational model of boolean circuits and prove that polynomial

More information

A Tableau Calculus for Minimal Modal Model Generation

A Tableau Calculus for Minimal Modal Model Generation M4M 2011 A Tableau Calculus for Minimal Modal Model Generation Fabio Papacchini 1 and Renate A. Schmidt 2 School of Computer Science, University of Manchester Abstract Model generation and minimal model

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

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

On Modal Logics of Partial Recursive Functions

On Modal Logics of Partial Recursive Functions arxiv:cs/0407031v1 [cs.lo] 12 Jul 2004 On Modal Logics of Partial Recursive Functions Pavel Naumov Computer Science Pennsylvania State University Middletown, PA 17057 naumov@psu.edu June 14, 2018 Abstract

More information

A refined calculus for Intuitionistic Propositional Logic

A refined calculus for Intuitionistic Propositional Logic A refined calculus for Intuitionistic Propositional Logic Mauro Ferrari 1, Camillo Fiorentini 2, Guido Fiorino 3 1 Dipartimento di Informatica e Comunicazione, Università degli Studi dell Insubria Via

More information

Database Theory VU , SS Complexity of Query Evaluation. Reinhard Pichler

Database Theory VU , SS Complexity of Query Evaluation. Reinhard Pichler Database Theory Database Theory VU 181.140, SS 2018 5. Complexity of Query Evaluation Reinhard Pichler Institut für Informationssysteme Arbeitsbereich DBAI Technische Universität Wien 17 April, 2018 Pichler

More information

Propositional logic (revision) & semantic entailment. p. 1/34

Propositional logic (revision) & semantic entailment. p. 1/34 Propositional logic (revision) & semantic entailment p. 1/34 Reading The background reading for propositional logic is Chapter 1 of Huth/Ryan. (This will cover approximately the first three lectures.)

More information

Decision Problems with TM s. Lecture 31: Halting Problem. Universe of discourse. Semi-decidable. Look at following sets: CSCI 81 Spring, 2012

Decision Problems with TM s. Lecture 31: Halting Problem. Universe of discourse. Semi-decidable. Look at following sets: CSCI 81 Spring, 2012 Decision Problems with TM s Look at following sets: Lecture 31: Halting Problem CSCI 81 Spring, 2012 Kim Bruce A TM = { M,w M is a TM and w L(M)} H TM = { M,w M is a TM which halts on input w} TOTAL TM

More information

WHAT IS AN SMT SOLVER? Jaeheon Yi - April 17, 2008

WHAT IS AN SMT SOLVER? Jaeheon Yi - April 17, 2008 WHAT IS AN SMT SOLVER? Jaeheon Yi - April 17, 2008 WHAT I LL TALK ABOUT Propositional Logic Terminology, Satisfiability, Decision Procedure First-Order Logic Terminology, Background Theories Satisfiability

More information

Proving Completeness for Nested Sequent Calculi 1

Proving Completeness for Nested Sequent Calculi 1 Proving Completeness for Nested Sequent Calculi 1 Melvin Fitting abstract. Proving the completeness of classical propositional logic by using maximal consistent sets is perhaps the most common method there

More information

Implicit Computational Complexity

Implicit Computational Complexity Implicit Computational Complexity Simone Martini Dipartimento di Scienze dell Informazione Università di Bologna Italy Bertinoro International Spring School for Graduate Studies in Computer Science, 6

More information

Classical First-Order Logic

Classical First-Order Logic Classical 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) First-Order Logic (Classical) MFES 2008/09

More information

Logical Structures in Natural Language: Propositional Logic II (Truth Tables and Reasoning

Logical Structures in Natural Language: Propositional Logic II (Truth Tables and Reasoning Logical Structures in Natural Language: Propositional Logic II (Truth Tables and Reasoning Raffaella Bernardi Università degli Studi di Trento e-mail: bernardi@disi.unitn.it Contents 1 What we have said

More information

PROPOSITIONAL MIXED LOGIC: ITS SYNTAX AND SEMANTICS

PROPOSITIONAL MIXED LOGIC: ITS SYNTAX AND SEMANTICS PROPOSITIONAL MIXED LOGIC: ITS SYNTAX AND SEMANTICS Karim NOUR 1 and Abir NOUR 2 Abstract In this paper, we present a propositional logic (called mixed logic) containing disjoint copies of minimal, intuitionistic

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

Introduction to Model Theory

Introduction to Model Theory Introduction to Model Theory Charles Steinhorn, Vassar College Katrin Tent, University of Münster CIRM, January 8, 2018 The three lectures Introduction to basic model theory Focus on Definability More

More information

PROOFS IN PREDICATE LOGIC AND COMPLETENESS; WHAT DECIDABILITY MEANS HUTH AND RYAN 2.3, SUPPLEMENTARY NOTES 2

PROOFS IN PREDICATE LOGIC AND COMPLETENESS; WHAT DECIDABILITY MEANS HUTH AND RYAN 2.3, SUPPLEMENTARY NOTES 2 PROOFS IN PREDICATE LOGIC AND COMPLETENESS; WHAT DECIDABILITY MEANS HUTH AND RYAN 2.3, SUPPLEMENTARY NOTES 2 Neil D. Jones DIKU 2005 12 September, 2005 Some slides today new, some based on logic 2004 (Nils

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

Propositional logic. First order logic. Alexander Clark. Autumn 2014

Propositional logic. First order logic. Alexander Clark. Autumn 2014 Propositional logic First order logic Alexander Clark Autumn 2014 Formal Logic Logical arguments are valid because of their form. Formal languages are devised to express exactly that relevant form and

More information

Team Semantics and Recursive Enumerability

Team Semantics and Recursive Enumerability Team Semantics and Recursive Enumerability Antti Kuusisto University of Wroc law, Poland, Technical University of Denmark Stockholm University, Sweden antti.j.kuusisto@uta.fi Abstract. It is well known

More information

On Sequent Calculi for Intuitionistic Propositional Logic

On Sequent Calculi for Intuitionistic Propositional Logic On Sequent Calculi for Intuitionistic Propositional Logic Vítězslav Švejdar Jan 29, 2005 The original publication is available at CMUC. Abstract The well-known Dyckoff s 1992 calculus/procedure for intuitionistic

More information

Decomposition of Computation via Linear Logic

Decomposition of Computation via Linear Logic 13/07/04, Turku p.1/44 Decomposition of Computation via Linear Logic Kazushige Terui terui@nii.ac.jp National Institute of Informatics, Tokyo 13/07/04, Turku p.2/44 Motivation (1) Linear Logic decomposes

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

Algorithmic Model Theory SS 2016

Algorithmic Model Theory SS 2016 Algorithmic Model Theory SS 2016 Prof. Dr. Erich Grädel and Dr. Wied Pakusa Mathematische Grundlagen der Informatik RWTH Aachen cbnd This work is licensed under: http://creativecommons.org/licenses/by-nc-nd/3.0/de/

More information

Theory of computation: initial remarks (Chapter 11)

Theory of computation: initial remarks (Chapter 11) Theory of computation: initial remarks (Chapter 11) For many purposes, computation is elegantly modeled with simple mathematical objects: Turing machines, finite automata, pushdown automata, and such.

More information

Propositional and Predicate Logic. jean/gbooks/logic.html

Propositional and Predicate Logic.   jean/gbooks/logic.html CMSC 630 February 10, 2009 1 Propositional and Predicate Logic Sources J. Gallier. Logic for Computer Science, John Wiley and Sons, Hoboken NJ, 1986. 2003 revised edition available on line at http://www.cis.upenn.edu/

More information

1. Propositional Calculus

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

More information

Classical First-Order Logic

Classical First-Order Logic Classical First-Order Logic Software Formal Verification Maria João Frade Departmento de Informática Universidade do Minho 2009/2010 Maria João Frade (DI-UM) First-Order Logic (Classical) MFES 2009/10

More information

Outline. Complexity Theory. Example. Sketch of a log-space TM for palindromes. Log-space computations. Example VU , SS 2018

Outline. Complexity Theory. Example. Sketch of a log-space TM for palindromes. Log-space computations. Example VU , SS 2018 Complexity Theory Complexity Theory Outline Complexity Theory VU 181.142, SS 2018 3. Logarithmic Space Reinhard Pichler Institute of Logic and Computation DBAI Group TU Wien 3. Logarithmic Space 3.1 Computational

More information

Theory of Computing Tamás Herendi

Theory of Computing Tamás Herendi Theory of Computing Tamás Herendi Theory of Computing Tamás Herendi Publication date 2014 Table of Contents 1 Preface 1 2 Formal languages 2 3 Order of growth rate 9 4 Turing machines 16 1 The definition

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

Preliminaries. Introduction to EF-games. Inexpressivity results for first-order logic. Normal forms for first-order logic

Preliminaries. Introduction to EF-games. Inexpressivity results for first-order logic. Normal forms for first-order logic Introduction to EF-games Inexpressivity results for first-order logic Normal forms for first-order logic Algorithms and complexity for specific classes of structures General complexity bounds Preliminaries

More information

07 Equational Logic and Algebraic Reasoning

07 Equational Logic and Algebraic Reasoning CAS 701 Fall 2004 07 Equational Logic and Algebraic Reasoning Instructor: W. M. Farmer Revised: 17 November 2004 1 What is Equational Logic? Equational logic is first-order logic restricted to languages

More information

THE LANGUAGE OF FIRST-ORDER LOGIC (FOL) Sec2 Sec1(1-16)

THE LANGUAGE OF FIRST-ORDER LOGIC (FOL) Sec2 Sec1(1-16) THE LANGUAGE OF FIRST-ORDER LOGIC (FOL) Sec2 Sec1(1-16) FOL: A language to formulate knowledge Logic is the study of entailment relationslanguages, truth conditions and rules of inference. FOL or Predicate

More information

The Complexity of Computing the Behaviour of Lattice Automata on Infinite Trees

The Complexity of Computing the Behaviour of Lattice Automata on Infinite Trees The Complexity of Computing the Behaviour of Lattice Automata on Infinite Trees Karsten Lehmann a, Rafael Peñaloza b a Optimisation Research Group, NICTA Artificial Intelligence Group, Australian National

More information

Propositional Dynamic Logic

Propositional Dynamic Logic Propositional Dynamic Logic Contents 1 Introduction 1 2 Syntax and Semantics 2 2.1 Syntax................................. 2 2.2 Semantics............................... 2 3 Hilbert-style axiom system

More information

Introduction to Kleene Algebra Lecture 14 CS786 Spring 2004 March 15, 2004

Introduction to Kleene Algebra Lecture 14 CS786 Spring 2004 March 15, 2004 Introduction to Kleene Algebra Lecture 14 CS786 Spring 2004 March 15, 2004 KAT and Hoare Logic In this lecture and the next we show that KAT subsumes propositional Hoare logic (PHL). Thus the specialized

More information

Turing Machines. Lecture 8

Turing Machines. Lecture 8 Turing Machines Lecture 8 1 Course Trajectory We will see algorithms, what can be done. But what cannot be done? 2 Computation Problem: To compute a function F that maps each input (a string) to an output

More information

Notes for Lecture 3... x 4

Notes for Lecture 3... x 4 Stanford University CS254: Computational Complexity Notes 3 Luca Trevisan January 18, 2012 Notes for Lecture 3 In this lecture we introduce the computational model of boolean circuits and prove that polynomial

More information

Stratifications and complexity in linear logic. Daniel Murfet

Stratifications and complexity in linear logic. Daniel Murfet Stratifications and complexity in linear logic Daniel Murfet Curry-Howard correspondence logic programming categories formula type objects sequent input/output spec proof program morphisms cut-elimination

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

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

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

More information

LOGIC PROPOSITIONAL REASONING

LOGIC PROPOSITIONAL REASONING LOGIC PROPOSITIONAL REASONING WS 2017/2018 (342.208) Armin Biere Martina Seidl biere@jku.at martina.seidl@jku.at Institute for Formal Models and Verification Johannes Kepler Universität Linz Version 2018.1

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

MTAT Complexity Theory October 13th-14th, Lecture 6

MTAT Complexity Theory October 13th-14th, Lecture 6 MTAT.07.004 Complexity Theory October 13th-14th, 2011 Lecturer: Peeter Laud Lecture 6 Scribe(s): Riivo Talviste 1 Logarithmic memory Turing machines working in logarithmic space become interesting when

More information

Lecture Notes on Linear Logic

Lecture Notes on Linear Logic Lecture Notes on Linear Logic 15-816: Modal Logic Frank Pfenning Lecture 23 April 20, 2010 1 Introduction In this lecture we will introduce linear logic [?] in its judgmental formulation [?,?]. Linear

More information

System description: CondLean

System description: CondLean System description: CondLean Nicola Olivetti, Gian Luca Pozzato Dip. di Informatica, Università degli studi di Torino Abstract. In this paper we present a theorem prover called CondLean for normal propositional

More information

NICTA Advanced Course. Theorem Proving Principles, Techniques, Applications

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

More information

Lecture 11: Measuring the Complexity of Proofs

Lecture 11: Measuring the Complexity of Proofs IAS/PCMI Summer Session 2000 Clay Mathematics Undergraduate Program Advanced Course on Computational Complexity Lecture 11: Measuring the Complexity of Proofs David Mix Barrington and Alexis Maciel July

More information

Motivation. CS389L: Automated Logical Reasoning. Lecture 10: Overview of First-Order Theories. Signature and Axioms of First-Order Theory

Motivation. CS389L: Automated Logical Reasoning. Lecture 10: Overview of First-Order Theories. Signature and Axioms of First-Order Theory Motivation CS389L: Automated Logical Reasoning Lecture 10: Overview of First-Order Theories Işıl Dillig Last few lectures: Full first-order logic In FOL, functions/predicates are uninterpreted (i.e., structure

More information