String diagrams. a functorial semantics of proofs and programs. Paul-André Melliès. CNRS, Université Paris Denis Diderot.

Size: px
Start display at page:

Download "String diagrams. a functorial semantics of proofs and programs. Paul-André Melliès. CNRS, Université Paris Denis Diderot."

Transcription

1 String diagrams a functorial semantics of proofs and programs Paul-André Melliès CNRS, Université Paris Denis Diderot Hopf-in-Lux Luxembourg 17 July

2 Proof-knots Aim: formulate an algebra of these logical knots 2

3 The purpose of semantics A mathematical study of programming languages and compilation schemes. Both functional and imperative languages, based on a kernel of λ-calculus: PCF Algol ML OCAML JAVA λ-calcul states exceptions modules concurrency higher order references objects synchronization typing threads recursion Languages designed between academic and industrial circles, between semantics (denotational or operational) and implementations. 2

4 The purpose of semantics A mathematical theory of programming languages from conception to compilation. Advanced programming language compilation Elementary commands of the machine A prerequisite to the complete verification of a given implementation. 3

5 The simply-typed λ-calculus Variable Abstraction Application Weakening Contraction Permutation x :X $ x :X Γ, x :A $ P :B Γ $ λx.p :A ñ B Γ $ P :A ñ B $ Q :A Γ, $ PQ :B Γ $ P :B Γ, x :A $ P :B Γ, x :A, y :A $ P :B Γ, z :A $ Prx, y Ð zs :B Γ, x :A, y :B, $ P :C Γ, y :B, x :A, $ P :C 4

6 Key idea Compilation itself is the ultimate semantics! Advanced programming language semantics Elementary transition systems There remains to describe the grammar of an idealized compilation. 5

7 Starting point: game semantics Every proof of formula A initiates a dialogue where Proponent tries to convince Opponent Opponent tries to refute Proponent An interactive approach to logic and programming languages 6

8 The formal proof of the drinker s formula Axiom Apx 0 q $ Apx 0 q Right Weakening Apx 0 q $ Apx 0 Right ñ $ Apx 0 q, Apx 0 q Right D $ Apx 0 q, Dy.tApyq Dy.tApyq Left Weakening Apy 0 q Dy.tApyq Right ñ $ Apy 0 q Dy.tApyq Right D $ Dy.tApyq Dy.tApyq Contraction $ Dy.tApyq 7

9 Game semantics Simply typed λ-calculus Games game semantics Games typically defined as 2-player decision trees 8

10 Sequential game semantics A proof π alternating sequences of moves A proof π Game semantics: an interleaving semantics of proofs. 9

11 Sequential games A sequential game pm, P, λq consists of M P M λ : M Ñ t 1, 1u a set of moves, a set of plays, a polarity function on moves. Alternatively, a sequential game is a polarized decision tree. 10

12 Strategies A strategy σ is a set of alternating plays of even-length s m 1 m 2k starting by an Opponent move such that: σ contains the empty play, σ is closed by n P M, s m n P σ ñ s P σ σ is P n 1, n 2 P M, s m n 1 P σ and s m n 2 P σ ñ n 1 n 2. 11

13 An interleaving semantics The boolean game B: V true q F false question Player in red Opponent in blue 12

14 Three algebraic operations on sequential games the negation A the tensor the sum A b B A ` B The same algebraic structure as in linear algebra! 13

15 Negation Proponent Program plays the game A Opponent Environment plays the game A Negation permutes the rôles of Proponent and Opponent 14

16 Negation Opponent Environment plays the game A Proponent Program plays the game A Negation permutes the rôles of Opponent and Proponent 15

17 Tensor product b Play the two games in parallel 16

18 Sum ` Proponent selects one component 17

19 A category G of games and strategies its objects A, B are the sequential games its morphisms A ÝÑ B are the strategies playing on A b B 18

20 A typical strategy R L R R L R L R L L 19

21 Composition of strategies The composite strategy of the two strategies A A ÝÑ C ÝÑ σ B B ÝÑ τ C is obtained by letting the strategies σ and τ interact on the game B. Describes the evaluation of a program and its procedure 20

22 A typical composition R L 21

23 The identity strategy The identity strategy A ÝÑ A is defined as the copycat strategy on the game A b A Clarifies the logical principle that : A or not A 22

24 An interleaving semantics The tensor product of two boolean games B 1 et B 2 : false 2 true 1 q 2 q 1 true 1 false 2 q 1 q 2 23

25 A step towards true concurrency: bend the branches! true 1 false 2 q 2 q 1 true 1 q2 q 1 false2 24

26 Asynchronous games: tile the diagram! V b q 2 true 1 V b q q b false 2 V b F q b q true 1 true 1 false 2 2 q q 1 b q 1 q 2 q b F b q q 1 false 2 b F 25

27 Asynchronous game semantics A proof π 1 trajectories in asynchronous transition spaces A proof π 2 Main result: innocent strategies are positional. 26

28 Illustration: the strategy (true b false) V b q 2 true 1 V b q q b false 2 V b F q b q true 1 true 1 false 2 2 q q 1 b q 1 q2 q b F b q q 1 false 2 b F Strategies seen as closure operators on complete lattices 27

29 Asynchronous games There are two sequential implementations of the conjunction operator ^ B b B ÝÑ B q q true q true true Left implementation B b B ÝÑ B q q true q true true Right implementation 28

30 Asynchronous games The game associated to B b B ÝÑ B looks like a flower with eight petals output cri question R input L input R input L question L question L inputr questionr question Left implementation one for each terminal position pinput L b input R q ÝÑ output of the game. 29

31 Asynchronous games true aie question R true L true R true L question L true R Left implementation question L questionr question 30

32 Asynchronous games true cri true R true L question R question L true L true R question L question R question Right implementation 31

33 Asynchronous games true cri question R true L true R true L question L question L true R questionr question Left implementation 32

34 Logical dualities in categories From orders to categories 33

35 Duality in a boolean algebra Negation defines a bijection negation B K B op negation between the boolean algebra B and its opposite boolean algebra B op. 34

36 Duality in a category Negation should define an equivalence negation C K C op negation between a cartesian closed category C and its opposite category C op. 35

37 However, in a cartesian closed category... Suppose that the category has an initial object 0. Then, Every morphism f : A ÝÑ 0 is an isomorphism. Its inverse is the unique map h making the diagram commute: id π 1 A h A 0 f π 2 A 0 36

38 In a self-dual cartesian closed category... Homp A, B q Homp A 1, B q Homp 1, A ñ B q Homp pa ñ Bq, 1 q Homp pa ñ Bq, 0 q Hence, every such self-dual category C is a preorder! 37

39 Duality in a heyting algebra Every object K defines an adjunction negation H K H op negation between the heyting algebra H and its opposite algebra H op. a H K b ðñ b H a K ðñ a K H op b 38

40 Duality in a dialogue category Negation defines an adjunction negation C K C op negation between the dialogue category C and its opposite category C op. Apa, K bq Apb, a Kq A op pa K, bq 39

41 String Diagrams A notation by Roger Penrose (1970) 40

42 Monoidal Categories A monoidal category is a category C equipped with a functor: b : C C ÝÑ C an object: I and three natural transformations: pa b Bq b C α ÝÑ A b pb b Cq I b A λ ÝÑ A A b I ρ ÝÑ A satisfying a series of coherence properties. 41

43 String Diagrams A morphism f : A b B b C ÝÑ D b E is depicted as: D E f A B C 42

44 Composition The morphism A f ÝÑ B g ÝÑ C is depicted as C C g g f = B f A A Vertical composition 43

45 The morphism pa f ÝÑ Bq b pc Tensor product g ÝÑ Dq is depicted as B D B D f g = g f A C A C Horizontal tensor product 44

46 Example B D f A D f b id D 45

47 Example B D f g A C p f b id D q pid A b gq 46

48 Example B g D f A C pid B b gq p f b id C q 47

49 Meaning preserved by deformation B D B D f g = f g A C A C p f b id D q pid A b gq = pid B b gq p f b id C q 48

50 Functorial boxes F B F B F f = f B F A F A F A F : C ÝÑ D A window on the blue C inside the ambiant D. 49

51 Functorial equalities F C F C F A F A g C g C A F B B = F B = f f B F A F A F A F A F A F A F A 50

52 Lax monoidal functor A lax monoidal functor is a functor F : C ÝÑ D equipped with morphisms m ra,bs : FA b FB ÝÑ FpA b Bq m r s : I ÝÑ FI satisfying a series of coherence relations. A strong monoidal functor is lax monoidal with invertible coercions. 51

53 The purpose of coercions F (A 1 A 2 A 3 ) F I A 1 A 2 A 3 I F A 1 A 2 A 3 F F A 1 F A 2 F A 3 m ra1,a 2,A 3 s m r s 52

54 Lax monoidal functor A lax monoidal functor is a box with many inputs - one output. F B f B F A 1 A k F A 1 F A k Fp f q m ra1,,a k s : FA 1 b b FA k ÝÑ FB 53

55 Functorial equalities (on lax functors) F C F C g C g C A 1 A k F B B = F B B f f F A 1 A i A j A k F A i A j F A 1 F A i F A j F A k F A 1 F A i F A j F A k 54

56 Strong monoidal functors A strong monoidal functor is a box with many inputs - many outputs 55

57 Functorial equalities (on strong functors) F C1 F C k F C 1 F C k C 1 C k C 1 C k g g B 1 B j = F F B 1 F B j f f F A 1 A i F A 1 A i F A 1 F A i F A 1 F A i 56

58 Functorial equalities (on strong functors) F B 1 F B k F D 1 F D l F B 1 F B k F D 1 F D l B 1 f B j D 1 g D l = B 1 f B j D 1 g D l F A 1 A i C 1 C k F A 1 A i F C 1 C k F A 1 F A i F C 1 F C k F A 1 F A i F C 1 F C k 57

59 Natural transformations A natural transformation θ : F ÝÑ G : C ÝÑ D satisfies the pictorial equality: GB GB θ F B B B f f F A = G A GA F A θ F A 58

60 Monoidal natural transformations A monoidal natural transformation θ : F ÝÑ G : C ÝÑ D satisfies the pictorial equality: GB GB θ F B B B f f F A 1 A k = G A 1 A k GA 1 GA k θ θ F A 1 F A k F A 1 F A k 59

61 The algebraic nature of knots Functorial knot theory in ribbon categories 60

62 Braided categories A monoidal category equipped with braid maps A b B γ A,B ÝÑ B b A B b A γ 1 A,B ÝÑ A b B B A A B A B B A 61

63 Coherence diagram for braids A b pb b Cq γ pb b Cq b A α α pa b Bq b C B b pc b Aq γbc pb b Aq b C α B b pa b Cq Bbγ 62

64 Topological deformation in string diagrams B C A B C A = A B C A B C 63

65 Coherence diagram for braids α 1 pa b Bq b C γ C b pa b Bq α 1 A b pb b Cq pc b Aq b B Abγ A b pc b Bq α 1 pa b Cq b B γbb 64

66 Topological deformation in string diagrams C A B C A B = A B C A B C 65

67 Duality A duality A % B is a pair of morphisms I η ÝÑ A b B B b A ɛ ÝÑ I A B A B 66

68 Duality satisfying the two zig-zag equalities: A A B B = = A A B B In that case, A is called a left dual of B. 67

69 Ribbon category A braided category in which every object A has a right dual A, satisfying: A A A A A A = = A A A A A A 68

70 Knot invariants Every ribbon category D induces a knot invariant free-ribbonpc q r s D C The free ribbon category is a category of framed tangles 69

71 Jones polynomial invariant 2 1 y2 x 2 x 4 x 2 2x 2 x 4 x 2 y 2 A compositional semantics of knots 70

72 The topological nature of negation At the interface between topology, algebra and logic 71

73 Cartesian closed categories A cartesian category C is closed when there exists a functor ñ : C op C ÝÑ C and a natural bijection ϕ A,B,C : C pa B, Cq C pa, B ñ Cq A B C A B C 72

74 The free cartesian closed category The objects of the category free-ccc(c ) are the formulas A, B :: X A B A ñ B 1 where X is an object of the category C. The morphisms are the simply-typed λ-terms, modulo βη-conversion. 73

75 The simply-typed λ-calculus Variable Abstraction Application Weakening Contraction Permutation x :X $ x :X Γ, x :A $ P :B Γ $ λx.p :A ñ B Γ $ P :A ñ B $ Q :A Γ, $ PQ :B Γ $ P :B Γ, x :A $ P :B Γ, x :A, y :A $ P :B Γ, z :A $ Prx, y Ð zs :B Γ, x :A, y :B, $ P :C Γ, y :B, x :A, $ P :C 74

76 Proof invariants Every ccc D induces a proof invariant r s modulo execution. free-cccpc q r s D C Hence the prejudice that proof theory is intrinsically syntactical... 75

77 Dialogue categories A symmetric monoidal category C equipped with a functor and a natural bijection : C op ÝÑ C ϕ A,B,C : C pa b B, Cq C pa, p B b C q q A B C A B C 76

78 The free dialogue category The objects of the category free-dialogue(c ) are dialogue games constructed by the grammar A, B :: X A b B A 1 where X is an object of the category C. The morphisms are total and innocent strategies on dialogue games. As we will see: proofs are 3-dimensional variants of knots... 77

79 A presentation of logic by generators and relations Negation defines a pair of adjoint functors L C K C op R witnessed by the series of bijection: C pa, Bq C pb, Aq C op p A, Bq 78

80 The 2-dimensional topology of adjunctions The unit and counit of the adjunction L % R are depicted as η : Id ÝÑ R L ε : L R ÝÑ Id η R L L R ε Opponent move = functor R Proponent move = functor L 79

81 A typical proof R L R R L R L R L L Reveals the algebraic nature of game semantics 80

82 A purely diagrammatic cut elimination R L 81

83 The 2-dimensional dynamic of adjunction L η ε L = L L R ε η R = R R Recovers the usual way to compose strategies in game semantics 82

84 Interesting fact There are just as many canonical proofs 2p hkkikkj hkkikkj R A $ 2q R A as there are maps rps ÝÑ rqs between the ordinals rps t0 1 p 1u and rqs. This fragment of logic has the same combinatorics as simplices. 83

85 The two generators of a monad Every increasing function is composite of faces and degeneracies: η : r0s $ r1s µ : r2s $ r1s Similarly, every proof is composite of the two generators: η : A $ A µ : A $ A The unit and multiplication of the double negation monad 84

86 The two generators in sequent calculus A $ A 2 A, A $ 1 A $ A A $ A 6 A, A $ 5 A $ A 4 A, A $ 3 A $ A 2 A, A $ 1 A $ A 85

87 The two generators in string diagrams The unit and multiplication of the monad R L are depicted as η : Id ÝÑ R L µ : R L R L ÝÑ R L R R η R L L R µ L L 86

88 Tensor and negation An atomist approach to proof theory 87

89 Four primitive components of logic r1s the negation r2s the linear conjunction b r3s the repetition modality! r4s the existential quantification D Logic = Data Structure + Duality 88

90 Tensor vs. negation A well-known fact: the continuation monad is strong p Aq b B ÝÑ pa b Bq The starting point of the algebraic theory of side effects 89

91 Tensor vs. negation Proofs are generated by a parametric strength κ X : px b Aq b B ÝÑ px b pa b Bqq which generalizes the usual notion of strong monad : κ : A b B ÝÑ pa b Bq 90

92 Proofs as 3-dimensional string diagrams The left-to-right proof of the sequent is depicted as A b B $ pa b Bq κ + κ + R ε L R L A R L B A B 91

93 Tensor vs. negation : conjunctive strength B R A 2 L A 1 κ ÝÑ B R L A 1 A 2 Linear distributivity in a continuation framework 92

94 Tensor vs. negation : disjunctive strength A L R B 1 B 2 κ ÝÑ A L B 2 R B 1 Linear distributivity in a continuation framework 93

95 A factorization theorem The four proofs η, ɛ, κ and κ generate every proof of the logic. Moreover, every such proof X ɛ ÝÑ κ ÝÑ ɛ ÝÑ ɛ ÝÑ η ÝÑ η ÝÑ κ ÝÑ ɛ ÝÑ η ÝÑ ɛ ÝÑ κ ÝÑ η ÝÑ η ÝÑ Z factors uniquely as X ɛ ÝÑÝÑ κ ÝÑÝÑ ÝÑÝÑ ÝÑÝÑ κ Z η Corollary: two proofs are equal iff they are equal as strategies 94

96 Evaluation of a strategy against a counter-strategy true η κ A κ B f actorisation κ X ε Y η Z κ C ε RLptrueq the formula X is -free and the formula Z is -free hence, the formula Y is both -free and -free hence, the formula Y it is a play! 95

97 Define a distributivity law Categorical combinatorics (Russ Harmer, Martin Hyland, PAM)!? λ ÝÑ?! between a monad? and a comonad! on a category of games. The category of dialogue games and innocent strategies recovered by a bi-kleisli construction! A ÝÑ? B Big step instead of small step 96

98 Multi-threaded strategies (Samuel Mimram, PAM) κr κ L R L R L Additional hypothesis that negation defines a monoidal functor 97

99 Revisiting the negative translation A rational reconstruction of linear logic 98

100 The algebraic point of view (in the style of Boole) The negated elements of a Heyting algebra form a Boolean algebra. 99

101 The algebraic point of view (in the style of Frege) A double negation monad is commutative iff it is idempotent. This amounts to the following diagrammatic equations: R R R R L L L L L L = L L R R = R R R R R R L L L L In that case, the negated elements form a -autonomous category. 100

102 Tensor logic tensor logic = a logic of tensor and negation = linear logic without A A = the very essence of polarized logic Offers a synthesis of linear logic, games and continuations Research program: recast every aspect of linear logic in this setting 101

103 A lax monoidal structure Typically, the family of n-ary connectives pa 1 A n q : p A 1 b b A k q : R p LA 1 LA k q is still associative, but all together, and in the lax sense. 102

104 A general phenomenon of adjunctions Given a 2-monad T and an adjunction L A K B every lax T-algebraic structure TB induces a lax T-algebraic structure R b ÝÑ B TA TL ÝÑ TB b ÝÑ B R ÝÑ A 103

105 A general phenomenon of adjunctions Consequently, every adjunction with a monoidal category B L A K B R induces a lax action of B on the category A B A B L ÝÑ B B b B ÝÑ B R ÝÑ A Enscopes the double negation monad and the arrow. 104

106 Distributivity laws seen as lax bimodules The distributivity law RpA LBq C κ ÝÑ RpA LpB Cqq may be seen as a lax notion of bimodule: pa Bq C ÝÑ A pb Cq A useful extension of the notion of strong monad (case A ) 105

107 Complementary objects in dialogue categories An involutive duality in continuations 106

108 Linearly distributive categories A category C equipped with a symmetric monoidal structure and true, a symmetric monoidal structure and false with a distributivity law δ L A,B,C δ R A,B,C : A pb Cq ÝÑ pa Bq C : pa Bq C ÝÑ A pb Cq 107

109 Pentagonal diagram ppa Bq Cq D α pa Bq pc Dq δ R A pb pc Dqq δ R D Aα pa pb Cqq D δ R A ppb Cq Dq 108

110 Pentagonal diagram ppa Bq Cq D δ R pa Bq pc Dq α A pb pc Dqq α D Aδ R pa pb Cqq D δ R A ppb Cq Dq 109

111 Pentagonal coherence diagram ppa Bq Cq D α pa Bq pc Dq δ L A pb pc Dqq δ L D Abα pa pb Cqq D δ L A ppb Cq Dq 110

112 Pentagonal coherence diagram pa Bq pc Dq δ L ppa Bq Cq D α A pb pc Dqq α D Abδ L pa pb Cqq D δ L A ppb Cq Dq 111

113 Pentagonal diagram ppa Bq Cq D δ L pa Bq pc Dq δ R A pb pc Dqq δ R D Aδ L pa pb Cqq D α A ppb Cq Dq 112

114 Pentagonal diagram ppa Bq Cq D δ R pa Bq pc Dq δ L A pb pc Dqq δ L D Abδ R pa pb Cqq D α A ppb Cq Dq 113

115 Triangular diagrams true pa Bq λ δ L A B λ B ptrue Aq B pa Bq b true ρ δ R A B Aρ A pb b trueq 114

116 Triangular diagrams A pb falseq Abρ δ L A B ρ pa Bq false pfalse Aq B λ B δ R λ A B false pa Bq 115

117 Right complementary A right complementary of the object A is an object B together with ax : true ÝÑ A A cut : A A ÝÑ false 116

118 Complementary pair making the diagrams A true Aax A pa Aq true A axa pa Aq A δ L δ R ρ pa A q A λ A pa A q A λ cuta false A A ρ A cut A false commute. 117

119 Fact A -autonomous category is the same thing as a linearly distributive category with a complementary object A for every object A. Established by Blute, Cockett and Seely 118

120 Linearly distributive adjunction A specific notion of adjunction L A K B R between two monoidal categories pa,, trueq and pb,, falseq. 119

121 Right complementary A right complementary of the object A is an object B together with ax : true ÝÑ RpA LAq cut : LpA RA q ÝÑ false 120

122 Theorem A dialogue category is the same thing as a linearly distributive adjunction with a complementary functor pa ÞÑ A q : A ÝÑ B 121

123 An amusing illustration Free monoids in games 122

124 Monoid A monoid is a game A equipped with two strategies 1 u m A A b A such that the diagrams A b A b A mba A b A 1 b A uba A b A Abu A b 1 Abm m λ m ρ A b A m A A A A commute. 123

125 Free commutative monoids Tensor algebra: Symmetric algebra: SA TA à n à n A bn A bn { Games: SA» n A bn Computed as an inductive limit in the category G of games 124

126 Computing the free commutative monoid Step 1. Compute the quotient A n A bn symmetry symmetry A bn quotient A n Step 2. The free commutative monoid SA is the inductive limit A 0 A 1 A 2 A n A n 1 The game SA is the game A where Proponent may backtrack for ever 125

127 Revisiting the drinker s formula The expressive power of resource modalities 126

128 Four primitive components of logic r1s the negation r2s the linear conjunction b r3s the repetition modality! r4s existential quantification D A theory of witnesses what remains of intuitionism

129 The classical formula translated as a game! Dy b!! Apyq Dx Apxq The repetition modality! gives an explicit account of the fact that Proponent is allowed to change her witness. 128

130 The classical formula translated as a game! Dy b!! Apyq Dx Apxq The formula explicates the exact rules of the game (and space of logical interaction) 129

131 The formal proof in tensor logic Axiom Apx 0 q $ Apx 0 q Dereliction!Apx 0 q $ Apx 0 q Left!Apx 0 q, Apx 0 q $ Weakening!Apx 0 q,! Dx Apxqq, Apx 0 q $ Right Apx 0 q $ p!apx 0 q b! Dx Apxqq Right D Apx 0 q $ Dy p!apyq b! Dx Apxqq Left Dy p!apyq b! Dx Apxqq, Apx 0 q $ Left D Dy p!apyq b! Dx Apxqq, Dx Apxq $ Dereliction Dy p!apyq b! Dx Apxqq,! Dx Apxq $ Weakening Dy p!apyq b! Dx Apxqq,!Apy 0 q,! Dx Apxq $ Right Dy p!apyq b! Dx Apxqq $ p!apy 0 q b! Dx Apxqq Right D Dy p!apyq b! Dx Apxqq $ Dy p!apyq b! Dx Apxqq Left Dy p!apyq b! Dx Apxqq, Dy p!apyq b! Dx Apxqq $ Contraction! Dy p!apyq b! Dx Apxqq $ Right $! Dy p!apyq b! Dx Apxqq 130

132 The intuitionistic formula translated as a game Dy b!! Apyq Dx Apxq This formula is not valid, because Proponent has to choose the witness y immediately and cannot change its mind later. 131

133 Conclusion Logic = Data Structure + Duality This point of view is accessible thanks to algebra 132

Quantum groupoids and logical dualities

Quantum groupoids and logical dualities Quantum groupoids and logical dualities (work in progress) Paul-André Melliès CNS, Université Paris Denis Diderot Categories, ogic and Foundations of Physics ondon 14 May 2008 1 Proof-knots Aim: formulate

More information

A quoi ressemblerait une géométrie du raisonnement?

A quoi ressemblerait une géométrie du raisonnement? Journée de la Fédération Charles Hermite A quoi ressemblerait une géométrie du raisonnement? Paul-André Melliès CNRS & Université Paris Diderot LORIA Nancy Mardi 14 octobre 2013 La prose du monde «La parole

More information

Programming Languages in String Diagrams. [ one ] String Diagrams. Paul-André Melliès. Oregon Summer School in Programming Languages June 2011

Programming Languages in String Diagrams. [ one ] String Diagrams. Paul-André Melliès. Oregon Summer School in Programming Languages June 2011 Programming Languages in String Diagrams [ one ] String Diagrams Paul-ndré Melliès Oregon Summer School in Programming Languages June 2011 String diagrams diagrammatic account o logic and programming 2

More information

Sémantique des jeux asynchrones et réécriture 2-dimensionnelle

Sémantique des jeux asynchrones et réécriture 2-dimensionnelle Sémantique des jeux asynchrones et réécriture 2-dimensionnelle Soutenance de thèse de doctorat Samuel Mimram Laboratoire PPS (CNRS Université Paris Diderot) 1 er décembre 2008 1 / 64 A program is a text

More information

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

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

More information

Theories With Duality DRAFT VERSION ONLY

Theories With Duality DRAFT VERSION ONLY Theories With Duality DRAFT VERSION ONLY John C. Baez Department of athematics, University of California Riverside, CA 9252 USA Paul-André elliès Laboratoire PPS Université Paris 7 - Denis Diderot Case

More information

An innocent model of linear logic

An innocent model of linear logic CTCS 2004 Preliminary Version Asynchronous games 3 An innocent model of linear logic Paul-André Melliès Equipe Preuves Programmes Systèmes CNRS et Université Denis Diderot Paris, France Abstract Since

More information

A Linear/Producer/Consumer model of Classical Linear Logic

A Linear/Producer/Consumer model of Classical Linear Logic A Linear/Producer/Consumer model of Classical Linear Logic Jennifer Paykin Steve Zdancewic February 14, 2014 Abstract This paper defines a new proof- and category-theoretic framework for classical linear

More information

1 The Hyland-Schalke functor G Rel. 2 Weakenings

1 The Hyland-Schalke functor G Rel. 2 Weakenings 1 The Hyland-Schalke functor G Rel Let G denote an appropriate category of games and strategies, and let Rel denote the category of sets and relations. It is known (Hyland, Schalke, 1996) that the following

More information

Asynchronous games 1: Uniformity by group invariance

Asynchronous games 1: Uniformity by group invariance synchronous games 1: Uniformity by group invariance Paul-ndré Melliès Équipe Preuves, Programmes, Systèmes CNRS, Université Paris 7 Received Ten years ago, bramsky, Jagadeesan,

More information

Programming Languages in String Diagrams. [ four ] Local stores. Paul-André Melliès. Oregon Summer School in Programming Languages June 2011

Programming Languages in String Diagrams. [ four ] Local stores. Paul-André Melliès. Oregon Summer School in Programming Languages June 2011 Programming Languages in String iagrams [ four ] Local stores Paul-André Melliès Oregon Summer School in Programming Languages June 2011 Finitary monads A monadic account of algebraic theories Algebraic

More information

A Differential Model Theory for Resource Lambda Calculi - Part I

A Differential Model Theory for Resource Lambda Calculi - Part I A Differential Model Theory for Resource Lambda Calculi - Part I Giulio Manzonetto g.manzonetto@cs.ru.nl Intelligent Systems Radboud University Nijmegen FMCS 2011 - Calgary - 11 th June 2011 Giulio Manzonetto

More information

A categorical view of computational effects

A categorical view of computational effects Emily Riehl Johns Hopkins University A categorical view of computational effects C mp se::conference 1. Functions, composition, and categories 2. Categories for computational effects (monads) 3. Categories

More information

University of Oxford, Michaelis November 16, Categorical Semantics and Topos Theory Homotopy type theor

University of Oxford, Michaelis November 16, Categorical Semantics and Topos Theory Homotopy type theor Categorical Semantics and Topos Theory Homotopy type theory Seminar University of Oxford, Michaelis 2011 November 16, 2011 References Johnstone, P.T.: Sketches of an Elephant. A Topos-Theory Compendium.

More information

A Linear/Producer/Consumer Model of Classical Linear Logic

A Linear/Producer/Consumer Model of Classical Linear Logic A Linear/Producer/Consumer Model of Classical Linear Logic Jennifer Paykin Steve Zdancewic University of Pennsylvania Philadelphia, USA jpaykin@seas.upenn.edu stevez@cis.upenn.edu This paper defines a

More information

INTRODUCTION TO PART V: CATEGORIES OF CORRESPONDENCES

INTRODUCTION TO PART V: CATEGORIES OF CORRESPONDENCES INTRODUCTION TO PART V: CATEGORIES OF CORRESPONDENCES 1. Why correspondences? This part introduces one of the two main innovations in this book the (, 2)-category of correspondences as a way to encode

More information

Resource lambda-calculus: the differential viewpoint

Resource lambda-calculus: the differential viewpoint Resource lambda-calculus: the differential viewpoint Preuves, Programmes et Systèmes (PPS) Université Paris Diderot and CNRS September 13, 2011 History ( 1985): Girard Girard had differential intuitions

More information

Teooriaseminar. TTÜ Küberneetika Instituut. May 10, Categorical Models. for Two Intuitionistic Modal Logics. Wolfgang Jeltsch.

Teooriaseminar. TTÜ Küberneetika Instituut. May 10, Categorical Models. for Two Intuitionistic Modal Logics. Wolfgang Jeltsch. TTÜ Küberneetika Instituut Teooriaseminar May 10, 2012 1 2 3 4 1 2 3 4 Modal logics used to deal with things like possibility, belief, and time in this talk only time two new operators and : ϕ now and

More information

Denotational semantics of linear logic

Denotational semantics of linear logic Denotational semantics of linear logic Lionel Vaux I2M, Université d Aix-Marseille, France LL2016, Lyon school: 7 and 8 November 2016 L. Vaux (I2M) Denotational semantics of linear logic LL2016 1 / 31

More information

DEFINITIONS: OPERADS, ALGEBRAS AND MODULES. Let S be a symmetric monoidal category with product and unit object κ.

DEFINITIONS: OPERADS, ALGEBRAS AND MODULES. Let S be a symmetric monoidal category with product and unit object κ. DEFINITIONS: OPERADS, ALGEBRAS AND MODULES J. P. MAY Let S be a symmetric monoidal category with product and unit object κ. Definition 1. An operad C in S consists of objects C (j), j 0, a unit map η :

More information

Boolean Algebra and Propositional Logic

Boolean Algebra and Propositional Logic Boolean Algebra and Propositional Logic Takahiro Kato September 10, 2015 ABSTRACT. This article provides yet another characterization of Boolean algebras and, using this characterization, establishes a

More information

Asynchronous Games vs. Concurrent Games

Asynchronous Games vs. Concurrent Games Asynchronous Games vs. Concurrent Games Paul-André Melliès Samuel Mimram Abstract Game semantics reveals the dynamic and interactive nature of logic, by interpreting every proof of a formula as a winning

More information

An introduction to Yoneda structures

An introduction to Yoneda structures An introduction to Yoneda structures Paul-André Melliès CNRS, Université Paris Denis Diderot Groupe de travail Catégories supérieures, polygraphes et homotopie Paris 21 May 2010 1 Bibliography Ross Street

More information

Boolean Algebra and Propositional Logic

Boolean Algebra and Propositional Logic Boolean Algebra and Propositional Logic Takahiro Kato June 23, 2015 This article provides yet another characterization of Boolean algebras and, using this characterization, establishes a more direct connection

More information

Olivia Caramello. University of Insubria - Como. Deductive systems and. Grothendieck topologies. Olivia Caramello. Introduction.

Olivia Caramello. University of Insubria - Como. Deductive systems and. Grothendieck topologies. Olivia Caramello. Introduction. duality University of Insubria - Como 2 / 27 duality Aim of the talk purpose of this talk is to illustrate the relevance of the notion of topology. I will show that the classical proof system of geometric

More information

A completeness theorem for symmetric product phase spaces

A completeness theorem for symmetric product phase spaces A completeness theorem for symmetric product phase spaces Thomas Ehrhard Fédération de Recherche des Unités de Mathématiques de Marseille CNRS FR 2291 Institut de Mathématiques de Luminy CNRS UPR 9016

More information

NON-SYMMETRIC -AUTONOMOUS CATEGORIES

NON-SYMMETRIC -AUTONOMOUS CATEGORIES NON-SYMMETRIC -AUTONOMOUS CATEGORIES MICHAEL BARR 1. Introduction In [Barr, 1979] (hereafter known as SCAT) the theory of -autonomous categories is outlined. Basically such a category is a symmetric monoidal

More information

Maps and Monads for Modal Frames

Maps and Monads for Modal Frames Robert Goldblatt Maps and Monads for Modal Frames Dedicated to the memory of Willem Johannes Blok. Abstract. The category-theoretic nature of general frames for modal logic is explored. A new notion of

More information

Conservation of Information

Conservation of Information Conservation of Information Amr Sabry (in collaboration with Roshan P. James) School of Informatics and Computing Indiana University May 8, 2012 Amr Sabry (in collaboration with Roshan P. James) (IU SOIC)

More information

Parameterizations and Fixed-Point Operators on Control Categories

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

More information

Relational semantics for a fragment of linear logic

Relational semantics for a fragment of linear logic Relational semantics for a fragment of linear logic Dion Coumans March 4, 2011 Abstract Relational semantics, given by Kripke frames, play an essential role in the study of modal and intuitionistic logic.

More information

Quantum Groups and Link Invariants

Quantum Groups and Link Invariants Quantum Groups and Link Invariants Jenny August April 22, 2016 1 Introduction These notes are part of a seminar on topological field theories at the University of Edinburgh. In particular, this lecture

More information

Pierre Clairambault 1

Pierre Clairambault 1 Theoretical Informatics and Applications Informatique Théorique et Applications Will be set by the publisher STRONG FUNCTORS AND INTERLEAVING FIXPOINTS IN GAME SEMANTICS Pierre Clairambault 1 Abstract.

More information

Multiple Conclusion Linear Logic: Cut-elimination and more

Multiple Conclusion Linear Logic: Cut-elimination and more Multiple Conclusion Linear Logic: Cut-elimination and more Harley Eades III Augusta University Valeria de Paiva Nuance Communications LFCS 2015 Full Intuitionistic linear Logic (FILL): Cut Elimination

More information

Categories of Coalgebraic Games with Selective Sum

Categories of Coalgebraic Games with Selective Sum Fundamenta Informaticae XX (2014) 1 20 1 DOI 10.3233/FI-2012-0000 IOS Press Categories of Coalgebraic Games with Selective Sum Furio Honsell Dipartimento di Matematica e Informatica, Università di Udine,

More information

Topos Theory. Lectures 17-20: The interpretation of logic in categories. Olivia Caramello. Topos Theory. Olivia Caramello.

Topos Theory. Lectures 17-20: The interpretation of logic in categories. Olivia Caramello. Topos Theory. Olivia Caramello. logic s Lectures 17-20: logic in 2 / 40 logic s Interpreting first-order logic in In Logic, first-order s are a wide class of formal s used for talking about structures of any kind (where the restriction

More information

MacLane s coherence theorem expressed as a word problem

MacLane s coherence theorem expressed as a word problem MacLane s coherence theorem expressed as a word problem Paul-André Melliès Preuves, Programmes, Systèmes CNRS UMR-7126, Université Paris 7 ÑÐÐ ÔÔ ºÙ ÙºÖ DRAFT In this draft, we reduce the coherence theorem

More information

Duality and Automata Theory

Duality and Automata Theory Duality and Automata Theory Mai Gehrke Université Paris VII and CNRS Joint work with Serge Grigorieff and Jean-Éric Pin Elements of automata theory A finite automaton a 1 2 b b a 3 a, b The states are

More information

The simple essence of automatic differentiation

The simple essence of automatic differentiation The simple essence of automatic differentiation Conal Elliott Target January/June 2018 Conal Elliott January/June 2018 1 / 51 Differentiable programming made easy Current AI revolution runs on large data,

More information

arxiv: v1 [cs.lo] 19 Aug 2017

arxiv: v1 [cs.lo] 19 Aug 2017 A COINTUITIONISTIC ADJOINT LOGIC e-mail address: heades@augusta.edu HARLEY EADES III AND GIANLUIGI BELLIN arxiv:1708.05896v1 [cs.lo] 19 Aug 2017 Computer Science, Augusta University, Augusta, GA e-mail

More information

A categorical model for a quantum circuit description language

A categorical model for a quantum circuit description language A categorical model for a quantum circuit description language Francisco Rios (joint work with Peter Selinger) Department of Mathematics and Statistics Dalhousie University CT July 16th 22th, 2017 What

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

1 Categorical Background

1 Categorical Background 1 Categorical Background 1.1 Categories and Functors Definition 1.1.1 A category C is given by a class of objects, often denoted by ob C, and for any two objects A, B of C a proper set of morphisms C(A,

More information

Monoidal-Closed Categories of Tree Automata

Monoidal-Closed Categories of Tree Automata Monoidal-Closed Categories of Tree Automata Colin Riba ENS de Lyon, Université de Lyon, LI colinriba@ens-lyonfr http://persoens-lyonfr/colinriba/ This paper surveys a new perspective on tree automata and

More information

Note on models of polarised intuitionistic logic

Note on models of polarised intuitionistic logic Note on models of polarised intuitionistic logic Guillaume Munch-Maccagnoni Team Gallinette, Inria Bretagne Atlantique, Univ. Nantes, LS2N, Nantes, France Guillaume.Munch-Maccagnoni@Inria.fr 3rd June 2017

More information

Sequential algorithms and strongly stable functions

Sequential algorithms and strongly stable functions Sequential algorithms and strongly stable functions Paul-André Melliès 1 Abstract Intuitionistic proofs (or PCF programs) may be interpreted as functions between domains, or as strategies on games. The

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

Thus we get. ρj. Nρj i = δ D(i),j.

Thus we get. ρj. Nρj i = δ D(i),j. 1.51. The distinguished invertible object. Let C be a finite tensor category with classes of simple objects labeled by a set I. Since duals to projective objects are projective, we can define a map D :

More information

NOTES ON ATIYAH S TQFT S

NOTES ON ATIYAH S TQFT S NOTES ON ATIYAH S TQFT S J.P. MAY As an example of categorification, I presented Atiyah s axioms [1] for a topological quantum field theory (TQFT) to undergraduates in the University of Chicago s summer

More information

Polarized Multigames. Furio Honsell 1, Marina Lenisa 1. Contents

Polarized Multigames. Furio Honsell 1, Marina Lenisa 1. Contents Under consideration for publication in Math. Struct. in Comp. Science Polarized Multigames Furio Honsell 1, Marina Lenisa 1 Dipartimento di Matematica e Informatica, Università di Udine, Italy furio.honsell@comune.udine.it,

More information

ENTROPIC HOPF ALGEBRAS AND MODELS OF NON-COMMUTATIVE LOGIC

ENTROPIC HOPF ALGEBRAS AND MODELS OF NON-COMMUTATIVE LOGIC Theory and Applications of Categories, Vol. 10, No. 17, 2002, pp. 424 460. ENTROPIC HOPF ALGEBRAS AND MODELS OF NON-COMMUTATIVE LOGIC RICHARD F. BLUTE, FRANÇOIS LAMARCHE, PAUL RUET ABSTRACT. We give a

More information

Cellularity, composition, and morphisms of algebraic weak factorization systems

Cellularity, composition, and morphisms of algebraic weak factorization systems Cellularity, composition, and morphisms of algebraic weak factorization systems Emily Riehl University of Chicago http://www.math.uchicago.edu/~eriehl 19 July, 2011 International Category Theory Conference

More information

What is a categorical model for Linear Logic?

What is a categorical model for Linear Logic? What is a categorical model for Linear Logic? ndrea Schalk Department of Computer Science University of Manchester October 15, 2004 The aim of these notes is to give an outline of the categorical structure

More information

FUNCTORS AND ADJUNCTIONS. 1. Functors

FUNCTORS AND ADJUNCTIONS. 1. Functors FUNCTORS AND ADJUNCTIONS Abstract. Graphs, quivers, natural transformations, adjunctions, Galois connections, Galois theory. 1.1. Graph maps. 1. Functors 1.1.1. Quivers. Quivers generalize directed graphs,

More information

Applications of 2-categorical algebra to the theory of operads. Mark Weber

Applications of 2-categorical algebra to the theory of operads. Mark Weber Applications of 2-categorical algebra to the theory of operads Mark Weber With new, more combinatorially intricate notions of operad arising recently in the algebraic approaches to higher dimensional algebra,

More information

A quantum double construction in Rel

A quantum double construction in Rel Under consideration for publication in Math. Struct. in Comp. Science A quantum double construction in Rel M A S A H I T O H A S E G A W A Research Institute for Mathematical Sciences, Kyoto University,

More information

Kathryn Hess. Category Theory, Algebra and Geometry Université Catholique de Louvain 27 May 2011

Kathryn Hess. Category Theory, Algebra and Geometry Université Catholique de Louvain 27 May 2011 MATHGEOM Ecole Polytechnique Fédérale de Lausanne Category Theory, Algebra and Geometry Université Catholique de Louvain 27 May 2011 Joint work with... Steve Lack (foundations) Jonathan Scott (application

More information

Categorical quantum mechanics

Categorical quantum mechanics Categorical quantum mechanics Chris Heunen 1 / 76 Categorical Quantum Mechanics? Study of compositional nature of (physical) systems Primitive notion: forming compound systems 2 / 76 Categorical Quantum

More information

Adjoint Logic and Its Concurrent Semantics

Adjoint Logic and Its Concurrent Semantics Adjoint Logic and Its Concurrent Semantics Frank Pfenning ABCD Meeting, Edinburgh, December 18-19, 2017 Joint work with Klaas Pruiksma and William Chargin Outline Proofs as programs Linear sequent proofs

More information

arxiv: v1 [cs.lo] 4 Aug 2016

arxiv: v1 [cs.lo] 4 Aug 2016 arxiv:1608.01560v1 [cs.lo] 4 Aug 2016 On partial traces and compactification of -autonomous Mix-categories Sergey Slavnov National Research University Higher School of Economics Moscow, Russia sslavnov@yandex.ru

More information

Dynamic Noninterference Analysis Using Context Sensitive Static Analyses. Gurvan Le Guernic July 14, 2007

Dynamic Noninterference Analysis Using Context Sensitive Static Analyses. Gurvan Le Guernic July 14, 2007 Dynamic Noninterference Analysis Using Context Sensitive Static Analyses Gurvan Le Guernic July 14, 2007 1 Abstract This report proposes a dynamic noninterference analysis for sequential programs. This

More information

via Topos Theory Olivia Caramello University of Cambridge The unification of Mathematics via Topos Theory Olivia Caramello

via Topos Theory Olivia Caramello University of Cambridge The unification of Mathematics via Topos Theory Olivia Caramello in University of Cambridge 2 / 23 in in In this lecture, whenever I use the word topos, I really mean Grothendieck topos. Recall that a Grothendieck topos can be seen as: a generalized space a mathematical

More information

The simple essence of automatic differentiation

The simple essence of automatic differentiation The simple essence of automatic differentiation Conal Elliott Target January/June 2018 Conal Elliott January/June 2018 1 / 52 Machine learning: promise and problems Current AI revolution runs on large

More information

Homological Algebra and Differential Linear Logic

Homological Algebra and Differential Linear Logic Homological Algebra and Differential Linear Logic Richard Blute University of Ottawa Ongoing discussions with Robin Cockett, Geoff Cruttwell, Keith O Neill, Christine Tasson, Trevor Wares February 24,

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

Subtractive Logic. To appear in Theoretical Computer Science. Tristan Crolard May 3, 1999

Subtractive Logic. To appear in Theoretical Computer Science. Tristan Crolard May 3, 1999 Subtractive Logic To appear in Theoretical Computer Science Tristan Crolard crolard@ufr-info-p7.jussieu.fr May 3, 1999 Abstract This paper is the first part of a work whose purpose is to investigate duality

More information

Zoran Petrić. 270 Minutes on Categorial Proof Theory

Zoran Petrić. 270 Minutes on Categorial Proof Theory Zoran Petrić 270 Minutes on Categorial Proof Theory Abstract. The aim of these notes is to provide an introduction of basic categorial notions to a reader interested in logic and proof theory. The first

More information

Duality in Probabilistic Automata

Duality in Probabilistic Automata Duality in Probabilistic Automata Chris Hundt Prakash Panangaden Joelle Pineau Doina Precup Gavin Seal McGill University MFPS May 2006 Genoa p.1/40 Overview We have discovered an - apparently - new kind

More information

How to combine diagrammatic logics

How to combine diagrammatic logics How to combine diagrammatic logics Dominique Duval To cite this version: Dominique Duval. How to combine diagrammatic logics. 2009. HAL Id: hal-00432330 https://hal.archives-ouvertes.fr/hal-00432330v2

More information

Embedding locales and formal topologies into positive topologies

Embedding locales and formal topologies into positive topologies Embedding locales and formal topologies into positive topologies Francesco Ciraulo Giovanni Sambin Department of Mathematics, University of Padova Via Trieste 63, 35121 Padova, Italy ciraulo@math.unipd.it,

More information

Copy-Cat Strategies and Information Flow in Physics, Geometry, Logic and Computation

Copy-Cat Strategies and Information Flow in Physics, Geometry, Logic and Computation Copy-Cat Strategies and Information Flow in Physics, Geometry, and Computation Samson Abramsky Oxford University Computing Laboratory Copy-Cat Strategies and Information Flow CQL Workshop August 2007 1

More information

Automata Theory and Formal Grammars: Lecture 1

Automata Theory and Formal Grammars: Lecture 1 Automata Theory and Formal Grammars: Lecture 1 Sets, Languages, Logic Automata Theory and Formal Grammars: Lecture 1 p.1/72 Sets, Languages, Logic Today Course Overview Administrivia Sets Theory (Review?)

More information

Partially commutative linear logic: sequent calculus and phase semantics

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

More information

Categories and Quantum Informatics

Categories and Quantum Informatics Categories and Quantum Informatics Week 6: Frobenius structures Chris Heunen 1 / 41 Overview Frobenius structure: interacting co/monoid, self-duality Normal forms: coherence theorem Frobenius law: coherence

More information

Duality in Logic. Duality in Logic. Lecture 2. Mai Gehrke. Université Paris 7 and CNRS. {ε} A ((ab) (ba) ) (ab) + (ba) +

Duality in Logic. Duality in Logic. Lecture 2. Mai Gehrke. Université Paris 7 and CNRS. {ε} A ((ab) (ba) ) (ab) + (ba) + Lecture 2 Mai Gehrke Université Paris 7 and CNRS A {ε} A ((ab) (ba) ) (ab) + (ba) + Further examples - revisited 1. Completeness of modal logic with respect to Kripke semantics was obtained via duality

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

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

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

Algebras. Larry Moss Indiana University, Bloomington. TACL 13 Summer School, Vanderbilt University

Algebras. Larry Moss Indiana University, Bloomington. TACL 13 Summer School, Vanderbilt University 1/39 Algebras Larry Moss Indiana University, Bloomington TACL 13 Summer School, Vanderbilt University 2/39 Binary trees Let T be the set which starts out as,,,, 2/39 Let T be the set which starts out as,,,,

More information

CATEGORY THEORY. Cats have been around for 70 years. Eilenberg + Mac Lane =. Cats are about building bridges between different parts of maths.

CATEGORY THEORY. Cats have been around for 70 years. Eilenberg + Mac Lane =. Cats are about building bridges between different parts of maths. CATEGORY THEORY PROFESSOR PETER JOHNSTONE Cats have been around for 70 years. Eilenberg + Mac Lane =. Cats are about building bridges between different parts of maths. Definition 1.1. A category C consists

More information

1. The Method of Coalgebra

1. The Method of Coalgebra 1. The Method of Coalgebra Jan Rutten CWI Amsterdam & Radboud University Nijmegen IMS, Singapore - 15 September 2016 Overview of Lecture one 1. Category theory (where coalgebra comes from) 2. Algebras

More information

1 Cartesian bicategories

1 Cartesian bicategories 1 Cartesian bicategories We now expand the scope of application of system Beta, by generalizing the notion of (discrete) cartesian bicategory 1. Here we give just a fragment of the theory, with a more

More information

On the categorical semantics of Elementary Linear Logic

On the categorical semantics of Elementary Linear Logic On the categorical semantics of Elementary Linear Logic Olivier Laurent Preuves Programmes Systèmes CNRS Université Paris VII bstract We introduce the notion of elementary Seely category as a notion of

More information

Categorical Semantics of Linear Logic

Categorical Semantics of Linear Logic Categorical Semantics of Linear Logic Paul-ndré Melliès Proof theory is the result of a short and tumultuous history, developed on the periphery of mainstream mathematics Hence, its language is often idiosyncratic:

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

Locally cartesian closed categories

Locally cartesian closed categories Locally cartesian closed categories Clive Newstead 80-814 Categorical Logic, Carnegie Mellon University Wednesday 1st March 2017 Abstract Cartesian closed categories provide a natural setting for the interpretation

More information

Boolean Algebras, Boolean Rings and Stone s Representation Theorem

Boolean Algebras, Boolean Rings and Stone s Representation Theorem Boolean Algebras, Boolean Rings and Stone s Representation Theorem Hongtaek Jung December 27, 2017 Abstract This is a part of a supplementary note for a Logic and Set Theory course. The main goal is to

More information

Algebras of Deductions in Category Theory. 1 Logical models from universal algebra

Algebras of Deductions in Category Theory. 1 Logical models from universal algebra THIRD MATHEMATICAL CONFERENCE OF THE REPUBLIC OF SRPSKA Trebinje, 7 and 8 June 2013 Algebras of Deductions in Category Theory Kosta Dosen Faculty of Philosophy, University of Belgrade, and Mathematical

More information

Type Systems as a Foundation for Reliable Computing

Type Systems as a Foundation for Reliable Computing Type Systems as a Foundation for Reliable Computing Robert Harper Carnegie Mellon University Summer School on Reliable Computing University of Oregon July, 2005 References These lectures are based on the

More information

Semantics of intuitionistic propositional logic

Semantics of intuitionistic propositional logic Semantics of intuitionistic propositional logic Erik Palmgren Department of Mathematics, Uppsala University Lecture Notes for Applied Logic, Fall 2009 1 Introduction Intuitionistic logic is a weakening

More information

Categorical relativistic quantum theory. Chris Heunen Pau Enrique Moliner Sean Tull

Categorical relativistic quantum theory. Chris Heunen Pau Enrique Moliner Sean Tull Categorical relativistic quantum theory Chris Heunen Pau Enrique Moliner Sean Tull 1 / 15 Idea Hilbert modules: naive quantum field theory Idempotent subunits: base space in any category Support: where

More information

The simple essence of automatic differentiation

The simple essence of automatic differentiation The simple essence of automatic differentiation Conal Elliott Target January 2018 Conal Elliott January 2018 1 / 45 What s a derivative? Number Vector Covector Matrix Higher derivatives Chain rule for

More information

Logical connections in the many-sorted setting

Logical connections in the many-sorted setting Logical connections in the many-sorted setting Jiří Velebil Czech Technical University in Prague Czech Republic joint work with Alexander Kurz University of Leicester United Kingdom AK & JV AsubL4 1/24

More information

The Safe λ-calculus. William Blum. Oxford University Computing Laboratory. DPhil Transfer thesis

The Safe λ-calculus. William Blum. Oxford University Computing Laboratory. DPhil Transfer thesis The Safe λ-calculus DPhil Transfer thesis William Blum Oxford University Computing Laboratory The Safe λ-calculus DPhil Transfer thesis The Safe λ-calculus DPhil Transfer thesis William Blum Submitted

More information

Categorical Proof Theory of Classical Propositional Calculus

Categorical Proof Theory of Classical Propositional Calculus Categorical Proof Theory of Classical Propositional Calculus Gianluigi Bellin a Martin Hyland b Edmund Robinson a Christian Urban c a Queen Mary, University of London, UK b University of Cambridge, UK

More information

C2.7: CATEGORY THEORY

C2.7: CATEGORY THEORY C2.7: CATEGORY THEORY PAVEL SAFRONOV WITH MINOR UPDATES 2019 BY FRANCES KIRWAN Contents Introduction 2 Literature 3 1. Basic definitions 3 1.1. Categories 3 1.2. Set-theoretic issues 4 1.3. Functors 5

More information

Monads and More: Part 4

Monads and More: Part 4 Monads and More: Part 4 Tarmo Uustalu, Institute of Cybernetics, Tallinn University of Nottingham, 14 18 May 2007 University of Udine, 2 6 July 2007 Comonads Comonads are the dual of monads. A comonad

More information

Notes about Filters. Samuel Mimram. December 6, 2012

Notes about Filters. Samuel Mimram. December 6, 2012 Notes about Filters Samuel Mimram December 6, 2012 1 Filters and ultrafilters Definition 1. A filter F on a poset (L, ) is a subset of L which is upwardclosed and downward-directed (= is a filter-base):

More information

A Differential Model Theory for Resource Lambda Calculi - Part II

A Differential Model Theory for Resource Lambda Calculi - Part II A Differential Model Theory for Resource Lambda Calculi - Part II Giulio Manzonetto (joint work with Bucciarelli, Ehrhard, Laird, McCusker) g.manzonetto@cs.ru.nl Intelligent Systems Radboud University

More information

Lecture Notes on Classical Linear Logic

Lecture Notes on Classical Linear Logic Lecture Notes on Classical Linear Logic 15-816: Linear Logic Frank Pfenning Lecture 25 April 23, 2012 Originally, linear logic was conceived by Girard [Gir87] as a classical system, with one-sided sequents,

More information