Characterizing First Order Logic

Size: px
Start display at page:

Download "Characterizing First Order Logic"

Transcription

1 Characterizing First Order Logic Jared Holshouser, Originally by Lindstrom September 16, 2014 We are following the presentation of Chang and Keisler. 1 A Brief Review of First Order Logic Definition 1. A language L is a collection of symbols, which are broken into three groups: relation symbols, function symbols and constant symbols. Definition 2. Let L be a language. A model for L is a pair A = (A, I), where we call A the universe of A and I an interpretation function. I must be as follows: Each n-ary function symbol F gets taken to an n-ary function G : A n A, Each n-ary relation symbols R gets taken to an n-ary relation P A n, and Each constant symbol c gets taken to a constant x A. Proposition 1. Suppose A is a model for the language L. Let X be a set. Then we can expand A to a model of L = A X. Proof. WLOG X is disjoint from L. Let I be an interpretation on X. Then A = (A, I I ) suffices. Definition 3. For A, A, L, L, and X as above, we call A the expansion of A to L and A the reduct of A to L. Definition 4. Two models A = (A, I) and B = (B, J ) of L are isomorphic if there is a function f : A B so that f is a bijection, For each relation symbol R, if R is n-ary, then for all x 1,, x n A I(R)(x 1,, x n ) J (R)(f(x 1 ),, f(x n )), For each function symbol F, if F is n-ary, then for all x 1,, x n A For each constant symbol c, f(i(c)) = J (c). We write f : A = B. I(F )(x 1,, x n ) = J (F )(f(x 1 ),, f(x n )), 1

2 Definition 5. Suppose A = (A, I) and B = (B, J ) are models of L. Then B is a submodel of A if B A and the following hold: for R an n-ary relation symbol, J (R) = I(R) B n, for F an n-ary function symbol, J (F ) = I(f) B n, and for c a constant symbol, J (c) = I(c). We now define first order logic, recursively. First the allowable symbols: We have parentheses (,); variables v 1,, v n, ; connectives and ; and the quantifier. Note that these are used in addition to the symbols of L and the symbol =. Definition 6. The collection of terms is defined recursively as follows: 1. A variable is a term, 2. a constant symbol is a term, and 3. if F is an n-ary function symbol, and t 1,, t n are terms, then F (t 1,, t n ) is a term. Definition 7. The collection of atomic formulas is defined recursively as follows: 1. if t 1 and t 2 are terms, then t 1 = t 2 is an atomic formula, 2. if R is an n-ary relation symbol and t 1,, t n are terms, then R(t 1,, t n ) is an atomic formula. Definition 8. The collection of formulas is defined recursively as follows: 1. atomic formulas are formulas, 2. if φ and ψ are formulas, then φ ψ and φ are formulas, 3. if v is a variable, and φ is a formula, then vφ is a formula. Definition 9. A sentence is a formula with no free variables. We now define model satisfaction: Definition 10. Fix a model A of a language L. We will define A = φ[ x] for formulas φ, and t[ x] for terms t. We begin with terms. If t is v i, then t[ x] := x i. If t is c, then t[ x] := I(c). If t is F (t 1,, t n ), then t[ x] = I(F )(t 1 [ x],, t n [ x]). Now we do atomic formulas. Suppose φ is t 1 = t 2. Then A = φ( x) t 1 [ x] = t 2 [ x]. Suppose φ is R(t 1,, t n ). Then A = φ( x) I(R)(t 1 [ x],, t n [ x]). Finally we do formulas. A = (φ ψ) iff A = φ and A = ψ. A = φ iff it is false that A = φ. A = v i φ[x 1,, x m ] (for i m) iff for all a A, A = φ[x 0,, x i 1, a, x i+1,, x m ] Remark 1. For sentences φ, we can write A = φ instead of A = φ[ x], as it does not depend on x. 2

3 Definition 11. Two models A and B of a language L are elementarily equivalent iff whenever φ is a sentence we have that A = φ iff B = φ. We write A B. Proposition 2. If A = B, then A B. Definition 12. Let Σ be a set of sentences of L. Then Σ has a model if there is a model A of L so that A = φ for all φ Σ. Theorem 1 (Compactness Theorem). A set of sentences Σ has a model iff every finite subset of Σ has a model. Theorem 2 (Downward Lowehnheim-Skolem Theorem). Every every consistent set of sentences in the language L has a model of size max{ω, L }. In particular, every valid sentence has a countable model. 3

4 2 Abstract Logics From here on, in order to simplify the argument, we restrict the discussion to lanaguages without function symbols. Definition 13. An abstract logic is a pair of classes (l, = l ) with the following properties: l is the class of sentences and = l is the satisfaction relation of the logic (l, = l ). 1. The Occurrence Property: For each φ l there is associated a finite language L φ called the set of symbols occuring in φ. The relation A = l φ is a relation between sentences φ of l and models A for languages L which contain L φ. 2. The Expansion Property: The relation A = l φ depends only on the reduct of A to L φ. I.e. if A = l φ and B is an expansion of A to a larger language, then B = l φ. 3. The Isomorphism Property: The relation A = l φ is preserved under isomorphism. 4. The Renaming Property: The relation A = l φ is preserved under renaming. That is, if we relabel the symbols of the logic, and modify the model accordingly, = l is preserved. 5. The Closure Property: l contains all atomic sentences, l is closed under the usual first order connectives, = l satisfies the usual rules for satisfaction of atomic formulas and first order connectives, and the set of symbols L φ behaves as expected for atomic sentences and first order connectives. 6. The Quantifier Property: l is closed under universal and existential quantifiers, and behaves as expected for them. 7. The Relativization Property: For each sentence φ l and relation R(x, b 1,, b n ) with R, b 1,, b n not in L φ, there is a new sentence φ R(x, b 1,, b n ), read φ relativized to R(x, b 1,, b n ) which has the set of symbols L φ {R, b 1,, b n } and is such that whenever B is the submodel of a model A for L φ with universe B = {a A : R(a, b 1,, b n )}, we have (A, R, b 1,, b n ) = l φ R(x, b 1,, b n ) iff B = l φ Remark 2. This notion of abstract logic does not have free variables, so l should be considered as a collection of sentences. Proposition 3. First order logic is an abstract logic. Proof. Properties 1-6 are either standard theorems or obviously true. We will prove that property 7 holds. Let φ be a sentence of first order logic, and R(x, b 1,, b n ) be a relation. Then the relativization of φ is formed as follows. Replace the quantifier xψ by and replace the quantifier xψ by x[r(x, b 1,, b n ) = ψ] x[r(x, b 1,, b n ) ψ] Remark 3. Every abstract logic l contains first order logic by the closure and quantifier properties. Definition 14. Two abstract logics l, l are equivalent if for all φ l, there is a ψ l so that L φ = L ψ and A = l φ iff A = l ψ for all A; and similarly for all ψ l. 4

5 Definition 15. By a model of a set T of sentences of an abstract logic l we mean a model A so that A = l φ for all φ T. Two models A and B for the same language l are l-elementarily equivalent if for each sentence φ l, A = l φ iff B = l φ. Definition 16. An abstract logic l is countably compact iff for every countable set T l, if every finite subset of T has a model, then T has a model. The Lowenheim number of l is the least cardinal α such that every sentence of l which has a model, has a model of power at most α. Remark 4. If the Lowenheim number of a logic l exists, it must be at least ω, as l contains every sentence of first order logic. Proposition 4. Let l be an abstract logic such that for each finite language L, the class {φ l : L φ L} is a set. Then the Lowenheim number of l exists. Proof. By renaming, we can WLOG assume that if φ l, then L φ V ω. This makes l a set. Define a map α : l ON by { ω if φ has no models α(φ) = κ if κ is the size of the smallest model of φ Then sup{α(φ) : φ l} exists, and is the Lowenheim number of l. Definition 17. Let A and B be models for a language L. A partial isomorphism I : A = p B is a relation I on the set of pairs of finite sequences (a 1,, a n ), (b 1,, b n ) of elements of A and B of the same length such that 1. I 2. If (a 1,, a n )I(b 1,, b n ), then (A, a 1,, a n ) and (B, b 1,, b n ) satisfy the same atomic sentences of L(c 1,, c n ) 3. If (a 1,, a n )I(b 1,, b n ), then and vice versa. c A d B[(a 1,, a n, c)i(b 1,, b n, d)] Proposition 5. Any two finite or countable partially isomorphic models are isomorpic. Proposition 6. Let l be an abstract logic which has Lowenheim number ω. Then any two models which are partially isomorphic are l-elementarily equivalent. Proof. Suppose A and B are models for a language L and I : A = p B. Suppose by way of contradiction that there is a φ l so that A = l φ and B = l φ. WLOG we may assume that L = L φ and that I is preserved under subsequences. For the first, use reducts, and for the second extend I in the obvious way. Define F : A <ω A A <ω and F : A <ω A <ω A <ω by and F ((a 1,, a n ), b) = (a 1,, a n, b) F ((a 1,, a n ), (b 1,, b m )) = (a 1,, a n, b 1,, b m ) Let A = (A A <ω, A, F, F ) be a model, where F and F are treated as relations. Similarly build B = (B B <ω, B, G, G ). WLOG, by the isomorphism property, A,A <ω, B, and B <ω are all disjoint from each other. Now consider C = (A, B, I). Then by the closure, quantifier, and relativization properties of l, there is a sentence ψ l so that C = l ψ and ψ = [(A = l φ) (B = l φ) (A = p B)] Then ψ has a countable model C 0, which gives us models A 0 and B 0 for L. Then A 0 = B0. This contradicts the isomorphism property, as C 0 = ψ. 5

6 3 The Main Theorem Theorem 3 (Lindstrom s Characterization of First Order Logic). Suppose l is an abstract logic which is countably compact and has Lowenheim number ω. Then l is equivalent to first order logic. Proof. Let l be a countably compact abstract logic with Lowenheim number ω. Let φ be a sentence of first order logic, and A be a model of L φ. Then by the closure and quantifier properties, A = φ iff A = l φ. Now we must prove the other direction. We first define some relations between models of a finite language L. Let A and B be models of L. We define relations I k for k ω between A and B recursively. Let (a 1,, a n ) A n and (B 1,, b n ) B n. ai 0 b iff a and b satisfy the same atomic formulas. ai k+1 b iff 1. c A d B((a 1,, a n, c)i k (b 1,, b n, d)) and 2. d B c A((a 1,, a n, c)i k (b 1,, b n, d)). We say A k B if I k. Since L is finite and has no function symbols, for each k there is a finite set Γ k of first order logic in L such that for all models A and B of L, A k B iff A and B agree on Γ k. Let φ l be a sentence so that L φ L. It suffices to show that there is a k so that for all models A and B of L, (A k B and A = l φ) = B = l φ For then we will know that for some boolean combination of sentences in Γ k, ψ, L φ = L ψ and for all models A of L φ, A = l φ iff A = ψ. We proceed by way of contradiction. For each k choose models A k and B k so that A k k B k and A = l φ and B = l φ (1) Taking a subsequence if necessary, we can assume that the A k satisfy the same atomic sentences. By the isomorphism property, we can assume that the A k interpret the constants of L the same way. Let A = k A k. Each A k is a submodel of A, and we can take the A k so that A k ω =. As in the previous proof, let A = (A A <ω, A, F, F ) Similarly define B and B. Let where R, S and I are so that C = (A, B, R, S, ω,, I) A k = {a A : R(a, k)}, B k = {b B : S(b, k)}, A <ω k = { a A <ω : R( a, k)}, B k <ω = { b B <ω : S( b, k)}, and for each k, I( a, b, k) holds iff ai k b. By the closure, quantifier, and relativization properties there is a sentence θ l so that C = l θ and θ implies that (ω, ) is a total order with immediate successors and predecessors except for the first element, and (1) holds for all k ω. By countable compactness, θ has a model Ĉ = (Â, ˆB, ˆR, Ŝ, ˆω, ˆ, Î) so that ˆω has a nonstandard element H. Then ÂH = l φ, ˆBH = l φ, and ÂH H ˆBH. Define J between ÂH and ˆB H by (a 1,, a n )J(b 1,, b n ) iff (a 1,, a n )ÎH n(b 1,, b n ) Then J is a partial isomorphism between ÂH and ˆB H. But then by the previous proposition and the fact that l has Lowenheim number ω, ÂH l ˆBH. This is a contradiction. 6

LINDSTRÖM S THEOREM SALMAN SIDDIQI

LINDSTRÖM S THEOREM SALMAN SIDDIQI LINDSTRÖM S THEOREM SALMAN SIDDIQI Abstract. This paper attempts to serve as an introduction to abstract model theory. We introduce the notion of abstract logics, explore first-order logic as an instance

More information

Introduction to Model Theory

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

More information

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

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

More information

Basics of Model Theory

Basics of Model Theory Chapter udf Basics of Model Theory bas.1 Reducts and Expansions mod:bas:red: defn:reduct mod:bas:red: prop:reduct Often it is useful or necessary to compare languages which have symbols in common, as well

More information

1 Completeness Theorem for Classical Predicate

1 Completeness Theorem for Classical Predicate 1 Completeness Theorem for Classical Predicate Logic The relationship between the first order models defined in terms of structures M = [M, I] and valuations s : V AR M and propositional models defined

More information

Löwenheim-Skolem Theorems, Countable Approximations, and L ω. David W. Kueker (Lecture Notes, Fall 2007)

Löwenheim-Skolem Theorems, Countable Approximations, and L ω. David W. Kueker (Lecture Notes, Fall 2007) Löwenheim-Skolem Theorems, Countable Approximations, and L ω 0. Introduction David W. Kueker (Lecture Notes, Fall 2007) In its simplest form the Löwenheim-Skolem Theorem for L ω1 ω states that if σ L ω1

More information

MATHEMATICS: CONCEPTS, AND FOUNDATIONS Vol. II - Model Theory - H. Jerome Keisler

MATHEMATICS: CONCEPTS, AND FOUNDATIONS Vol. II - Model Theory - H. Jerome Keisler ATHEATCS: CONCEPTS, AND FOUNDATONS Vol. - odel Theory - H. Jerome Keisler ODEL THEORY H. Jerome Keisler Department of athematics, University of Wisconsin, adison Wisconsin U.S.A. Keywords: adapted probability

More information

PRESERVATION THEOREMS IN LUKASIEWICZ MODEL THEORY

PRESERVATION THEOREMS IN LUKASIEWICZ MODEL THEORY Iranian Journal of Fuzzy Systems Vol. 10, No. 3, (2013) pp. 103-113 103 PRESERVATION THEOREMS IN LUKASIEWICZ MODEL THEORY S. M. BAGHERI AND M. MONIRI Abstract. We present some model theoretic results for

More information

More Model Theory Notes

More Model Theory Notes More Model Theory Notes Miscellaneous information, loosely organized. 1. Kinds of Models A countable homogeneous model M is one such that, for any partial elementary map f : A M with A M finite, and any

More information

EXCURSIONS IN MODEL THEORY

EXCURSIONS IN MODEL THEORY EXCURSIONS IN MODEL THEORY RAFAEL WINGESTER RIBEIRO DE OLIVEIRA Abstract. This paper aims to introduce the reader familiar with undergraduate level logic to some fundamental constructions in Model Theory.

More information

ULTRAPRODUCTS AND MODEL THEORY

ULTRAPRODUCTS AND MODEL THEORY ULTRAPRODUCTS AND MODEL THEORY AARON HALPER Abstract. The first-order model-theoretic description of mathematical structures is unable to always uniquely characterize models up to isomorphism when the

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

Overview of Topics. Finite Model Theory. Finite Model Theory. Connections to Database Theory. Qing Wang

Overview of Topics. Finite Model Theory. Finite Model Theory. Connections to Database Theory. Qing Wang Overview of Topics Finite Model Theory Part 1: Introduction 1 What is finite model theory? 2 Connections to some areas in CS Qing Wang qing.wang@anu.edu.au Database theory Complexity theory 3 Basic definitions

More information

Fundamentals of Model Theory

Fundamentals of Model Theory Fundamentals of Model Theory William Weiss and Cherie D Mello Department of Mathematics University of Toronto c 2015 W.Weiss and C. D Mello 1 Introduction Model Theory is the part of mathematics which

More information

COMPLETENESS OF THE RANDOM GRAPH: TWO PROOFS

COMPLETENESS OF THE RANDOM GRAPH: TWO PROOFS COMPLETENESS OF THE RANDOM GRAPH: TWO PROOFS EUGENIA FUCHS Abstract. We take a countably infinite random graph, state its axioms as a theory in first-order logic, and prove its completeness in two distinct

More information

Harmonious Logic: Craig s Interpolation Theorem and its Descendants. Solomon Feferman Stanford University

Harmonious Logic: Craig s Interpolation Theorem and its Descendants. Solomon Feferman Stanford University Harmonious Logic: Craig s Interpolation Theorem and its Descendants Solomon Feferman Stanford University http://math.stanford.edu/~feferman Interpolations Conference in Honor of William Craig 13 May 2007

More information

VAUGHT S THEOREM: THE FINITE SPECTRUM OF COMPLETE THEORIES IN ℵ 0. Contents

VAUGHT S THEOREM: THE FINITE SPECTRUM OF COMPLETE THEORIES IN ℵ 0. Contents VAUGHT S THEOREM: THE FINITE SPECTRUM OF COMPLETE THEORIES IN ℵ 0 BENJAMIN LEDEAUX Abstract. This expository paper introduces model theory with a focus on countable models of complete theories. Vaught

More information

Completeness in the Monadic Predicate Calculus. We have a system of eight rules of proof. Let's list them:

Completeness in the Monadic Predicate Calculus. We have a system of eight rules of proof. Let's list them: Completeness in the Monadic Predicate Calculus We have a system of eight rules of proof. Let's list them: PI At any stage of a derivation, you may write down a sentence φ with {φ} as its premiss set. TC

More information

Pseudo-finite model theory

Pseudo-finite model theory Mat. Contemp. 24 (2003), 169-183. Pseudo-finite model theory Jouko Väänänen Department of Mathematics University of Helsinki Helsinki, Finland jouko.vaananen@helsinki.fi September 24, 2002 Abstract We

More information

A MODEL-THEORETIC PROOF OF HILBERT S NULLSTELLENSATZ

A MODEL-THEORETIC PROOF OF HILBERT S NULLSTELLENSATZ A MODEL-THEORETIC PROOF OF HILBERT S NULLSTELLENSATZ NICOLAS FORD Abstract. The goal of this paper is to present a proof of the Nullstellensatz using tools from a branch of logic called model theory. In

More information

Final Exam (100 points)

Final Exam (100 points) Final Exam (100 points) Honor Code: Each question is worth 10 points. There is one bonus question worth 5 points. In contrast to the homework assignments, you may not collaborate on this final exam. You

More information

FINITE MODEL THEORY (MATH 285D, UCLA, WINTER 2017) LECTURE NOTES IN PROGRESS

FINITE MODEL THEORY (MATH 285D, UCLA, WINTER 2017) LECTURE NOTES IN PROGRESS FINITE MODEL THEORY (MATH 285D, UCLA, WINTER 2017) LECTURE NOTES IN PROGRESS ARTEM CHERNIKOV 1. Intro Motivated by connections with computational complexity (mostly a part of computer scientice today).

More information

Clearly C B, for every C Q. Suppose that we may find v 1, v 2,..., v n

Clearly C B, for every C Q. Suppose that we may find v 1, v 2,..., v n 10. Algebraic closure Definition 10.1. Let K be a field. The algebraic closure of K, denoted K, is an algebraic field extension L/K such that every polynomial in K[x] splits in L. We say that K is algebraically

More information

Math 225A Model Theory. Speirs, Martin

Math 225A Model Theory. Speirs, Martin Math 5A Model Theory Speirs, Martin Autumn 013 General Information These notes are based on a course in Metamathematics taught by Professor Thomas Scanlon at UC Berkeley in the Autumn of 013. The course

More information

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

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

More information

Herbrand Theorem, Equality, and Compactness

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

More information

ω-stable Theories: Introduction

ω-stable Theories: Introduction ω-stable Theories: Introduction 1 ω - Stable/Totally Transcendental Theories Throughout let T be a complete theory in a countable language L having infinite models. For an L-structure M and A M let Sn

More information

Short notes on Axioms of set theory, Well orderings and Ordinal Numbers

Short notes on Axioms of set theory, Well orderings and Ordinal Numbers Short notes on Axioms of set theory, Well orderings and Ordinal Numbers August 29, 2013 1 Logic and Notation Any formula in Mathematics can be stated using the symbols and the variables,,,, =, (, ) v j

More information

Scott Sentences in Uncountable Structures

Scott Sentences in Uncountable Structures Rose-Hulman Undergraduate Mathematics Journal Volume 18 Issue 1 Article 14 Scott Sentences in Uncountable Structures Brian Tyrrell Trinity College Dublin Follow this and additional works at: http://scholar.rose-hulman.edu/rhumj

More information

NOTES ON WELL ORDERING AND ORDINAL NUMBERS. 1. Logic and Notation Any formula in Mathematics can be stated using the symbols

NOTES ON WELL ORDERING AND ORDINAL NUMBERS. 1. Logic and Notation Any formula in Mathematics can be stated using the symbols NOTES ON WELL ORDERING AND ORDINAL NUMBERS TH. SCHLUMPRECHT 1. Logic and Notation Any formula in Mathematics can be stated using the symbols,,,, =, (, ) and the variables v j : where j is a natural number.

More information

Introduction to Model Theory

Introduction to Model Theory Introduction to Model Theory Jouko Väänänen 1,2 1 Department of Mathematics and Statistics, University of Helsinki 2 Institute for Logic, Language and Computation, University of Amsterdam Beijing, June

More information

tp(c/a) tp(c/ab) T h(m M ) is assumed in the background.

tp(c/a) tp(c/ab) T h(m M ) is assumed in the background. Model Theory II. 80824 22.10.2006-22.01-2007 (not: 17.12) Time: The first meeting will be on SUNDAY, OCT. 22, 10-12, room 209. We will try to make this time change permanent. Please write ehud@math.huji.ac.il

More information

October 12, Complexity and Absoluteness in L ω1,ω. John T. Baldwin. Measuring complexity. Complexity of. concepts. to first order.

October 12, Complexity and Absoluteness in L ω1,ω. John T. Baldwin. Measuring complexity. Complexity of. concepts. to first order. October 12, 2010 Sacks Dicta... the central notions of model theory are absolute absoluteness, unlike cardinality, is a logical concept. That is why model theory does not founder on that rock of undecidability,

More information

Friendly Logics, Fall 2015, Lecture Notes 5

Friendly Logics, Fall 2015, Lecture Notes 5 Friendly Logics, Fall 2015, Lecture Notes 5 Val Tannen 1 FO definability In these lecture notes we restrict attention to relational vocabularies i.e., vocabularies consisting only of relation symbols (or

More information

1 Completeness Theorem for First Order Logic

1 Completeness Theorem for First Order Logic 1 Completeness Theorem for First Order Logic There are many proofs of the Completeness Theorem for First Order Logic. We follow here a version of Henkin s proof, as presented in the Handbook of Mathematical

More information

Mathematical Logic (IX)

Mathematical Logic (IX) Mathematical Logic (IX) Yijia Chen 1. The Löwenheim-Skolem Theorem and the Compactness Theorem Using the term-interpretation, it is routine to verify: Theorem 1.1 (Löwenheim-Skolem). Let Φ L S be at most

More information

Categoricity Without Equality

Categoricity Without Equality Categoricity Without Equality H. Jerome Keisler and Arnold W. Miller Abstract We study categoricity in power for reduced models of first order logic without equality. 1 Introduction The object of this

More information

Lecture 13: Soundness, Completeness and Compactness

Lecture 13: Soundness, Completeness and Compactness Discrete Mathematics (II) Spring 2017 Lecture 13: Soundness, Completeness and Compactness Lecturer: Yi Li 1 Overview In this lecture, we will prvoe the soundness and completeness of tableau proof system,

More information

The Vaught Conjecture Do uncountable models count?

The Vaught Conjecture Do uncountable models count? The Vaught Conjecture Do uncountable models count? John T. Baldwin Department of Mathematics, Statistics and Computer Science University of Illinois at Chicago May 22, 2005 1 Is the Vaught Conjecture model

More information

This is logically equivalent to the conjunction of the positive assertion Minimal Arithmetic and Representability

This is logically equivalent to the conjunction of the positive assertion Minimal Arithmetic and Representability 16.2. MINIMAL ARITHMETIC AND REPRESENTABILITY 207 If T is a consistent theory in the language of arithmetic, we say a set S is defined in T by D(x) if for all n, if n is in S, then D(n) is a theorem of

More information

Solutions to Unique Readability Homework Set 30 August 2011

Solutions to Unique Readability Homework Set 30 August 2011 s to Unique Readability Homework Set 30 August 2011 In the problems below L is a signature and X is a set of variables. Problem 0. Define a function λ from the set of finite nonempty sequences of elements

More information

The Absoluteness of Constructibility

The Absoluteness of Constructibility Lecture: The Absoluteness of Constructibility We would like to show that L is a model of V = L, or, more precisely, that L is an interpretation of ZF + V = L in ZF. We have already verified that σ L holds

More information

CHAPTER 2. FIRST ORDER LOGIC

CHAPTER 2. FIRST ORDER LOGIC CHAPTER 2. FIRST ORDER LOGIC 1. Introduction First order logic is a much richer system than sentential logic. Its interpretations include the usual structures of mathematics, and its sentences enable us

More information

Notes for Math 601, Fall based on Introduction to Mathematical Logic by Elliott Mendelson Fifth edition, 2010, Chapman & Hall

Notes for Math 601, Fall based on Introduction to Mathematical Logic by Elliott Mendelson Fifth edition, 2010, Chapman & Hall Notes for Math 601, Fall 2010 based on Introduction to Mathematical Logic by Elliott Mendelson Fifth edition, 2010, Chapman & Hall All first-order languages contain the variables: v 0, v 1, v 2,... the

More information

2.2 Lowenheim-Skolem-Tarski theorems

2.2 Lowenheim-Skolem-Tarski theorems Logic SEP: Day 1 July 15, 2013 1 Some references Syllabus: http://www.math.wisc.edu/graduate/guide-qe Previous years qualifying exams: http://www.math.wisc.edu/ miller/old/qual/index.html Miller s Moore

More information

Axioms for Set Theory

Axioms for Set Theory Axioms for Set Theory The following is a subset of the Zermelo-Fraenkel axioms for set theory. In this setting, all objects are sets which are denoted by letters, e.g. x, y, X, Y. Equality is logical identity:

More information

A Note on Graded Modal Logic

A Note on Graded Modal Logic A Note on Graded Modal Logic Maarten de Rijke Studia Logica, vol. 64 (2000), pp. 271 283 Abstract We introduce a notion of bisimulation for graded modal logic. Using these bisimulations the model theory

More information

SEPARABLE MODELS OF RANDOMIZATIONS

SEPARABLE MODELS OF RANDOMIZATIONS SEPARABLE MODELS OF RANDOMIZATIONS URI ANDREWS AND H. JEROME KEISLER Abstract. Every complete first order theory has a corresponding complete theory in continuous logic, called the randomization theory.

More information

USING ULTRAPOWERS TO CHARACTERIZE ELEMENTARY EQUIVALENCE

USING ULTRAPOWERS TO CHARACTERIZE ELEMENTARY EQUIVALENCE USING ULTRAPOWERS TO CHARACTERIZE ELEMENTARY EQUIVALENCE MIKAYLA KELLEY Abstract. This paper will establish that ultrapowers can be used to determine whether or not two models have the same theory. More

More information

Propositional and Predicate Logic - VII

Propositional and Predicate Logic - VII Propositional and Predicate Logic - VII Petr Gregor KTIML MFF UK WS 2015/2016 Petr Gregor (KTIML MFF UK) Propositional and Predicate Logic - VII WS 2015/2016 1 / 11 Theory Validity in a theory A theory

More information

Introduction. Itaï Ben-Yaacov C. Ward Henson. September American Institute of Mathematics Workshop. Continuous logic Continuous model theory

Introduction. Itaï Ben-Yaacov C. Ward Henson. September American Institute of Mathematics Workshop. Continuous logic Continuous model theory Itaï Ben-Yaacov C. Ward Henson American Institute of Mathematics Workshop September 2006 Outline Continuous logic 1 Continuous logic 2 The metric on S n (T ) Origins Continuous logic Many classes of (complete)

More information

Morley s Proof. Winnipeg June 3, 2007

Morley s Proof. Winnipeg June 3, 2007 Modern Model Theory Begins Theorem (Morley 1965) If a countable first order theory is categorical in one uncountable cardinal it is categorical in all uncountable cardinals. Outline 1 2 3 SELF-CONSCIOUS

More information

Model Theory MARIA MANZANO. University of Salamanca, Spain. Translated by RUY J. G. B. DE QUEIROZ

Model Theory MARIA MANZANO. University of Salamanca, Spain. Translated by RUY J. G. B. DE QUEIROZ Model Theory MARIA MANZANO University of Salamanca, Spain Translated by RUY J. G. B. DE QUEIROZ CLARENDON PRESS OXFORD 1999 Contents Glossary of symbols and abbreviations General introduction 1 xix 1 1.0

More information

A1 Logic (25 points) Using resolution or another proof technique of your stated choice, establish each of the following.

A1 Logic (25 points) Using resolution or another proof technique of your stated choice, establish each of the following. A1 Logic (25 points) Using resolution or another proof technique of your stated choice, establish each of the following. = ( x)( y)p (x, y, f(x, y)) ( x)( y)( z)p (x, y, z)). b. (6.25 points) Γ = ( x)p

More information

A generalization of modal definability

A generalization of modal definability A generalization of modal definability Tin Perkov Polytechnic of Zagreb Abstract. Known results on global definability in basic modal logic are generalized in the following sense. A class of Kripke models

More information

Scott processes. Paul B. Larson June 23, 2014

Scott processes. Paul B. Larson June 23, 2014 Scott processes Paul B. Larson June 23, 2014 Abstract The Scott process of a relational structure M is the sequence of sets of formulas given by the Scott analysis of M. We present axioms for the class

More information

1 Introductory notes on the model theory of valued fields

1 Introductory notes on the model theory of valued fields 1 Introductory notes on the model theory of valued fields Zoé Chatzidakis a (CNRS - Université Paris 7) These notes will give some very basic definitions and results from model theory. They contain many

More information

Incomplete version for students of easllc2012 only. 6.6 The Model Existence Game 99

Incomplete version for students of easllc2012 only. 6.6 The Model Existence Game 99 98 First-Order Logic 6.6 The Model Existence Game In this section we learn a new game associated with trying to construct a model for a sentence or a set of sentences. This is of fundamental importance

More information

What is the right type-space? Humboldt University. July 5, John T. Baldwin. Which Stone Space? July 5, Tameness.

What is the right type-space? Humboldt University. July 5, John T. Baldwin. Which Stone Space? July 5, Tameness. Goals The fundamental notion of a Stone space is delicate for infinitary logic. I will describe several possibilities. There will be a quiz. Infinitary Logic and Omitting Types Key Insight (Chang, Lopez-Escobar)

More information

Propositional and Predicate Logic - IV

Propositional and Predicate Logic - IV Propositional and Predicate Logic - IV Petr Gregor KTIML MFF UK ZS 2015/2016 Petr Gregor (KTIML MFF UK) Propositional and Predicate Logic - IV ZS 2015/2016 1 / 19 Tableau method (from the previous lecture)

More information

Syntactic Characterisations in Model Theory

Syntactic Characterisations in Model Theory Department of Mathematics Bachelor Thesis (7.5 ECTS) Syntactic Characterisations in Model Theory Author: Dionijs van Tuijl Supervisor: Dr. Jaap van Oosten June 15, 2016 Contents 1 Introduction 2 2 Preliminaries

More information

03 Review of First-Order Logic

03 Review of First-Order Logic CAS 734 Winter 2014 03 Review of First-Order Logic William M. Farmer Department of Computing and Software McMaster University 18 January 2014 What is First-Order Logic? First-order logic is the study of

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

A Local Normal Form Theorem for Infinitary Logic with Unary Quantifiers

A Local Normal Form Theorem for Infinitary Logic with Unary Quantifiers mlq header will be provided by the publisher Local Normal Form Theorem for Infinitary Logic with Unary Quantifiers H. Jerome Keisler 1 and Wafik Boulos Lotfallah 2 1 Department of Mathematics University

More information

Qualifying Exam Logic August 2005

Qualifying Exam Logic August 2005 Instructions: Qualifying Exam Logic August 2005 If you signed up for Computability Theory, do two E and two C problems. If you signed up for Model Theory, do two E and two M problems. If you signed up

More information

Finite Model Theory: First-Order Logic on the Class of Finite Models

Finite Model Theory: First-Order Logic on the Class of Finite Models 1 Finite Model Theory: First-Order Logic on the Class of Finite Models Anuj Dawar University of Cambridge Modnet Tutorial, La Roche, 21 April 2008 2 Finite Model Theory In the 1980s, the term finite model

More information

Algebraizing Hybrid Logic. Evangelos Tzanis University of Amsterdam Institute of Logic, Language and Computation

Algebraizing Hybrid Logic. Evangelos Tzanis University of Amsterdam Institute of Logic, Language and Computation Algebraizing Hybrid Logic Evangelos Tzanis University of Amsterdam Institute of Logic, Language and Computation etzanis@science.uva.nl May 1, 2005 2 Contents 1 Introduction 5 1.1 A guide to this thesis..........................

More information

MODEL THEORY FOR ALGEBRAIC GEOMETRY

MODEL THEORY FOR ALGEBRAIC GEOMETRY MODEL THEORY FOR ALGEBRAIC GEOMETRY VICTOR ZHANG Abstract. We demonstrate how several problems of algebraic geometry, i.e. Ax-Grothendieck, Hilbert s Nullstellensatz, Noether- Ostrowski, and Hilbert s

More information

Math 280A Fall Axioms of Set Theory

Math 280A Fall Axioms of Set Theory Math 280A Fall 2009 1. Axioms of Set Theory Let V be the collection of all sets and be a membership relation. We consider (V, ) as a mathematical structure. Analogy: A group is a mathematical structure

More information

RANK HIERARCHIES FOR GENERALIZED QUANTIFIERS

RANK HIERARCHIES FOR GENERALIZED QUANTIFIERS RANK HIERARCHIES FOR GENERALIZED QUANTIFIERS H. JEROME KEISLER AND WAFIK BOULOS LOTFALLAH Abstract. We show that for each n and m, there is an existential first order sentence which is NOT logically equivalent

More information

Infinite and Finite Model Theory Part II

Infinite and Finite Model Theory Part II Infinite and Finite Model Theory Part II Anuj Dawar Computer Laboratory University of Cambridge Lent 2002 3/2002 0 Finite Model Theory Finite Model Theory motivated by computational issues; relationship

More information

Relative categoricity in abelian groups

Relative categoricity in abelian groups Relative categoricity in abelian groups Wilfrid Hodges and Anatoly Yakovlev Abstract We consider structures A consisting of an abelian group with a subgroup A P distinguished by a 1-ary relation symbol

More information

Handout: Proof of the completeness theorem

Handout: Proof of the completeness theorem MATH 457 Introduction to Mathematical Logic Spring 2016 Dr. Jason Rute Handout: Proof of the completeness theorem Gödel s Compactness Theorem 1930. For a set Γ of wffs and a wff ϕ, we have the following.

More information

The constructible universe

The constructible universe The constructible universe In this set of notes I want to sketch Gödel s proof that CH is consistent with the other axioms of set theory. Gödel s argument goes well beyond this result; his identification

More information

GÖDEL S CONSTRUCTIBLE UNIVERSE

GÖDEL S CONSTRUCTIBLE UNIVERSE GÖDEL S CONSTRUCTIBLE UNIVERSE MICHAEL WOLMAN Abstract. This paper is about Gödel s Constructible Universe and the relative consistency of Zermelo-Fraenkel set theory, the Continuum Hypothesis and the

More information

March 3, The large and small in model theory: What are the amalgamation spectra of. infinitary classes? John T. Baldwin

March 3, The large and small in model theory: What are the amalgamation spectra of. infinitary classes? John T. Baldwin large and large and March 3, 2015 Characterizing cardinals by L ω1,ω large and L ω1,ω satisfies downward Lowenheim Skolem to ℵ 0 for sentences. It does not satisfy upward Lowenheim Skolem. Definition sentence

More information

Pseudo-finite model theory

Pseudo-finite model theory Pseudo-finite model theory Jouko Väänänen Department of Mathematics University of Helsinki Helsinki, Finland jouko.vaananen@helsinki.fi August 1, 2016 Abstract We consider the restriction of first order

More information

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

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

More information

INDEPENDENCE RELATIONS IN RANDOMIZATIONS

INDEPENDENCE RELATIONS IN RANDOMIZATIONS INDEPENDENE RELATIONS IN RANDOMIZATIONS URI ANDREWS, ISAA GOLDBRING, AND H. JEROME KEISLER Abstract. The randomization of a complete first order theory T is the complete continuous theory T R with two

More information

AMS regional meeting Bloomington, IN April 1, 2017

AMS regional meeting Bloomington, IN April 1, 2017 Joint work with: W. Boney, S. Friedman, C. Laskowski, M. Koerwien, S. Shelah, I. Souldatos University of Illinois at Chicago AMS regional meeting Bloomington, IN April 1, 2017 Cantor s Middle Attic Uncountable

More information

Part II Logic and Set Theory

Part II Logic and Set Theory Part II Logic and Set Theory Theorems Based on lectures by I. B. Leader Notes taken by Dexter Chua Lent 2015 These notes are not endorsed by the lecturers, and I have modified them (often significantly)

More information

Decidability of integer multiplication and ordinal addition. Two applications of the Feferman-Vaught theory

Decidability of integer multiplication and ordinal addition. Two applications of the Feferman-Vaught theory Decidability of integer multiplication and ordinal addition Two applications of the Feferman-Vaught theory Ting Zhang Stanford University Stanford February 2003 Logic Seminar 1 The motivation There are

More information

Set Theory and the Foundation of Mathematics. June 19, 2018

Set Theory and the Foundation of Mathematics. June 19, 2018 1 Set Theory and the Foundation of Mathematics June 19, 2018 Basics Numbers 2 We have: Relations (subsets on their domain) Ordered pairs: The ordered pair x, y is the set {{x, y}, {x}}. Cartesian products

More information

Π 0 1-presentations of algebras

Π 0 1-presentations of algebras Π 0 1-presentations of algebras Bakhadyr Khoussainov Department of Computer Science, the University of Auckland, New Zealand bmk@cs.auckland.ac.nz Theodore Slaman Department of Mathematics, The University

More information

Abstract model theory for extensions of modal logic

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

More information

MORLEY S CATEGORICITY THEOREM

MORLEY S CATEGORICITY THEOREM MORLEY S CATEGORICITY THEOREM NICK RAMSEY Abstract. A theory is called κ-categorical, or categorical in power κ, if it has one model up to isomorphism of cardinality κ. Morley s Categoricity Theorem states

More information

A Vaught s conjecture toolbox

A Vaught s conjecture toolbox Chris Laskowski University of Maryland 2 nd Vaught s conjecture conference UC-Berkeley 1 June, 2015 Everything begins with the work of Robert Vaught. Everything begins with the work of Robert Vaught. Fix

More information

Continuum Harvard. April 11, Constructing Borel Models in the. Continuum Harvard. John T. Baldwin. University of Illinois at Chicago

Continuum Harvard. April 11, Constructing Borel Models in the. Continuum Harvard. John T. Baldwin. University of Illinois at Chicago April 11, 2013 Today s Topics 1 2 3 4 5 6 Pseudo-minimal 7 Further Applications Section 1: { Models in L ω1,ω L ω1,ω satisfies downward Löwenheim Skolem to ℵ 0 for sentences. It does not satisfy upward

More information

TABLEAU SYSTEM FOR LOGIC OF CATEGORIAL PROPOSITIONS AND DECIDABILITY

TABLEAU SYSTEM FOR LOGIC OF CATEGORIAL PROPOSITIONS AND DECIDABILITY Bulletin of the Section of Logic Volume 37:3/4 (2008), pp. 223 231 Tomasz Jarmużek TABLEAU SYSTEM FOR LOGIC OF CATEGORIAL PROPOSITIONS AND DECIDABILITY Abstract In the article we present an application

More information

Lecture 10: Predicate Logic and Its Language

Lecture 10: Predicate Logic and Its Language Discrete Mathematics (II) Spring 2017 Lecture 10: Predicate Logic and Its Language Lecturer: Yi Li 1 Predicates and Quantifiers In this action, we show you why a richer language should be introduced than

More information

Gödel s Completeness Theorem

Gödel s Completeness Theorem A.Miller M571 Spring 2002 Gödel s Completeness Theorem We only consider countable languages L for first order logic with equality which have only predicate symbols and constant symbols. We regard the symbols

More information

THE METAMATHEMATICS OF RANDOM GRAPHS

THE METAMATHEMATICS OF RANDOM GRAPHS THE METAMATHEMATICS OF RANDOM GRAPHS John T. Baldwin Department of Mathematics, Statistics and Computer Science University of Illinois at Chicago Abstract We explain and summarize the use of logic to provide

More information

Axiomatisation of Hybrid Logic

Axiomatisation of Hybrid Logic Imperial College London Department of Computing Axiomatisation of Hybrid Logic by Louis Paternault Submitted in partial fulfilment of the requirements for the MSc Degree in Advanced Computing of Imperial

More information

3. Only sequences that were formed by using finitely many applications of rules 1 and 2, are propositional formulas.

3. Only sequences that were formed by using finitely many applications of rules 1 and 2, are propositional formulas. 1 Chapter 1 Propositional Logic Mathematical logic studies correct thinking, correct deductions of statements from other statements. Let us make it more precise. A fundamental property of a statement is

More information

Logical Theories of Trees

Logical Theories of Trees Logical Theories of Trees by Ruaan Kellerman under the supervision of Prof. V. F. Goranko Prof. M. Möller School of Mathematics University of the Witwatersrand Johannesburg South Africa A thesis submitted

More information

Almost Galois ω-stable classes

Almost Galois ω-stable classes Almost Galois ω-stable classes John T. Baldwin Paul B. Larson Saharon Shelah March 11, 2015 Abstract Theorem. Suppose that k = (K, k ) is an ℵ 0-presentable abstract elementary class with Löwenheim-Skolem

More information

Introduction to Model theory Zoé Chatzidakis CNRS (Paris 7) Notes for Luminy, November 2001

Introduction to Model theory Zoé Chatzidakis CNRS (Paris 7) Notes for Luminy, November 2001 Introduction to Model theory Zoé Chatzidakis CNRS (Paris 7) Notes for Luminy, November 2001 These notes aim at giving the basic definitions and results from model theory. My intention in writing them,

More information

0-1 LAWS IN LOGIC: AN OVERVIEW

0-1 LAWS IN LOGIC: AN OVERVIEW 0-1 LAWS IN LOGIC: AN OVERVIEW ANAND ABRAHAM Abstract. I give an overview of 0-1 laws in logic. I give a proof of the 0-1 law for first-order logic, and then guide the reader through a series of extensions

More information

20 Ordinals. Definition A set α is an ordinal iff: (i) α is transitive; and. (ii) α is linearly ordered by. Example 20.2.

20 Ordinals. Definition A set α is an ordinal iff: (i) α is transitive; and. (ii) α is linearly ordered by. Example 20.2. 20 Definition 20.1. A set α is an ordinal iff: (i) α is transitive; and (ii) α is linearly ordered by. Example 20.2. (a) Each natural number n is an ordinal. (b) ω is an ordinal. (a) ω {ω} is an ordinal.

More information

DIVIDING AND WEAK QUASI-DIMENSIONS IN ARBITRARY THEORIES

DIVIDING AND WEAK QUASI-DIMENSIONS IN ARBITRARY THEORIES DIVIDING AND WEAK QUASI-DIMENSIONS IN ARBITRARY THEORIES ISAAC GODBRING AND HENRY TOWSNER Abstract. We show that any countable model of a model complete theory has an elementary extension with a pseudofinite-like

More information