VI. Church-Turing Thesis

Size: px
Start display at page:

Download "VI. Church-Turing Thesis"

Transcription

1 VI. Church-Turing Thesis Yuxi Fu BASICS, Shanghai Jiao Tong University

2 Fundamental Question How do computation models characterize the informal notion of effective computability? Computability Theory, by Y. Fu VI. Church-Turing Thesis 1 / 41

3 Fundamental Result Theorem. The set of functions definable in λ-calculus (Turing Machine Model, Unlimited Random Access Machine Model) is precisely the set of recursive functions. Proof. We have already showed that µ-definable λ-definable Turing definable URM-definable. We have to show that URM-definable µ-definable. Computability Theory, by Y. Fu VI. Church-Turing Thesis 2 / 41

4 Synopsis 1. Gödel Encoding 2. Kleene s Proof 3. Church-Turing Thesis Computability Theory, by Y. Fu VI. Church-Turing Thesis 3 / 41

5 Gödel Encoding Computability Theory, by Y. Fu VI. Church-Turing Thesis 4 / 41

6 Godel s Insight The set of syntactical objects of a formal system is denumerable. More importantly, every syntactical object can be coded up effectively by a number in such a way that a unique syntactical object can be recovered from the number. This is the crucial technique Gödel used in his proof of the Incompleteness Theorem. Computability Theory, by Y. Fu VI. Church-Turing Thesis 5 / 41

7 Enumeration An enumeration of a set X is a surjection g : ω X ; this is often represented by writing {x 0, x 1, x 2,...}. It is an enumeration without repetition if g is injective. Computability Theory, by Y. Fu VI. Church-Turing Thesis 6 / 41

8 Denumeration A set X is denumerable if there is a bijection f : X ω. (denumerate = denote + enumerate) Let X be a set of finite objects. Then X is effectively denumerable if there is a bijection f : X ω such that both f and f 1 are computable. Computability Theory, by Y. Fu VI. Church-Turing Thesis 7 / 41

9 Encoding Pair Fact. ω ω is effectively denumerable. Proof. A bijection π : ω ω ω is defined by π(m, n) π 1 (l) def = 2 m (2n + 1) 1, def = (π 1 (l), π 2 (l)), where π 1 (x) π 2 (x) def = (x + 1) 1, def = ((x + 1)/2 π 1(x) 1)/2. Computability Theory, by Y. Fu VI. Church-Turing Thesis 8 / 41

10 Encoding Tuple Fact. ω + ω + ω + is effectively denumerable. Proof. A bijection ζ : ω + ω + ω + ω is defined by ζ(m, n, q) ζ 1 (l) def = π(π(m 1, n 1), q 1), def = (π 1 (π 1 (l)) + 1, π 2 (π 1 (l)) + 1, π 2 (l) + 1). Computability Theory, by Y. Fu VI. Church-Turing Thesis 9 / 41

11 Encoding Finite String Fact. k>0 ωk is effectively denumerable. Proof. A bijection τ : k>0 ωk ω is defined by τ(a 1,..., a k ) def = 2 a a 1+a a 1+a 2 +a a 1+a 2 +a ,a k +k 1 1. Now given x it is easy to find b 1 < b 2 <... < b k such that 2 b b b b k = x + 1. It is then clear how to calculate a 1, a 2, a 3,..., a k. Details are next. Computability Theory, by Y. Fu VI. Church-Turing Thesis 10 / 41

12 Encoding Finite String A number x ω has a unique expression as x = α i 2 i, i=0 where α i is either 0 or 1 for all i The function α(i, x) = α i is primitive recursive: α(i, x) = rm(2, qt(2 i, x)). 2. The function l(x) = if x > 0 then k else 0 is primitive recursive: l(x) = i<x α(i, x). Computability Theory, by Y. Fu VI. Church-Turing Thesis 11 / 41

13 Encoding Finite String 3. If x > 0 then it has a unique expression as x = 2 b b b k, where 1 k and 0 b 1 < b 2 <... < b k. The function b(i, x) = if (x > 0) (1 i l(x)) then b i else 0 is primitive recursive: { ( ) µy<x b(i, x) = k y α(k, x) = i, if (x > 0) (1 i l(x)); 0, otherwise. Computability Theory, by Y. Fu VI. Church-Turing Thesis 12 / 41

14 Encoding Finite String 4. If x > 0 then it has a unique expression as x = 2 a a 1+a a l +a a k +k 1. The function a(i, x) = a i is primitive recursive: a(i, x) = b(i, x), if i = 0 or i = 1, a(i + 1, x) = (b(i + 1, x) b(i, x)) 1, if i 1. We conclude that a 1, a 2, a 3,..., a k can be calculated by primitive recursive functions. Computability Theory, by Y. Fu VI. Church-Turing Thesis 13 / 41

15 Encoding Programme Let I be the set of all instructions. Let P be the set of all programs. The objects in I, and P as well, are finite objects. Computability Theory, by Y. Fu VI. Church-Turing Thesis 14 / 41

16 Encoding Programme Theorem. I is effectively denumerable. Proof. The bijection β : I ω is defined as follows: β(z(n)) = 4(n 1), β(s(n)) = 4(n 1) + 1, β(t (m, n)) = 4π(m 1, n 1) + 2, β(j(m, n, q)) = 4ζ(m, n, q) + 3. The converse β 1 is easy. Computability Theory, by Y. Fu VI. Church-Turing Thesis 15 / 41

17 Encoding Programme Theorem. P is effectively denumerable. Proof. The bijection γ : P ω is defined as follows: assuming P = I 1,..., I s. The converse γ 1 is obvious. γ(p) = τ(β(i 1 ),..., β(i s )), Computability Theory, by Y. Fu VI. Church-Turing Thesis 16 / 41

18 Gödel Number of Programme The value γ(p) is called the Gödel number of P. P n = the programme with Godel index n = γ 1 (n) We shall fix this particular encoding function γ throughout. Computability Theory, by Y. Fu VI. Church-Turing Thesis 17 / 41

19 Example Let P be the program T (1, 3), S(4), Z(6). β(t (1, 3)) = 18, β(s(4)) = 13, β(z(6)) = 20. γ(p) = Computability Theory, by Y. Fu VI. Church-Turing Thesis 18 / 41

20 Example Consider P = β(i 1 ) = 4 + 1, β(i 2 ) = 4π(1, 0) + 2. So P 4127 is S(2); T (2, 1). Computability Theory, by Y. Fu VI. Church-Turing Thesis 19 / 41

21 Kleene s Proof Computability Theory, by Y. Fu VI. Church-Turing Thesis 20 / 41

22 Kleene demonstrated how to prove that machine computable functions are recursive functions. Computability Theory, by Y. Fu VI. Church-Turing Thesis 21 / 41

23 Proof in Detail The state of the computation of the program P e ( x) can be described by a configuration and an instruction number. A state can be coded up by the number σ = π(c, j), where c is the configuration that codes up the current values in the registers c = 2 r 1 3 r 2... = i 1 p r i i, and j is the next instruction number. Computability Theory, by Y. Fu VI. Church-Turing Thesis 22 / 41

24 Proof in Detail To describe the changes of the states of P e ( x), we introduce three (n + 2)-ary functions: c n (e, x, t) = the configuration after t steps of P e ( x), j n (e, x, t) = the number of the next instruction after t steps of P e ( x) (it is 0 if P e ( x) stops in t or less steps), σ n (e, x, t) = π(c n (e, x, t), j n (e, x, t)). If σ n is primitive recursive, then c n, j n are primitive recursive. Computability Theory, by Y. Fu VI. Church-Turing Thesis 23 / 41

25 Proof in Detail If the computation of P e ( x) stops, it does so in µt(j n (e, x, t) = 0) steps. Then the final configuration is c n (e, x, µt(j n (e, x, t) = 0)). We conclude that the value of the computation P e ( x) is (c n (e, x, µt(j n (e, x, t) = 0))) 1. Computability Theory, by Y. Fu VI. Church-Turing Thesis 24 / 41

26 Proof in Detail The function σ n can be defined as follows: σ n (e, x, 0) = π(2 x 1 3 x 2... pn xn, 1), σ n (e, x, t + 1) = π(config(e, σ n (e, x, t)), next(e, σ n (e, x, t))), where config(e, π(c, j)) is the configuration after t + 1 steps; next(e, π(c, j)) is the new number after t + 1 steps. Computability Theory, by Y. Fu VI. Church-Turing Thesis 25 / 41

27 Proof in Detail ln(e) = the number of instructions in P e ; gn(e, j) = { the code of Ij in P e, if 1 j ln(e), 0, otherwise. Both functions are primitive recursive since ln(e) = l(e + 1), gn(e, j) = a(j, e + 1). Computability Theory, by Y. Fu VI. Church-Turing Thesis 26 / 41

28 Proof in Detail u(z) = m whenever z = β(z(m)) or z = β(s(m)): u(z) = qt(4, z) + 1. u 1 (z) = m 1 and u 2 (z) = m 2 whenever z = β(t (m 1, m 2 )): u 1 (z) = π 1 (qt(4, z)) + 1, u 2 (z) = π 2 (qt(4, z)) + 1. v 1 (z) = m 1 and v 2 (z) = m 2 and v 3 (z) = q if z = β(j(m 1, m 2, q)): v 1 (z) = π 1 (π 1 (qt(4, z))) + 1, v 2 (z) = π 2 (π 1 (qt(4, z))) + 1, v 3 (z) = π 2 (qt(4, z)) + 1. Computability Theory, by Y. Fu VI. Church-Turing Thesis 27 / 41

29 Proof in Detail The change in the configuration c effected by instruction Z(m): zero(c, m) = qt(p m (c)m, c). The change in the configuration c effected by instruction S(m): succ(c, m) = p m c. The change in the configuration c effected by instruction T (m, n): tran(c, m, n) = qt(p (c)n n, p n (c)m c). Computability Theory, by Y. Fu VI. Church-Turing Thesis 28 / 41

30 Proof in Detail The following function ch(c, z) = the resulting configuration when the configuration c is operated on by the instruction with code number z. is primitive recursive since zero(c, u(z)), if rm(4, z) = 0, succ(c, u(z)), if rm(4, z) = 1, ch(c, z) = tran(c, u 1 (z), u 2 (z)), if rm(4, z) = 2, c, if rm(4, z) = 3. Computability Theory, by Y. Fu VI. Church-Turing Thesis 29 / 41

31 Proof in Detail The following function the number j of the next instruction when the configuration c is operated if j > 0, v(c, j, z) = on by the jth instruction with code z, 0, if j = 0. is primitive recursive since j + 1, if rm(4, z) 3, v(c, j, z) = j + 1, v 3 (z), if rm(4, z) = 3 (c) v1 (z) (c) v2 (z), if rm(4, z) = 3 (c) v1 (z) = (c) v2 (z). Computability Theory, by Y. Fu VI. Church-Turing Thesis 30 / 41

32 Proof in Detail config(e, σ) = { ch(π1 (σ), gn(e, π 2 (σ))), if 1 π 2 (σ) ln(e), π 1 (σ), otherwise. next(e, σ) = { v(π1 (σ), π 2 (σ), gn(e, π 2 (σ))), if 1 π 2 (σ) ln(e), 0, otherwise. Computability Theory, by Y. Fu VI. Church-Turing Thesis 31 / 41

33 Proof in Detail We conclude that the functions c n, j n, σ n are primitive recursive. Computability Theory, by Y. Fu VI. Church-Turing Thesis 32 / 41

34 Further Constructions For each n 1, the following predicates are primitive recursive: 1. S n (e, x, y, t) def = P e ( x) y in t or fewer steps. 2. H n (e, x, t) def = P e ( x) in t or fewer steps. They are defined by S n (e, x, y, t) H n (e, x, t) def = j n (e, x, t) = 0 (c n (e, x, t)) 1 = y, def = j n (e, x, t) = 0. Computability Theory, by Y. Fu VI. Church-Turing Thesis 33 / 41

35 Kleene s Normal Form Theorem Let φ (n) e denote the n-ary function computed by P e. Theorem. (Kleene) There is a primitive recursive function U(x) and, for each n 1, a primitive recursive predicate T n (e, x, z) such that 1. φ (n) e ( x) is defined if and only if z.t n (e, x, z). 2. φ (n) e ( x) U(µzT n (e, x, z)). Proof. (1) T n (e, x, z) = S n (e, x, π 1 (z), π 2 (z)). (2) Let U(x) = π 1 (x). Then φ (n) e ( x) U(µz.T n (e, x, z)). Computability Theory, by Y. Fu VI. Church-Turing Thesis 34 / 41

36 Every computable function can be obtained from a primitive recursive function by using at most one application of the µ-operator in a standard manner. Computability Theory, by Y. Fu VI. Church-Turing Thesis 35 / 41

37 Church-Turing Thesis Computability Theory, by Y. Fu VI. Church-Turing Thesis 36 / 41

38 Church-Turing Thesis. The functions definable in all computation models are the same. They are precisely the computable functions. Church believed that all computable functions are λ-definable. Kleene termed it Church Thesis. Gödel accepted it only after he saw Turing s equivalence proof. Church-Turing Thesis is now universally accepted. Computability Theory, by Y. Fu VI. Church-Turing Thesis 37 / 41

39 Computable Function Let C be the set of all computable functions. Let C n be the set of all n-ary computable functions. Computability Theory, by Y. Fu VI. Church-Turing Thesis 38 / 41

40 Power of Church-Turing Thesis Noone has come up with a computable function that is not in C. When you are convincing people of your model of computation, you are constructing an effective translation from your model to a well-known computation model. Computability Theory, by Y. Fu VI. Church-Turing Thesis 39 / 41

41 Making Use of Church-Turing Thesis Church-Turing Thesis allows us to give an informal argument for the computability of a function. We will make use of CTT in this way without explicitly defining it. Computability Theory, by Y. Fu VI. Church-Turing Thesis 40 / 41

42 Comment on Church-Turing Thesis CTT and Physical Implementation Deterministic Turing Machines are physically implementable. This is the well-known von Neumann Architecture. Are quantum computers physically implementable? Can a quantum computer compute more or more efficiently? CTT, is it a Law of Nature or a Wisdom of Human? Computability Theory, by Y. Fu VI. Church-Turing Thesis 41 / 41

IV. Turing Machine. Yuxi Fu. BASICS, Shanghai Jiao Tong University

IV. Turing Machine. Yuxi Fu. BASICS, Shanghai Jiao Tong University IV. Turing Machine Yuxi Fu BASICS, Shanghai Jiao Tong University Alan Turing Alan Turing (23Jun.1912-7Jun.1954), an English student of Church, introduced a machine model for effective calculation in On

More information

Theory of Computation

Theory of Computation Thomas Zeugmann Hokkaido University Laboratory for Algorithmics http://www-alg.ist.hokudai.ac.jp/ thomas/toc/ Lecture 12: Turing Machines Turing Machines I After having dealt with partial recursive functions,

More information

Computability. Part II. 6 Models of Computation. Register Machines

Computability. Part II. 6 Models of Computation. Register Machines Part II Computability 6 Models of Computation What is a computable function? Our modern intuition is that a function f : N N is computable if there is a a program in a computer language like C ++, PASCAL

More information

Automata Theory. Definition. Computational Complexity Theory. Computability Theory

Automata Theory. Definition. Computational Complexity Theory. Computability Theory Outline THEORY OF COMPUTATION CS363, SJTU What is Theory of Computation? History of Computation Branches and Development Xiaofeng Gao Dept. of Computer Science Shanghai Jiao Tong University 2 The Essential

More information

Tape encoding of lists of numbers

Tape encoding of lists of numbers L7 74 We ve seen that a Turing machine s computation can be implemented by a register machine. The converse holds: the computation of a register machine can be implemented by a Turing machine. To make

More information

The Turing machine model of computation

The Turing machine model of computation The Turing machine model of computation For most of the remainder of the course we will study the Turing machine model of computation, named after Alan Turing (1912 1954) who proposed the model in 1936.

More information

Introduction to Turing Machines

Introduction to Turing Machines Introduction to Turing Machines Deepak D Souza Department of Computer Science and Automation Indian Institute of Science, Bangalore. 12 November 2015 Outline 1 Turing Machines 2 Formal definitions 3 Computability

More information

Computability. Part II. 6 Models of Computation. Register Machines

Computability. Part II. 6 Models of Computation. Register Machines Part II Computability 6 Models of Computation What is a computable function? Our modern intuition is that a function f : N N is computable if there is a a program in a computer language like C ++, PASCAL

More information

Predicate Logic - Undecidability

Predicate Logic - Undecidability CS402, Spring 2016 Undecidable Problems Does the following program halts? (1) N : n, total, x, y, z (2) n GetUserInput() (3) total 3 (4) while true (5) for x 1 to total 2 (6) for y 1 to total x 1 (7) z

More information

FINAL EXAM FOR PHIL 152 MICHAEL BEESON

FINAL EXAM FOR PHIL 152 MICHAEL BEESON FINAL EXAM FOR PHIL 152 MICHAEL BEESON Directions. This is an open-book, open-notes, open-homework. You can even search the Internet, but all the answers can be found in the lecture notes and homework

More information

23.1 Gödel Numberings and Diagonalization

23.1 Gödel Numberings and Diagonalization Applied Logic Lecture 23: Unsolvable Problems in Logic CS 4860 Spring 2009 Tuesday, April 14, 2009 The fact that Peano Arithmetic is expressive enough to represent all computable functions means that some

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

XII. Elementary Function

XII. Elementary Function XII. Elementary Function Yuxi Fu BASICS, Shanghai Jiao Tong University What is the class of arithmetic functions we use in mathematics? Computability Theory, by Y. Fu XII. Elementary Function 1 / 17 Definition

More information

Decidability. William Chan

Decidability. William Chan Decidability William Chan Preface : In 1928, David Hilbert gave a challenge known as the Entscheidungsproblem, which is German for Decision Problem. Hilbert s problem asked for some purely mechanical procedure

More information

16.1 Countability. CS125 Lecture 16 Fall 2014

16.1 Countability. CS125 Lecture 16 Fall 2014 CS125 Lecture 16 Fall 2014 16.1 Countability Proving the non-existence of algorithms for computational problems can be very difficult. Indeed, we do not know how to prove P NP. So a natural question is

More information

Lecture notes on Turing machines

Lecture notes on Turing machines Lecture notes on Turing machines Ivano Ciardelli 1 Introduction Turing machines, introduced by Alan Turing in 1936, are one of the earliest and perhaps the best known model of computation. The importance

More information

Turing Machines A Turing Machine is a 7-tuple, (Q, Σ, Γ, δ, q0, qaccept, qreject), where Q, Σ, Γ are all finite

Turing Machines A Turing Machine is a 7-tuple, (Q, Σ, Γ, δ, q0, qaccept, qreject), where Q, Σ, Γ are all finite The Church-Turing Thesis CS60001: Foundations of Computing Science Professor, Dept. of Computer Sc. & Engg., Turing Machines A Turing Machine is a 7-tuple, (Q, Σ, Γ, δ, q 0, q accept, q reject ), where

More information

CS 275 Automata and Formal Language Theory

CS 275 Automata and Formal Language Theory CS 275 Automata and Formal Language Theory Course Notes Part III: Limits of Computation Chapter III.1: Introduction Anton Setzer http://www.cs.swan.ac.uk/ csetzer/lectures/ automataformallanguage/current/index.html

More information

Computability Theory. CS215, Lecture 6,

Computability Theory. CS215, Lecture 6, Computability Theory CS215, Lecture 6, 2000 1 The Birth of Turing Machines At the end of the 19th century, Gottlob Frege conjectured that mathematics could be built from fundamental logic In 1900 David

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

Computation. Some history...

Computation. Some history... Computation Motivating questions: What does computation mean? What are the similarities and differences between computation in computers and in natural systems? What are the limits of computation? Are

More information

Turing Machines (TM) The Turing machine is the ultimate model of computation.

Turing Machines (TM) The Turing machine is the ultimate model of computation. TURING MACHINES Turing Machines (TM) The Turing machine is the ultimate model of computation. Alan Turing (92 954), British mathematician/engineer and one of the most influential scientists of the last

More information

XI. Computational Complexity

XI. Computational Complexity XI. Computational Complexity Yuxi Fu BASICS, Shanghai Jiao Tong University Mathematic proofs, like computations, are energy consuming business. There are mathematical theorems, and computational tasks,

More information

CS 275 Automata and Formal Language Theory

CS 275 Automata and Formal Language Theory CS 275 Automata and Formal Language Theory Course Notes Part III: Limits of Computation Chapt. III.1: Introduction Anton Setzer http://www.cs.swan.ac.uk/ csetzer/lectures/ automataformallanguage/current/index.html

More information

Opleiding Informatica

Opleiding Informatica Opleiding Informatica Tape-quantifying Turing machines in the arithmetical hierarchy Simon Heijungs Supervisors: H.J. Hoogeboom & R. van Vliet BACHELOR THESIS Leiden Institute of Advanced Computer Science

More information

(a) Definition of TMs. First Problem of URMs

(a) Definition of TMs. First Problem of URMs Sec. 4: Turing Machines First Problem of URMs (a) Definition of the Turing Machine. (b) URM computable functions are Turing computable. (c) Undecidability of the Turing Halting Problem That incrementing

More information

The Church-Turing Thesis and Relative Recursion

The Church-Turing Thesis and Relative Recursion The Church-Turing Thesis and Relative Recursion Yiannis N. Moschovakis UCLA and University of Athens Amsterdam, September 7, 2012 The Church -Turing Thesis (1936) in a contemporary version: CT : For every

More information

Examples of Unlimited Register Machine programs for Turingcomputable

Examples of Unlimited Register Machine programs for Turingcomputable Examples of Unlimited Register Machine programs for Turingcomputable functions 18 February 2012 at 13:01 Public It will be a matter of interest for me over the next few months to formulate (and collect)

More information

Turing machines and linear bounded automata

Turing machines and linear bounded automata and linear bounded automata Informatics 2A: Lecture 29 John Longley School of Informatics University of Edinburgh jrl@inf.ed.ac.uk 27 November 2015 1 / 15 The Chomsky hierarchy: summary Level Language

More information

TOWARD A THEORY OF INTRINSIC COMPUTABILITY

TOWARD A THEORY OF INTRINSIC COMPUTABILITY latest update February 28, 2005 TOWARD A THEORY OF INTRINSIC COMPUTABILITY MARCO GIUNTI Università di Cagliari, Italy Abstract: This paper investigates the foundations of the view that (i) computation

More information

Complexity 6: AIT. Outline. Dusko Pavlovic. Kolmogorov. Solomonoff. Chaitin: The number of wisdom RHUL Spring Complexity 6: AIT.

Complexity 6: AIT. Outline. Dusko Pavlovic. Kolmogorov. Solomonoff. Chaitin: The number of wisdom RHUL Spring Complexity 6: AIT. Outline Complexity Theory Part 6: did we achieve? Algorithmic information and logical depth : Algorithmic information : Algorithmic probability : The number of wisdom RHUL Spring 2012 : Logical depth Outline

More information

CSCE 551: Chin-Tser Huang. University of South Carolina

CSCE 551: Chin-Tser Huang. University of South Carolina CSCE 551: Theory of Computation Chin-Tser Huang huangct@cse.sc.edu University of South Carolina Church-Turing Thesis The definition of the algorithm came in the 1936 papers of Alonzo Church h and Alan

More information

Part I: Definitions and Properties

Part I: Definitions and Properties Turing Machines Part I: Definitions and Properties Finite State Automata Deterministic Automata (DFSA) M = {Q, Σ, δ, q 0, F} -- Σ = Symbols -- Q = States -- q 0 = Initial State -- F = Accepting States

More information

COMP-330 Theory of Computation. Fall Prof. Claude Crépeau. Lec. 14 : Turing Machines

COMP-330 Theory of Computation. Fall Prof. Claude Crépeau. Lec. 14 : Turing Machines COMP-330 Theory of Computation Fall 2012 -- Prof. Claude Crépeau Lec. 14 : Turing Machines 1 COMP 330 Fall 2012: Lectures Schedule 1. Introduction 1.5. Some basic mathematics 2. Deterministic finite automata

More information

The complexity of recursive constraint satisfaction problems.

The complexity of recursive constraint satisfaction problems. The complexity of recursive constraint satisfaction problems. Victor W. Marek Department of Computer Science University of Kentucky Lexington, KY 40506, USA marek@cs.uky.edu Jeffrey B. Remmel Department

More information

What are the recursion theoretic properties of a set of axioms? Understanding a paper by William Craig Armando B. Matos

What are the recursion theoretic properties of a set of axioms? Understanding a paper by William Craig Armando B. Matos What are the recursion theoretic properties of a set of axioms? Understanding a paper by William Craig Armando B. Matos armandobcm@yahoo.com February 5, 2014 Abstract This note is for personal use. It

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

Cogito ergo sum non machina!

Cogito ergo sum non machina! Cogito ergo sum non machina! About Gödel s First Incompleteness Theorem and Turing machines. Ricardo Pereira Tassinari 1 Philosophy Department of State University of São Paulo - UNESP - Campus Marília

More information

Large Numbers, Busy Beavers, Noncomputability and Incompleteness

Large Numbers, Busy Beavers, Noncomputability and Incompleteness Large Numbers, Busy Beavers, Noncomputability and Incompleteness Food For Thought November 1, 2007 Sam Buss Department of Mathematics U.C. San Diego PART I Large Numbers, Busy Beavers, and Undecidability

More information

COMP-330 Theory of Computation. Fall Prof. Claude Crépeau. Lec. 16 : Turing Machines

COMP-330 Theory of Computation. Fall Prof. Claude Crépeau. Lec. 16 : Turing Machines COMP-330 Theory of Computation Fall 2017 -- Prof. Claude Crépeau Lec. 16 : Turing Machines COMP 330 Fall 2017: Lectures Schedule 1-2. Introduction 1.5. Some basic mathematics 2-3. Deterministic finite

More information

HUMAN COMPUTATION FROM A STRICTLY DYNAMICAL POINT OF VIEW

HUMAN COMPUTATION FROM A STRICTLY DYNAMICAL POINT OF VIEW Cagliari Colloquium on the Extended Mind, Dynamicism, and Computation. Cagliari, June 10, 2013 HUMAN COMPUTATION FROM A STRICTLY DYNAMICAL POINT OF VIEW Marco Giunti - ALOPHIS, Università di Cagliari SUMMARY

More information

Turing machines and linear bounded automata

Turing machines and linear bounded automata and linear bounded automata Informatics 2A: Lecture 30 John Longley School of Informatics University of Edinburgh jrl@inf.ed.ac.uk 25 November 2016 1 / 17 The Chomsky hierarchy: summary Level Language

More information

Decidable Languages - relationship with other classes.

Decidable Languages - relationship with other classes. CSE2001, Fall 2006 1 Last time we saw some examples of decidable languages (or, solvable problems). Today we will start by looking at the relationship between the decidable languages, and the regular and

More information

Theory of Computation Lecture Notes. Problems and Algorithms. Class Information

Theory of Computation Lecture Notes. Problems and Algorithms. Class Information Theory of Computation Lecture Notes Prof. Yuh-Dauh Lyuu Dept. Computer Science & Information Engineering and Department of Finance National Taiwan University Problems and Algorithms c 2004 Prof. Yuh-Dauh

More information

Linear-time Temporal Logic

Linear-time Temporal Logic Linear-time Temporal Logic Pedro Cabalar Department of Computer Science University of Corunna, SPAIN cabalar@udc.es 2015/2016 P. Cabalar ( Department Linear oftemporal Computer Logic Science University

More information

Recap (1) 1. Automata, grammars and other formalisms can be considered as mechanical devices to solve mathematical problems

Recap (1) 1. Automata, grammars and other formalisms can be considered as mechanical devices to solve mathematical problems Computability 1 Recap (1) 1. Automata, grammars and other formalisms can be considered as mechanical devices to solve mathematical problems Mathematical problems are often the formalization of some practical

More information

7.1 The Origin of Computer Science

7.1 The Origin of Computer Science CS125 Lecture 7 Fall 2016 7.1 The Origin of Computer Science Alan Mathison Turing (1912 1954) turing.jpg 170!201 pixels On Computable Numbers, with an Application to the Entscheidungsproblem 1936 1936:

More information

A version of for which ZFC can not predict a single bit Robert M. Solovay May 16, Introduction In [2], Chaitin introd

A version of for which ZFC can not predict a single bit Robert M. Solovay May 16, Introduction In [2], Chaitin introd CDMTCS Research Report Series A Version of for which ZFC can not Predict a Single Bit Robert M. Solovay University of California at Berkeley CDMTCS-104 May 1999 Centre for Discrete Mathematics and Theoretical

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

Q = Set of states, IE661: Scheduling Theory (Fall 2003) Primer to Complexity Theory Satyaki Ghosh Dastidar

Q = Set of states, IE661: Scheduling Theory (Fall 2003) Primer to Complexity Theory Satyaki Ghosh Dastidar IE661: Scheduling Theory (Fall 2003) Primer to Complexity Theory Satyaki Ghosh Dastidar Turing Machine A Turing machine is an abstract representation of a computing device. It consists of a read/write

More information

CSE 105 THEORY OF COMPUTATION

CSE 105 THEORY OF COMPUTATION CSE 105 THEORY OF COMPUTATION Spring 2016 http://cseweb.ucsd.edu/classes/sp16/cse105-ab/ Today's learning goals Sipser Ch 3.3, 4.1 State and use the Church-Turing thesis. Give examples of decidable problems.

More information

Turing machines and computable functions

Turing machines and computable functions Turing machines and computable functions In this chapter we address the question: how can we define the class of discrete functions that are computable? Probably, most of you are familiar with a few programming

More information

Primitive recursive functions: decidability problems

Primitive recursive functions: decidability problems Primitive recursive functions: decidability problems Armando B. Matos October 24, 2014 Abstract Although every primitive recursive (PR) function is total, many problems related to PR functions are undecidable.

More information

Turing Machine Variants

Turing Machine Variants CS311 Computational Structures Turing Machine Variants Lecture 12 Andrew Black Andrew Tolmach 1 The Church-Turing Thesis The problems that can be decided by an algorithm are exactly those that can be decided

More information

Peano Arithmetic. CSC 438F/2404F Notes (S. Cook) Fall, Goals Now

Peano Arithmetic. CSC 438F/2404F Notes (S. Cook) Fall, Goals Now CSC 438F/2404F Notes (S. Cook) Fall, 2008 Peano Arithmetic Goals Now 1) We will introduce a standard set of axioms for the language L A. The theory generated by these axioms is denoted PA and called Peano

More information

An Intuitively Complete Analysis of Gödel s Incompleteness

An Intuitively Complete Analysis of Gödel s Incompleteness An Intuitively Complete Analysis of Gödel s Incompleteness JASON W. STEINMETZ (Self-funded) A detailed and rigorous analysis of Gödel s proof of his first incompleteness theorem is presented. The purpose

More information

Turing machines and linear bounded automata

Turing machines and linear bounded automata and linear bounded automata Informatics 2A: Lecture 29 John Longley School of Informatics University of Edinburgh jrl@inf.ed.ac.uk 25 November, 2011 1 / 13 1 The Chomsky hierarchy: summary 2 3 4 2 / 13

More information

TURING MAHINES

TURING MAHINES 15-453 TURING MAHINES TURING MACHINE FINITE STATE q 10 CONTROL AI N P U T INFINITE TAPE read write move 0 0, R, R q accept, R q reject 0 0, R 0 0, R, L read write move 0 0, R, R q accept, R 0 0, R 0 0,

More information

FORMAL LANGUAGES, AUTOMATA AND COMPUTABILITY

FORMAL LANGUAGES, AUTOMATA AND COMPUTABILITY 15-453 FORMAL LANGUAGES, AUTOMATA AND COMPUTABILITY Chomsky Normal Form and TURING MACHINES TUESDAY Feb 4 CHOMSKY NORMAL FORM A context-free grammar is in Chomsky normal form if every rule is of the form:

More information

COMP/MATH 300 Topics for Spring 2017 June 5, Review and Regular Languages

COMP/MATH 300 Topics for Spring 2017 June 5, Review and Regular Languages COMP/MATH 300 Topics for Spring 2017 June 5, 2017 Review and Regular Languages Exam I I. Introductory and review information from Chapter 0 II. Problems and Languages A. Computable problems can be expressed

More information

cse303 ELEMENTS OF THE THEORY OF COMPUTATION Professor Anita Wasilewska

cse303 ELEMENTS OF THE THEORY OF COMPUTATION Professor Anita Wasilewska cse303 ELEMENTS OF THE THEORY OF COMPUTATION Professor Anita Wasilewska LECTURE 13 CHAPTER 4 TURING MACHINES 1. The definition of Turing machine 2. Computing with Turing machines 3. Extensions of Turing

More information

The purpose here is to classify computational problems according to their complexity. For that purpose we need first to agree on a computational

The purpose here is to classify computational problems according to their complexity. For that purpose we need first to agree on a computational 1 The purpose here is to classify computational problems according to their complexity. For that purpose we need first to agree on a computational model. We'll remind you what a Turing machine is --- you

More information

Theory of Computation

Theory of Computation Thomas Zeugmann Hokkaido University Laboratory for Algorithmics http://www-alg.ist.hokudai.ac.jp/ thomas/toc/ Lecture 14: Applications of PCP Goal of this Lecture Our goal is to present some typical undecidability

More information

Limits of Computability

Limits of Computability Limits of Computability Wolfgang Schreiner Wolfgang.Schreiner@risc.jku.at Research Institute for Symbolic Computation (RISC) Johannes Kepler University, Linz, Austria http://www.risc.jku.at Wolfgang Schreiner

More information

Chomsky Normal Form and TURING MACHINES. TUESDAY Feb 4

Chomsky Normal Form and TURING MACHINES. TUESDAY Feb 4 Chomsky Normal Form and TURING MACHINES TUESDAY Feb 4 CHOMSKY NORMAL FORM A context-free grammar is in Chomsky normal form if every rule is of the form: A BC A a S ε B and C aren t start variables a is

More information

1 Deterministic Turing Machines

1 Deterministic Turing Machines Time and Space Classes Exposition by William Gasarch 1 Deterministic Turing Machines Turing machines are a model of computation. It is believed that anything that can be computed can be computed by a Turing

More information

Fundamentals of Computer Science

Fundamentals of Computer Science Fundamentals of Computer Science Chapter 8: Turing machines Henrik Björklund Umeå University February 17, 2014 The power of automata Finite automata have only finite memory. They recognize the regular

More information

X-machines - a computational model framework.

X-machines - a computational model framework. Chapter 2. X-machines - a computational model framework. This chapter has three aims: To examine the main existing computational models and assess their computational power. To present the X-machines as

More information

Review of unsolvability

Review of unsolvability Review of unsolvability L L H To prove unsolvability: show a reduction. To prove solvability: show an algorithm. Unsolvable problems (main insight) Turing machine (algorithm) properties Pattern matching

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

König s Lemma and Kleene Tree

König s Lemma and Kleene Tree König s Lemma and Kleene Tree Andrej Bauer May 3, 2006 Abstract I present a basic result about Cantor space in the context of computability theory: the computable Cantor space is computably non-compact.

More information

α-recursion Theory and Ordinal Computability

α-recursion Theory and Ordinal Computability α-recursion Theory and Ordinal Computability by Peter Koepke University of Bonn 1 3. 2. 2007 Abstract Motivated by a talk of S. D. Friedman at BIWOC we show that the α-recursive and α-recursively enumerable

More information

Chapter 11 Evolution by Permutation

Chapter 11 Evolution by Permutation Chapter 11 Evolution by Permutation In what follows a very brief account of reversible evolution and, in particular, reversible computation by permutation will be presented We shall follow Mermin s account

More information

Elementary Recursive Function Theory

Elementary Recursive Function Theory Chapter 9 Elementary Recursive Function Theory 9.1 Acceptable Indexings In a previous Section, we have exhibited a specific indexing of the partial computable functions by encoding the RAM programs. Using

More information

Great Theoretical Ideas in Computer Science. Lecture 7: Introduction to Computational Complexity

Great Theoretical Ideas in Computer Science. Lecture 7: Introduction to Computational Complexity 15-251 Great Theoretical Ideas in Computer Science Lecture 7: Introduction to Computational Complexity September 20th, 2016 What have we done so far? What will we do next? What have we done so far? > Introduction

More information

(9-5) Def Turing machine, Turing computable functions. (9-7) Def Primitive recursive functions, Primitive recursive implies Turing computable.

(9-5) Def Turing machine, Turing computable functions. (9-7) Def Primitive recursive functions, Primitive recursive implies Turing computable. (9-5) Def Turing machine, Turing computable functions. A.Miller M773 Computability Theory Fall 2001 (9-7) Def Primitive recursive functions, Primitive recursive implies Turing computable. 1. Prove f(n)

More information

ELEMENTS IN MATHEMATICS FOR INFORMATION SCIENCE NO.6 TURING MACHINE AND COMPUTABILITY. Tatsuya Hagino

ELEMENTS IN MATHEMATICS FOR INFORMATION SCIENCE NO.6 TURING MACHINE AND COMPUTABILITY. Tatsuya Hagino 1 ELEMENTS IN MATHEMATICS FOR INFORMATION SCIENCE NO.6 TURING MACHINE AND COMPUTABILITY Tatsuya Hagino hagino@sfc.keio.ac.jp 2 So far Computation flow chart program while program recursive function primitive

More information

Computability Theory for Neuroscience

Computability Theory for Neuroscience Computability Theory for Neuroscience by Doug Rubino Abstract Neuronal circuits are ubiquitously held to be the substrate of computation in the brain, information processing in single neurons is though

More information

Turing Machines and the Church-Turing Thesis

Turing Machines and the Church-Turing Thesis CSE2001, Fall 2006 1 Turing Machines and the Church-Turing Thesis Today our goal is to show that Turing Machines are powerful enough to model digital computers, and to see discuss some evidence for the

More information

5. Peano arithmetic and Gödel s incompleteness theorem

5. Peano arithmetic and Gödel s incompleteness theorem 5. Peano arithmetic and Gödel s incompleteness theorem In this chapter we give the proof of Gödel s incompleteness theorem, modulo technical details treated in subsequent chapters. The incompleteness theorem

More information

Computability Theory

Computability Theory Computability Theory Cristian S. Calude May 2012 Computability Theory 1 / 1 Bibliography M. Sipser. Introduction to the Theory of Computation, PWS 1997. (textbook) Computability Theory 2 / 1 Supplementary

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

Expansions with P = NP. Christine Gaßner Greifswald

Expansions with P = NP. Christine Gaßner Greifswald Expansions with P = NP Greifswald Expansions with P = NP 1. 2. The complexity classes P Σ, NP Σ, DEC Σ 3. Why is it difficult to find an R with P ΣR = NP ΣR? 4. How to construct a relation R such that

More information

From Constructibility and Absoluteness to Computability and Domain Independence

From Constructibility and Absoluteness to Computability and Domain Independence From Constructibility and Absoluteness to Computability and Domain Independence Arnon Avron School of Computer Science Tel Aviv University, Tel Aviv 69978, Israel aa@math.tau.ac.il Abstract. Gödel s main

More information

Ma/CS 117c Handout # 5 P vs. NP

Ma/CS 117c Handout # 5 P vs. NP Ma/CS 117c Handout # 5 P vs. NP We consider the possible relationships among the classes P, NP, and co-np. First we consider properties of the class of NP-complete problems, as opposed to those which are

More information

highlights proof by contradiction what about the real numbers?

highlights proof by contradiction what about the real numbers? CSE 311: Foundations of Computing Fall 2013 Lecture 27: Turing machines and decidability highlights Cardinality A set S is countableiffwe can writeit as S={s 1, s 2, s 3,...} indexed by N Set of rationals

More information

7. The Recursion Theorem

7. The Recursion Theorem 7. The Recursion Theorem Main result in this section: Kleene s Recursion Theorem. Recursive functions are closed under a very general form of recursion. For proof we will use the S-m-n-theorem. Used in

More information

Computable Functions

Computable Functions Computable Functions Part I: Non Computable Functions Computable and Partially Computable Functions Computable Function Exists a Turing Machine M -- M Halts on All Input -- M(x) = f (x) Partially Computable

More information

Lecture 13: Foundations of Math and Kolmogorov Complexity

Lecture 13: Foundations of Math and Kolmogorov Complexity 6.045 Lecture 13: Foundations of Math and Kolmogorov Complexity 1 Self-Reference and the Recursion Theorem 2 Lemma: There is a computable function q : Σ* Σ* such that for every string w, q(w) is the description

More information

COMPUTABILITY. An introduction to recursive function theory NIGEL CUTLAND CAMBRIDGE UNIVERSITY PRESS

COMPUTABILITY. An introduction to recursive function theory NIGEL CUTLAND CAMBRIDGE UNIVERSITY PRESS COMPUTABILITY COMPUTABILITY An introduction to recursive function theory NIGEL CUTLAND Department of Pure Mathematics, University of Hull CAMBRIDGE UNIVERSITY PRESS Cambridge London New York New Rochelle

More information

The cardinal comparison of sets

The cardinal comparison of sets (B) The cardinal comparison of sets I think we can agree that there is some kind of fundamental difference between finite sets and infinite sets. For a finite set we can count its members and so give it

More information

Gödel, Turing, the Undecidability Results and the Nature of Human Mind

Gödel, Turing, the Undecidability Results and the Nature of Human Mind Gödel, Turing, the Undecidability Results and the Nature of Human Mind Riccardo Bruni riccardobruni@hotmail.com Dipartimento di Filosofia Università degli Studi di Firenze (Italy) Computability in Europe

More information

Ordinal Computability

Ordinal Computability Ordinal Computability by Peter Koepke University of Bonn Mathematisches Institut, Beringstraße 1, D 53115 Bonn, Germany Email: koepke@math.uni-bonn.de February 7, 2009 Abstract Ordinal computability uses

More information

Part II. Logic and Set Theory. Year

Part II. Logic and Set Theory. Year Part II Year 2018 2017 2016 2015 2014 2013 2012 2011 2010 2009 2008 2007 2006 2005 2018 60 Paper 4, Section II 16G State and prove the ǫ-recursion Theorem. [You may assume the Principle of ǫ- Induction.]

More information

Lecture 14 Rosser s Theorem, the length of proofs, Robinson s Arithmetic, and Church s theorem. Michael Beeson

Lecture 14 Rosser s Theorem, the length of proofs, Robinson s Arithmetic, and Church s theorem. Michael Beeson Lecture 14 Rosser s Theorem, the length of proofs, Robinson s Arithmetic, and Church s theorem Michael Beeson The hypotheses needed to prove incompleteness The question immediate arises whether the incompleteness

More information

Finite Automata Theory and Formal Languages TMV027/DIT321 LP4 2018

Finite Automata Theory and Formal Languages TMV027/DIT321 LP4 2018 Finite Automata Theory and Formal Languages TMV027/DIT321 LP4 2018 Lecture 15 Ana Bove May 17th 2018 Recap: Context-free Languages Chomsky hierarchy: Regular languages are also context-free; Pumping lemma

More information

CITS2211 Discrete Structures (2017) Cardinality and Countability

CITS2211 Discrete Structures (2017) Cardinality and Countability CITS2211 Discrete Structures (2017) Cardinality and Countability Highlights What is cardinality? Is it the same as size? Types of cardinality and infinite sets Reading Sections 45 and 81 84 of Mathematics

More information

Notes on Complexity Theory Last updated: October, Lecture 6

Notes on Complexity Theory Last updated: October, Lecture 6 Notes on Complexity Theory Last updated: October, 2015 Lecture 6 Notes by Jonathan Katz, lightly edited by Dov Gordon 1 PSPACE and PSPACE-Completeness As in our previous study of N P, it is useful to identify

More information

2 Plain Kolmogorov Complexity

2 Plain Kolmogorov Complexity 2 Plain Kolmogorov Complexity In this section, we introduce plain Kolmogorov Complexity, prove the invariance theorem - that is, the complexity of a string does not depend crucially on the particular model

More information