SlideShare ist ein Scribd-Unternehmen logo
1 von 33
Downloaden Sie, um offline zu lesen
Truth, Deduction,
Computation
Lecture F
Untyped λ... and other things
Vlad Patryshev
SCU
2013
Functions
f: X → Y; X - domain, X - codomain.
∀ x:X ∃ y:Y (y=f(x))

y

y

x
A Function

x
Not a Function
Functions. Definitions
Monomorphism, aka injective function, aka one-to-one function

∀x ∀y (f(x)=f(y) → x=y)
f: X ↣ Y
Functions. Definitions
Epimorphism, aka surjective function, aka onto function

∀y ∃x (f(x)=y)
f: X ↠ Y
Functions. Definitions
Bijection, aka bijective function, aka one-to-one correspondence

f is injection and surjection
f: A
Functions. Composition
● f: X → Y
● g: Y → Z
● h=g∘f

(g∘f)(x) = g(f(x))
h

→
Functions. Identity
● id: X → X
● id∘f=f=f∘id

IdX

→

X

id(x)=x
Functions. Make a monoid
f,g: X → X
● binary operation: f∘g
● neutral element: id
● associativity: (f∘g)∘h = f∘(g∘h)
Currying
Having a function
f: (x1,x2,...xn) → y
is equivalent to having a function
f c: x 1 → x 2 → … → x n → y
Functions in Programming languages
Language

Code Sample

Java

interface Function<X,Y> {
public Y apply(x: X)
}
Function<Int,String> f =
new Function<Int,String>() {
public String apply(n: Int) {
return "n=" + n;
}

Scala

val f:(Int => String) = (n:Int) => "n=" + n

Javascript

f = function(n) { return "n=" + n }
Peano Arithmetic
1.
2.
3.
4.
5.
6.
7.
8.

objects are called natural numbers
equality is defined, with usual properties
0 is a natural number
function s: s(x) is natural number
∀x (s(x) ≠ 0)
∀x∀y (s(x) = s(y) → x = y)
P(0), ∀x (P(x)→P(s(x))) ⊢ ∀x P(x)
define 1 as s(0)
Peano Arithmetic Illustrated

Giuseppe Peano

Domino model of Peano Arithmetic
Peano Arithmetic: define +
● x+0 = x
● x+s(y) = s(x+y)
● have a monoid
Peano Arithmetic: define ×
● x×0 = 0
● x×s(y) = x + (x×y)
● have a monoid
Peano Arithmetic: define ↑ etc
● x↑0 = 1
● x↑s(y) = x × (x↑y)
● (strangely, no associativity)
● x⇑↑0 = 1
● x⇑s(y) = x ↑ (x⇑y)
(Some people argue lately that this makes it
inconsistent)
Peano Arithmetic: Universal Property
Alonzo Church
●
●
●

Peano arithmetics is undecidable
Every effectively calculable function is a
computable function
Invented λ-calculus which is equivalent to
effectively calculable functions

Is it so that all that machines can do is equivalent to
lambdas?
Church-Rosser thesis: YES!
https://files.nyu.edu/cb125/public/Lambda/barendregt.94.pdf
So, can we build Peano arithmetic?
They are called Church Numerals
0:
1:
2:
…
n:

f → id
f → f
f → f∘f
f → f∘…∘f

}

●
●
●
●
●

n times
Simplest Language for Calculations
●
●
●
●

<λ
<λ
<λ
<λ

term>::=<variable>
term>::=<λ term> <λ term>
term>::=(λ <variable> <λ term>)
term>::=(<λ term>)

application
abstraction

http://www.itu.dk/people/sestoft/lamreduce/lamframes.html
Javascript Interpretation
● we have as many variables as we like
● λ x N ≡ function(x) {return N}
● (M N) ≡ M(N)

http://myjavatools.com/js.html
Examples of λ terms
●
●
●
●
●

x
λ x x
(x y)
((λ x x)(z t))
λ x ((x x) (x x))
Does not make much sense so far, right?
Same things in Javascript
●
●
●
●
●

x
function(x) {return x}
x(y)
(function(x) {return x})(z(t))
function(x) {return x(x)(x(x))}
Rules of Transformation
● α-equivalence, renaming bound(*) variables
● β-conversion (substitution/λ intro)
● η-conversion
Substitutions
1.
2.
3.
4.
5.

x[x:=N]
y[x:=N]
(M1 M2)[x:=N]
(λx M)[x:=N]
(λy M)[x:=N]

≡
≡
≡
≡
≡

N
y, if x ≠ y
(M1[x:=N]) (M2[x:=N])
λx M
λy (M[x:=N])//if x≠y and

y∉FV(N)
α-equivalence rule
Bound variable in a lambda expression - the one
which name is found right after λ.

● λx (λy (x (y z)))
Two lambda expressions differing only in names of
bound variables are equivalent.

λx (λy (x (y z))) ⇔ λt (λw (t (w z)))
λx (λy (x (y z))) ⇔ λz (λw (z (w z)))
Like in Javascript
function(x) {
return function(y) {
return y(function(z) { return z(x) }
}
}
// same as
function(a) {
return function(b) {
return b(function(c) { return c(a) }
}
}
β-conversion rule
(λx E) E’ ⇔ E[x := E’]

●
●
●
●

(λx
(λx
(λx
(λy

x) (y z) ⇔ (y z)
x) (λy y) ⇔ λy y ⇔ λx x
x) (λy y y) ⇔ λy y y
y y) (λx x) ⇔ (λx x) (λx x) ⇔ (λx x)
β-conversion is
β-reduction + β-abstraction
β-reduction
(λx E) E’ ⇒ E[x := E’]

β-abstraction
(λx E) E’ ⇐ E[x := E’]
β-reduction in Javascript
(function(x) {return M})(N)
Substitute all x in M with N
β-reduction - tautological case
●
●
●
●

t =
t t
(λx
(λx

λx x // identity function, right?
= ?
x) M = M
x) (λa a) = λa a
β-reduction - tautology, Javascript
id = function(x) { println(“<<x>>”);
return x }
id(id)
β-reduction - weird case
●
●
●
●

t =
t t
(λx
(λx

λx (x x)
= ?
(x x)) (λx (x x)) =...
(x x)) (λx (x x)) - oops.
That’s it for today

Weitere ähnliche Inhalte

Was ist angesagt?

Inverse composite functions
Inverse composite functionsInverse composite functions
Inverse composite functionsDebra Wallace
 
Admissions in india 2015
Admissions in india 2015Admissions in india 2015
Admissions in india 2015Edhole.com
 
Tutorials--Graphs of Rational Functions
Tutorials--Graphs of Rational FunctionsTutorials--Graphs of Rational Functions
Tutorials--Graphs of Rational FunctionsMedia4math
 
4 5 inverse functions
4 5 inverse functions4 5 inverse functions
4 5 inverse functionshisema01
 
Exponential and logarithmic functions
Exponential and logarithmic functionsExponential and logarithmic functions
Exponential and logarithmic functionsNjabulo Nkabinde
 
Pre-Cal 40S Slides February 29, 2008
Pre-Cal 40S Slides February 29, 2008Pre-Cal 40S Slides February 29, 2008
Pre-Cal 40S Slides February 29, 2008Darren Kuropatwa
 
Inverse Functions
Inverse FunctionsInverse Functions
Inverse Functionstschmucker
 
Continuity Of Functions
Continuity Of FunctionsContinuity Of Functions
Continuity Of FunctionsYash Thakkar
 
5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.Jan Plaza
 
Math 4 6
Math 4 6Math 4 6
Math 4 6dears11
 
7.7 one to_one_functions_-_inverse_functions
7.7 one to_one_functions_-_inverse_functions7.7 one to_one_functions_-_inverse_functions
7.7 one to_one_functions_-_inverse_functionsarvin gutierrez
 
53 inverse function (optional)
53 inverse function (optional)53 inverse function (optional)
53 inverse function (optional)math126
 
Graphing rational functions
Graphing rational functionsGraphing rational functions
Graphing rational functionsJessica Garcia
 
Top School in Delhi NCR
Top School in Delhi NCRTop School in Delhi NCR
Top School in Delhi NCREdhole.com
 
Graphing rational functions
Graphing rational functionsGraphing rational functions
Graphing rational functionsrey castro
 

Was ist angesagt? (19)

Matlab
MatlabMatlab
Matlab
 
Inverse composite functions
Inverse composite functionsInverse composite functions
Inverse composite functions
 
24 modelling
24 modelling24 modelling
24 modelling
 
Admissions in india 2015
Admissions in india 2015Admissions in india 2015
Admissions in india 2015
 
Tutorials--Graphs of Rational Functions
Tutorials--Graphs of Rational FunctionsTutorials--Graphs of Rational Functions
Tutorials--Graphs of Rational Functions
 
Tipos de funciones
Tipos de funcionesTipos de funciones
Tipos de funciones
 
4 5 inverse functions
4 5 inverse functions4 5 inverse functions
4 5 inverse functions
 
Exponential and logarithmic functions
Exponential and logarithmic functionsExponential and logarithmic functions
Exponential and logarithmic functions
 
Pre-Cal 40S Slides February 29, 2008
Pre-Cal 40S Slides February 29, 2008Pre-Cal 40S Slides February 29, 2008
Pre-Cal 40S Slides February 29, 2008
 
Inverse Functions
Inverse FunctionsInverse Functions
Inverse Functions
 
Continuity Of Functions
Continuity Of FunctionsContinuity Of Functions
Continuity Of Functions
 
Fun37
Fun37Fun37
Fun37
 
5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.5.3 Basic functions. Dynamic slides.
5.3 Basic functions. Dynamic slides.
 
Math 4 6
Math 4 6Math 4 6
Math 4 6
 
7.7 one to_one_functions_-_inverse_functions
7.7 one to_one_functions_-_inverse_functions7.7 one to_one_functions_-_inverse_functions
7.7 one to_one_functions_-_inverse_functions
 
53 inverse function (optional)
53 inverse function (optional)53 inverse function (optional)
53 inverse function (optional)
 
Graphing rational functions
Graphing rational functionsGraphing rational functions
Graphing rational functions
 
Top School in Delhi NCR
Top School in Delhi NCRTop School in Delhi NCR
Top School in Delhi NCR
 
Graphing rational functions
Graphing rational functionsGraphing rational functions
Graphing rational functions
 

Andere mochten auch

Natural Language Access to Data via Deduction
Natural Language Access to Data via DeductionNatural Language Access to Data via Deduction
Natural Language Access to Data via Deductiondiannepatricia
 
Deduction theorem of propositional logic
Deduction theorem of propositional logicDeduction theorem of propositional logic
Deduction theorem of propositional logicSaurabh Gupta
 
Logic Notes
Logic NotesLogic Notes
Logic Notesacavis
 
Formal methods 4 - Z notation
Formal methods   4 - Z notationFormal methods   4 - Z notation
Formal methods 4 - Z notationVlad Patryshev
 
Formal Methods lecture 01
Formal Methods lecture 01Formal Methods lecture 01
Formal Methods lecture 01Sidra Ashraf
 
#1 formal methods – introduction for software engineering
#1 formal methods – introduction for software engineering#1 formal methods – introduction for software engineering
#1 formal methods – introduction for software engineeringSharif Omar Salem
 
Formal Specification in Software Engineering SE9
Formal Specification in Software Engineering SE9Formal Specification in Software Engineering SE9
Formal Specification in Software Engineering SE9koolkampus
 
Propositional logic & inference
Propositional logic & inferencePropositional logic & inference
Propositional logic & inferenceSlideshare
 
Syntax and semantics of propositional logic
Syntax and semantics of propositional logicSyntax and semantics of propositional logic
Syntax and semantics of propositional logicJanet Stemwedel
 
Judgment and proposition or logical statement
Judgment and proposition or logical statementJudgment and proposition or logical statement
Judgment and proposition or logical statementling selanoba
 
Discrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكرو
Discrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكروDiscrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكرو
Discrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكروDr. Khaled Bakro
 
Discrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكرو
Discrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكروDiscrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكرو
Discrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكروDr. Khaled Bakro
 
Propositional And First-Order Logic
Propositional And First-Order LogicPropositional And First-Order Logic
Propositional And First-Order Logicankush_kumar
 
Translating English to Propositional Logic
Translating English to Propositional LogicTranslating English to Propositional Logic
Translating English to Propositional LogicJanet Stemwedel
 

Andere mochten auch (17)

Natural Language Access to Data via Deduction
Natural Language Access to Data via DeductionNatural Language Access to Data via Deduction
Natural Language Access to Data via Deduction
 
Deduction theorem of propositional logic
Deduction theorem of propositional logicDeduction theorem of propositional logic
Deduction theorem of propositional logic
 
Logic Notes
Logic NotesLogic Notes
Logic Notes
 
Formal methods 4 - Z notation
Formal methods   4 - Z notationFormal methods   4 - Z notation
Formal methods 4 - Z notation
 
Z specification
Z specificationZ specification
Z specification
 
Formal Methods lecture 01
Formal Methods lecture 01Formal Methods lecture 01
Formal Methods lecture 01
 
Formal Methods
Formal MethodsFormal Methods
Formal Methods
 
#1 formal methods – introduction for software engineering
#1 formal methods – introduction for software engineering#1 formal methods – introduction for software engineering
#1 formal methods – introduction for software engineering
 
Formal Specification in Software Engineering SE9
Formal Specification in Software Engineering SE9Formal Specification in Software Engineering SE9
Formal Specification in Software Engineering SE9
 
Propositional logic & inference
Propositional logic & inferencePropositional logic & inference
Propositional logic & inference
 
Syntax and semantics of propositional logic
Syntax and semantics of propositional logicSyntax and semantics of propositional logic
Syntax and semantics of propositional logic
 
Judgment and proposition or logical statement
Judgment and proposition or logical statementJudgment and proposition or logical statement
Judgment and proposition or logical statement
 
Discrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكرو
Discrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكروDiscrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكرو
Discrete mathematics Ch1 sets Theory_Dr.Khaled.Bakro د. خالد بكرو
 
Logic Ppt
Logic PptLogic Ppt
Logic Ppt
 
Discrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكرو
Discrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكروDiscrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكرو
Discrete mathematics Ch2 Propositional Logic_Dr.khaled.Bakro د. خالد بكرو
 
Propositional And First-Order Logic
Propositional And First-Order LogicPropositional And First-Order Logic
Propositional And First-Order Logic
 
Translating English to Propositional Logic
Translating English to Propositional LogicTranslating English to Propositional Logic
Translating English to Propositional Logic
 

Ähnlich wie Truth, deduction, computation lecture f

Hyperfunction method for numerical integration and Fredholm integral equation...
Hyperfunction method for numerical integration and Fredholm integral equation...Hyperfunction method for numerical integration and Fredholm integral equation...
Hyperfunction method for numerical integration and Fredholm integral equation...HidenoriOgata
 
237654933 mathematics-t-form-6
237654933 mathematics-t-form-6237654933 mathematics-t-form-6
237654933 mathematics-t-form-6homeworkping3
 
Integration+using+u-substitutions
Integration+using+u-substitutionsIntegration+using+u-substitutions
Integration+using+u-substitutionstutorcircle1
 
Functions for Grade 10
Functions for Grade 10Functions for Grade 10
Functions for Grade 10Boipelo Radebe
 
CVPR2010: higher order models in computer vision: Part 1, 2
CVPR2010: higher order models in computer vision: Part 1, 2CVPR2010: higher order models in computer vision: Part 1, 2
CVPR2010: higher order models in computer vision: Part 1, 2zukun
 
Calculus- Basics
Calculus- BasicsCalculus- Basics
Calculus- BasicsRabin BK
 
Truth, deduction, computation lecture a
Truth, deduction, computation   lecture aTruth, deduction, computation   lecture a
Truth, deduction, computation lecture aVlad Patryshev
 
CAT Functions and Graphs basics
CAT Functions and Graphs basicsCAT Functions and Graphs basics
CAT Functions and Graphs basicsGeorge Prep
 
AP Calculus Slides September 18, 2007
AP Calculus Slides September 18, 2007AP Calculus Slides September 18, 2007
AP Calculus Slides September 18, 2007Darren Kuropatwa
 
A Brief Introduction to Linear Regression
A Brief Introduction to Linear RegressionA Brief Introduction to Linear Regression
A Brief Introduction to Linear RegressionNidhal Selmi
 
Numerical integration based on the hyperfunction theory
Numerical integration based on the hyperfunction theoryNumerical integration based on the hyperfunction theory
Numerical integration based on the hyperfunction theoryHidenoriOgata
 
Lesson 1
Lesson 1Lesson 1
Lesson 1urenaa
 
WEEK-4-Piecewise-Function-and-Rational-Function.pptx
WEEK-4-Piecewise-Function-and-Rational-Function.pptxWEEK-4-Piecewise-Function-and-Rational-Function.pptx
WEEK-4-Piecewise-Function-and-Rational-Function.pptxExtremelyDarkness2
 
Lesson 1
Lesson 1Lesson 1
Lesson 1urenaa
 

Ähnlich wie Truth, deduction, computation lecture f (20)

.
..
.
 
Hyperfunction method for numerical integration and Fredholm integral equation...
Hyperfunction method for numerical integration and Fredholm integral equation...Hyperfunction method for numerical integration and Fredholm integral equation...
Hyperfunction method for numerical integration and Fredholm integral equation...
 
Matrix calculus
Matrix calculusMatrix calculus
Matrix calculus
 
237654933 mathematics-t-form-6
237654933 mathematics-t-form-6237654933 mathematics-t-form-6
237654933 mathematics-t-form-6
 
Integration+using+u-substitutions
Integration+using+u-substitutionsIntegration+using+u-substitutions
Integration+using+u-substitutions
 
Functions for Grade 10
Functions for Grade 10Functions for Grade 10
Functions for Grade 10
 
CVPR2010: higher order models in computer vision: Part 1, 2
CVPR2010: higher order models in computer vision: Part 1, 2CVPR2010: higher order models in computer vision: Part 1, 2
CVPR2010: higher order models in computer vision: Part 1, 2
 
R lecture co4_math 21-1
R lecture co4_math 21-1R lecture co4_math 21-1
R lecture co4_math 21-1
 
A taste of Functional Programming
A taste of Functional ProgrammingA taste of Functional Programming
A taste of Functional Programming
 
Calculus- Basics
Calculus- BasicsCalculus- Basics
Calculus- Basics
 
Lecture Notes In Algebra
Lecture Notes In AlgebraLecture Notes In Algebra
Lecture Notes In Algebra
 
Chapter 4 and half
Chapter 4 and halfChapter 4 and half
Chapter 4 and half
 
Truth, deduction, computation lecture a
Truth, deduction, computation   lecture aTruth, deduction, computation   lecture a
Truth, deduction, computation lecture a
 
CAT Functions and Graphs basics
CAT Functions and Graphs basicsCAT Functions and Graphs basics
CAT Functions and Graphs basics
 
AP Calculus Slides September 18, 2007
AP Calculus Slides September 18, 2007AP Calculus Slides September 18, 2007
AP Calculus Slides September 18, 2007
 
A Brief Introduction to Linear Regression
A Brief Introduction to Linear RegressionA Brief Introduction to Linear Regression
A Brief Introduction to Linear Regression
 
Numerical integration based on the hyperfunction theory
Numerical integration based on the hyperfunction theoryNumerical integration based on the hyperfunction theory
Numerical integration based on the hyperfunction theory
 
Lesson 1
Lesson 1Lesson 1
Lesson 1
 
WEEK-4-Piecewise-Function-and-Rational-Function.pptx
WEEK-4-Piecewise-Function-and-Rational-Function.pptxWEEK-4-Piecewise-Function-and-Rational-Function.pptx
WEEK-4-Piecewise-Function-and-Rational-Function.pptx
 
Lesson 1
Lesson 1Lesson 1
Lesson 1
 

Mehr von Vlad Patryshev

Formal methods 8 - category theory (last one)
Formal methods   8 - category theory (last one)Formal methods   8 - category theory (last one)
Formal methods 8 - category theory (last one)Vlad Patryshev
 
Formal methods 6 - elements of algebra
Formal methods   6 - elements of algebraFormal methods   6 - elements of algebra
Formal methods 6 - elements of algebraVlad Patryshev
 
Formal methods 5 - Pi calculus
Formal methods   5 - Pi calculusFormal methods   5 - Pi calculus
Formal methods 5 - Pi calculusVlad Patryshev
 
Formal methods 3 - languages and machines
Formal methods   3 - languages and machinesFormal methods   3 - languages and machines
Formal methods 3 - languages and machinesVlad Patryshev
 
Formal methods 2 - languages and machines
Formal methods   2 - languages and machinesFormal methods   2 - languages and machines
Formal methods 2 - languages and machinesVlad Patryshev
 
Formal methods 1 - introduction
Formal methods   1 - introductionFormal methods   1 - introduction
Formal methods 1 - introductionVlad Patryshev
 
Formal methods 7 - category theory
Formal methods   7 - category theoryFormal methods   7 - category theory
Formal methods 7 - category theoryVlad Patryshev
 
Truth, deduction, computation lecture i (last one)
Truth, deduction, computation   lecture i (last one)Truth, deduction, computation   lecture i (last one)
Truth, deduction, computation lecture i (last one)Vlad Patryshev
 
Truth, deduction, computation lecture h
Truth, deduction, computation   lecture hTruth, deduction, computation   lecture h
Truth, deduction, computation lecture hVlad Patryshev
 
Truth, deduction, computation lecture e
Truth, deduction, computation   lecture eTruth, deduction, computation   lecture e
Truth, deduction, computation lecture eVlad Patryshev
 
Truth, deduction, computation lecture d
Truth, deduction, computation   lecture dTruth, deduction, computation   lecture d
Truth, deduction, computation lecture dVlad Patryshev
 
Truth, deduction, computation lecture c
Truth, deduction, computation   lecture cTruth, deduction, computation   lecture c
Truth, deduction, computation lecture cVlad Patryshev
 
Truth, deduction, computation lecture b
Truth, deduction, computation   lecture bTruth, deduction, computation   lecture b
Truth, deduction, computation lecture bVlad Patryshev
 
Truth, deduction, computation lecture 9
Truth, deduction, computation   lecture 9Truth, deduction, computation   lecture 9
Truth, deduction, computation lecture 9Vlad Patryshev
 
Truth, deduction, computation lecture 8
Truth, deduction, computation   lecture 8Truth, deduction, computation   lecture 8
Truth, deduction, computation lecture 8Vlad Patryshev
 
Truth, deduction, computation lecture 7
Truth, deduction, computation   lecture 7Truth, deduction, computation   lecture 7
Truth, deduction, computation lecture 7Vlad Patryshev
 
Truth, deduction, computation lecture 6
Truth, deduction, computation   lecture 6Truth, deduction, computation   lecture 6
Truth, deduction, computation lecture 6Vlad Patryshev
 
Truth, deduction, computation; lecture 5
Truth, deduction, computation;  lecture 5Truth, deduction, computation;  lecture 5
Truth, deduction, computation; lecture 5Vlad Patryshev
 
Truth, deduction, computation; lecture 4
Truth, deduction, computation;  lecture 4Truth, deduction, computation;  lecture 4
Truth, deduction, computation; lecture 4Vlad Patryshev
 
Truth, deduction, computation; lecture 3
Truth, deduction, computation;  lecture 3Truth, deduction, computation;  lecture 3
Truth, deduction, computation; lecture 3Vlad Patryshev
 

Mehr von Vlad Patryshev (20)

Formal methods 8 - category theory (last one)
Formal methods   8 - category theory (last one)Formal methods   8 - category theory (last one)
Formal methods 8 - category theory (last one)
 
Formal methods 6 - elements of algebra
Formal methods   6 - elements of algebraFormal methods   6 - elements of algebra
Formal methods 6 - elements of algebra
 
Formal methods 5 - Pi calculus
Formal methods   5 - Pi calculusFormal methods   5 - Pi calculus
Formal methods 5 - Pi calculus
 
Formal methods 3 - languages and machines
Formal methods   3 - languages and machinesFormal methods   3 - languages and machines
Formal methods 3 - languages and machines
 
Formal methods 2 - languages and machines
Formal methods   2 - languages and machinesFormal methods   2 - languages and machines
Formal methods 2 - languages and machines
 
Formal methods 1 - introduction
Formal methods   1 - introductionFormal methods   1 - introduction
Formal methods 1 - introduction
 
Formal methods 7 - category theory
Formal methods   7 - category theoryFormal methods   7 - category theory
Formal methods 7 - category theory
 
Truth, deduction, computation lecture i (last one)
Truth, deduction, computation   lecture i (last one)Truth, deduction, computation   lecture i (last one)
Truth, deduction, computation lecture i (last one)
 
Truth, deduction, computation lecture h
Truth, deduction, computation   lecture hTruth, deduction, computation   lecture h
Truth, deduction, computation lecture h
 
Truth, deduction, computation lecture e
Truth, deduction, computation   lecture eTruth, deduction, computation   lecture e
Truth, deduction, computation lecture e
 
Truth, deduction, computation lecture d
Truth, deduction, computation   lecture dTruth, deduction, computation   lecture d
Truth, deduction, computation lecture d
 
Truth, deduction, computation lecture c
Truth, deduction, computation   lecture cTruth, deduction, computation   lecture c
Truth, deduction, computation lecture c
 
Truth, deduction, computation lecture b
Truth, deduction, computation   lecture bTruth, deduction, computation   lecture b
Truth, deduction, computation lecture b
 
Truth, deduction, computation lecture 9
Truth, deduction, computation   lecture 9Truth, deduction, computation   lecture 9
Truth, deduction, computation lecture 9
 
Truth, deduction, computation lecture 8
Truth, deduction, computation   lecture 8Truth, deduction, computation   lecture 8
Truth, deduction, computation lecture 8
 
Truth, deduction, computation lecture 7
Truth, deduction, computation   lecture 7Truth, deduction, computation   lecture 7
Truth, deduction, computation lecture 7
 
Truth, deduction, computation lecture 6
Truth, deduction, computation   lecture 6Truth, deduction, computation   lecture 6
Truth, deduction, computation lecture 6
 
Truth, deduction, computation; lecture 5
Truth, deduction, computation;  lecture 5Truth, deduction, computation;  lecture 5
Truth, deduction, computation; lecture 5
 
Truth, deduction, computation; lecture 4
Truth, deduction, computation;  lecture 4Truth, deduction, computation;  lecture 4
Truth, deduction, computation; lecture 4
 
Truth, deduction, computation; lecture 3
Truth, deduction, computation;  lecture 3Truth, deduction, computation;  lecture 3
Truth, deduction, computation; lecture 3
 

Kürzlich hochgeladen

1029 - Danh muc Sach Giao Khoa 10 . pdf
1029 -  Danh muc Sach Giao Khoa 10 . pdf1029 -  Danh muc Sach Giao Khoa 10 . pdf
1029 - Danh muc Sach Giao Khoa 10 . pdfQucHHunhnh
 
Contemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptx
Contemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptxContemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptx
Contemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptxRoyAbrique
 
Q4-W6-Restating Informational Text Grade 3
Q4-W6-Restating Informational Text Grade 3Q4-W6-Restating Informational Text Grade 3
Q4-W6-Restating Informational Text Grade 3JemimahLaneBuaron
 
Z Score,T Score, Percential Rank and Box Plot Graph
Z Score,T Score, Percential Rank and Box Plot GraphZ Score,T Score, Percential Rank and Box Plot Graph
Z Score,T Score, Percential Rank and Box Plot GraphThiyagu K
 
BASLIQ CURRENT LOOKBOOK LOOKBOOK(1) (1).pdf
BASLIQ CURRENT LOOKBOOK  LOOKBOOK(1) (1).pdfBASLIQ CURRENT LOOKBOOK  LOOKBOOK(1) (1).pdf
BASLIQ CURRENT LOOKBOOK LOOKBOOK(1) (1).pdfSoniaTolstoy
 
microwave assisted reaction. General introduction
microwave assisted reaction. General introductionmicrowave assisted reaction. General introduction
microwave assisted reaction. General introductionMaksud Ahmed
 
Grant Readiness 101 TechSoup and Remy Consulting
Grant Readiness 101 TechSoup and Remy ConsultingGrant Readiness 101 TechSoup and Remy Consulting
Grant Readiness 101 TechSoup and Remy ConsultingTechSoup
 
Accessible design: Minimum effort, maximum impact
Accessible design: Minimum effort, maximum impactAccessible design: Minimum effort, maximum impact
Accessible design: Minimum effort, maximum impactdawncurless
 
SOCIAL AND HISTORICAL CONTEXT - LFTVD.pptx
SOCIAL AND HISTORICAL CONTEXT - LFTVD.pptxSOCIAL AND HISTORICAL CONTEXT - LFTVD.pptx
SOCIAL AND HISTORICAL CONTEXT - LFTVD.pptxiammrhaywood
 
URLs and Routing in the Odoo 17 Website App
URLs and Routing in the Odoo 17 Website AppURLs and Routing in the Odoo 17 Website App
URLs and Routing in the Odoo 17 Website AppCeline George
 
Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991
Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991
Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991RKavithamani
 
Paris 2024 Olympic Geographies - an activity
Paris 2024 Olympic Geographies - an activityParis 2024 Olympic Geographies - an activity
Paris 2024 Olympic Geographies - an activityGeoBlogs
 
POINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptx
POINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptxPOINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptx
POINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptxSayali Powar
 
Web & Social Media Analytics Previous Year Question Paper.pdf
Web & Social Media Analytics Previous Year Question Paper.pdfWeb & Social Media Analytics Previous Year Question Paper.pdf
Web & Social Media Analytics Previous Year Question Paper.pdfJayanti Pande
 
Advanced Views - Calendar View in Odoo 17
Advanced Views - Calendar View in Odoo 17Advanced Views - Calendar View in Odoo 17
Advanced Views - Calendar View in Odoo 17Celine George
 
The Most Excellent Way | 1 Corinthians 13
The Most Excellent Way | 1 Corinthians 13The Most Excellent Way | 1 Corinthians 13
The Most Excellent Way | 1 Corinthians 13Steve Thomason
 

Kürzlich hochgeladen (20)

1029 - Danh muc Sach Giao Khoa 10 . pdf
1029 -  Danh muc Sach Giao Khoa 10 . pdf1029 -  Danh muc Sach Giao Khoa 10 . pdf
1029 - Danh muc Sach Giao Khoa 10 . pdf
 
Contemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptx
Contemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptxContemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptx
Contemporary philippine arts from the regions_PPT_Module_12 [Autosaved] (1).pptx
 
Q4-W6-Restating Informational Text Grade 3
Q4-W6-Restating Informational Text Grade 3Q4-W6-Restating Informational Text Grade 3
Q4-W6-Restating Informational Text Grade 3
 
Mattingly "AI & Prompt Design: The Basics of Prompt Design"
Mattingly "AI & Prompt Design: The Basics of Prompt Design"Mattingly "AI & Prompt Design: The Basics of Prompt Design"
Mattingly "AI & Prompt Design: The Basics of Prompt Design"
 
Z Score,T Score, Percential Rank and Box Plot Graph
Z Score,T Score, Percential Rank and Box Plot GraphZ Score,T Score, Percential Rank and Box Plot Graph
Z Score,T Score, Percential Rank and Box Plot Graph
 
BASLIQ CURRENT LOOKBOOK LOOKBOOK(1) (1).pdf
BASLIQ CURRENT LOOKBOOK  LOOKBOOK(1) (1).pdfBASLIQ CURRENT LOOKBOOK  LOOKBOOK(1) (1).pdf
BASLIQ CURRENT LOOKBOOK LOOKBOOK(1) (1).pdf
 
INDIA QUIZ 2024 RLAC DELHI UNIVERSITY.pptx
INDIA QUIZ 2024 RLAC DELHI UNIVERSITY.pptxINDIA QUIZ 2024 RLAC DELHI UNIVERSITY.pptx
INDIA QUIZ 2024 RLAC DELHI UNIVERSITY.pptx
 
microwave assisted reaction. General introduction
microwave assisted reaction. General introductionmicrowave assisted reaction. General introduction
microwave assisted reaction. General introduction
 
Grant Readiness 101 TechSoup and Remy Consulting
Grant Readiness 101 TechSoup and Remy ConsultingGrant Readiness 101 TechSoup and Remy Consulting
Grant Readiness 101 TechSoup and Remy Consulting
 
Accessible design: Minimum effort, maximum impact
Accessible design: Minimum effort, maximum impactAccessible design: Minimum effort, maximum impact
Accessible design: Minimum effort, maximum impact
 
SOCIAL AND HISTORICAL CONTEXT - LFTVD.pptx
SOCIAL AND HISTORICAL CONTEXT - LFTVD.pptxSOCIAL AND HISTORICAL CONTEXT - LFTVD.pptx
SOCIAL AND HISTORICAL CONTEXT - LFTVD.pptx
 
URLs and Routing in the Odoo 17 Website App
URLs and Routing in the Odoo 17 Website AppURLs and Routing in the Odoo 17 Website App
URLs and Routing in the Odoo 17 Website App
 
Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991
Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991
Industrial Policy - 1948, 1956, 1973, 1977, 1980, 1991
 
Staff of Color (SOC) Retention Efforts DDSD
Staff of Color (SOC) Retention Efforts DDSDStaff of Color (SOC) Retention Efforts DDSD
Staff of Color (SOC) Retention Efforts DDSD
 
Paris 2024 Olympic Geographies - an activity
Paris 2024 Olympic Geographies - an activityParis 2024 Olympic Geographies - an activity
Paris 2024 Olympic Geographies - an activity
 
POINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptx
POINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptxPOINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptx
POINT- BIOCHEMISTRY SEM 2 ENZYMES UNIT 5.pptx
 
Web & Social Media Analytics Previous Year Question Paper.pdf
Web & Social Media Analytics Previous Year Question Paper.pdfWeb & Social Media Analytics Previous Year Question Paper.pdf
Web & Social Media Analytics Previous Year Question Paper.pdf
 
Advanced Views - Calendar View in Odoo 17
Advanced Views - Calendar View in Odoo 17Advanced Views - Calendar View in Odoo 17
Advanced Views - Calendar View in Odoo 17
 
The Most Excellent Way | 1 Corinthians 13
The Most Excellent Way | 1 Corinthians 13The Most Excellent Way | 1 Corinthians 13
The Most Excellent Way | 1 Corinthians 13
 
Código Creativo y Arte de Software | Unidad 1
Código Creativo y Arte de Software | Unidad 1Código Creativo y Arte de Software | Unidad 1
Código Creativo y Arte de Software | Unidad 1
 

Truth, deduction, computation lecture f