Univalent Foundations and Set Theory

Similar documents
The equivalence axiom and univalent models of type theory.

Model Theory in the Univalent Foundations

Dependent type theory

A very short note on homotopy λ-calculus

Categorical models of homotopy type theory

From syntax to semantics of Dependent Type Theories - Formalized

Equality and dependent type theory. CIRM, May 31

Homotopy and Directed Type Theory: a Sample

Weak ω-groupoids in Type Theory

Introduction to type theory and homotopy theory

1 / A bird s-eye view of type theory. 2 A bird s-eye view of homotopy theory. 3 Path spaces and identity types. 4 Homotopy type theory

The synthetic theory of -categories vs the synthetic theory of -categories

Programming with Higher Inductive Types

Internalizing the simplicial model structure in Homotopy Type Theory. Simon Boulier

Homotopy theory in type theory

Categorical Homotopy Type Theory

Homotopy Type Theory

Higher Inductive types

Notes on homotopy λ-calculus

Journal of Pure and Applied Algebra

Homotopy theory in type theory

Algebraic models of homotopy type theory

Univalence for Free. Matthieu Sozeau Joint work with Nicolas Tabareau - INRIA. GT Types & Réalisabilité March 13th 2013

Type Theory and Univalent Foundation

Homotopy Type Theory. Benno van den Berg. LoLaCo, 29 September 2014

Recent progress in Homotopy type theory

Homotopy type theory

WHAT IS AN ELEMENTARY HIGHER TOPOS?

Higher Inductive Types: The circle and friends, axiomatically

Computer Proof Assistants and Univalent Foundations of Mathematics

PART III.3. IND-COHERENT SHEAVES ON IND-INF-SCHEMES

THE SIMPLICIAL MODEL OF UNIVALENT FOUNDATIONS

Depending on equations

Sheaf models of type theory

EXAMPLES AND EXERCISES IN BASIC CATEGORY THEORY

Structural Foundations for Abstract Mathematics

Category theory and set theory: algebraic set theory as an example of their interaction

Dependent Type Theories. Lecture 4. Computing the B-sets for C-systems CC(RR)[LM]. The term C-systems of type theories.

HOMOTOPY TYPE THEORY AND VOEVODSKY S UNIVALENT FOUNDATIONS

Combinatorial Models for M (Lecture 10)

Homotopy Probability Theory in the Univalent Foundations

Derived Algebraic Geometry I: Stable -Categories

Homotopy type theory: towards Grothendieck s dream

Derived Algebraic Geometry IX: Closed Immersions

Derived Algebraic Geometry III: Commutative Algebra

PART II.2. THE!-PULLBACK AND BASE CHANGE

arxiv: v1 [math.lo] 26 Dec 2015

Cubical Type Theory: a constructive interpretation of the univalence axiom

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

The Goldman-Millson theorem revisited

INTRODUCTION TO PART V: CATEGORIES OF CORRESPONDENCES

ON COSTELLO S CONSTRUCTION OF THE WITTEN GENUS: L SPACES AND DG-MANIFOLDS

Algebraic Geometry

Univalent Foundations and the equivalence principle

arxiv: v1 [math.ct] 10 Jul 2016

Grothendieck duality for affine M 0 -schemes.

Lecture 2: Syntax. January 24, 2018

Inductive and higher inductive types

Inductive and higher inductive types

Homotopy type theory: a new connection between logic, category theory and topology

Homotopy Type Theory Lecture Notes

T -spectra. Rick Jardine. March 2, University of Western Ontario

POL502: Foundations. Kosuke Imai Department of Politics, Princeton University. October 10, 2005

THE TOTAL SURGERY OBSTRUCTION III

Notes on Logical Frameworks

Lecture 17: Invertible Topological Quantum Field Theories

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

1. Model existence theorem.

Kathryn Hess. Conference on Algebraic Topology, Group Theory and Representation Theory Isle of Skye 9 June 2009

Algebraic models for higher categories

1 Notations and Statement of the Main Results

Algebraic models for higher categories

De Rham Cohomology. Smooth singular cochains. (Hatcher, 2.1)

Higher Inductive Types as Homotopy-Initial Algebras

Axiomatic set theory. Chapter Why axiomatic set theory?

A Meaning Explanation for HoTT

Completeness for FOL

Higher toposes Internal logic Modalities Sub- -toposes Formalization. Modalities in HoTT. Egbert Rijke, Mike Shulman, Bas Spitters 1706.

We then have an analogous theorem. Theorem 1.2.

58 CHAPTER 2. COMPUTATIONAL METHODS

An inner model from Ω-logic. Daisuke Ikegami

LECTURE 3: RELATIVE SINGULAR HOMOLOGY

MODEL STRUCTURES ON PRO-CATEGORIES

PERVERSE SHEAVES ON A TRIANGULATED SPACE

arxiv: v1 [math.ct] 6 Aug 2017

A model-independent theory of -categories

Three Descriptions of the Cohomology of Bun G (X) (Lecture 4)

Type Theory and Constructive Mathematics. Type Theory and Constructive Mathematics Thierry Coquand. University of Gothenburg

SECTION 5: EILENBERG ZILBER EQUIVALENCES AND THE KÜNNETH THEOREMS

Homology and Cohomology of Stacks (Lecture 7)

Groups and higher groups in homotopy type theory

A categorical model for a quantum circuit description language

Algebraic Cobordism Lecture 1: Complex cobordism and algebraic cobordism

Chern classes à la Grothendieck

The Curry-Howard Isomorphism

Isomorphism is equality

Formalization of Mathematics: why Algebraic Topology?

which is a group homomorphism, such that if W V U, then

APPENDIX C. Groupoids

MULTIPLE DISJUNCTION FOR SPACES OF POINCARÉ EMBEDDINGS

Transcription:

Univalent Foundations and Set Theory Talk by Vladimir Voevodsky from Institute for Advanced Study in Princeton, NJ. May 8, 2013 1

Univalent foundations - are based on a class of formal deduction systems which we currently refer to as homotopy type theories. These theories are extensions of Martin-Lof type theories which are compatible with the univalent model. The univalent model is that which connects univalent foundations with set theoretic foundations and serves as means to ensure that the deduction systems which we construct are at least as consistent as ZFC. The main difficulty in explaining univalent foundations lies in the fact that type theories encompass a wide class of deduction systems which currently does not have a generally accepted definition. 2

Sentences of type systems In a typical type system one works with four kinds of sentences: x 1 : T 1,..., x n : T n T type x 1 : T 1,..., x n : T n t : T x 1 : T 1,..., x n : T n T = T x 1 : T 1,..., x n : T n t = t : T where x 1,..., x n are names of variables and T 1,..., T n, T, t, t are expressions of the system of expressions underlying the type system. 3

Derivation rules Type system is specified by the underlying system of expressions and a collection of derivation rules which show which sentences are derivable in the theory. For example most type systems would have the following derivation rule for sentences of the second kind where the object expression t starts with λ: Γ, x : T o : T Γ λx : T, o : x : T, T the following derivation rule for sentences of the first kind where the type expression starts with Id: Γ o 1 : T Γ o 2 : T Γ Id T o 1 o 2 type 4

h-levels May be the most important feature of homotopy type theories is the notion of h-levels. Given a type expression T in context Γ and an object n of type nat of natural numbers we can write a new type expression isofhlevel n T in Γ. This expressions are defined inductively from the standard type constructors as follows: isofhlevel 0 T = x : T, x : T, Id T, x, x isofhlevel (1 + n) T = x : T, x : T, isofhlevel n (Id T, x, x ) Proving that a type expression is of h-level n means constructing (in a given context) of an object of type isofhlevel n T i.e. deriving a sentence of the form Γ o : isofhlevel n T 5

h-levels (cont.) For example the type nat is provably of h-level 2 which intuitively corresponds to sets and the unit type and empty type are of h-level 1. The univalent model suggests the following interpretation of types of small h-levels: Types of h-level 1 are propositions. Inhabited types of h-level 1 are provable propositions. Thus the proposition as types correspondence is modified in homotopy type theory by interpreting only types of h-level 1 as propositions. Types of h-level 2 are sets. Thus most of mathematics deals with types of h-level 2 and their objects. Types of h-level 3 correspond to groupoids. For example the collection of all finite groups in homotopy type theory is a type of h-level 3. 6

Models of type theories Equivalence classes of sentences of the first and second kind of a type system T modulo the equivalence relations defined by sentences of the third and the fourth kind are denoted B n+1 (T ) and B n (T ) where n is the length of the context. One also formally adds B 0 (T ) which contains one element pt. The properties of sentences such as their ability under substitution e.g. Γ o : S Γ, x : S, Γ T type Γ, Γ [o/x] T [o/x] type define a number partial defined operations on B n s and B n s. With this partially defined operations B-sets of a type theory form a model of a quasi-algebraic theory. 7

Models of type theories (cont.) Derivation rules of a type system add operations and equations to the theory such that ultimately the system of B-sets or B-system of a type theory becomes initial model of a complex quasi-algebraic theory. A model of the type theory is a homomorphism from its B-system to another B-system. Since under the right choice of operations B-sets of a type system form an initial model of a theory constructing a model of a type system is equivalent to constructing a B-system with a list of additional operations and axioms. 8

Models of type theories (cont.) The key machinery for constructing such B-systems is the machinery of categories with universes. Let C be a category and p : Ũ U a morphism. Let us fix a final object pt of C. Let us further fix for any morphism f : X U a pull-back square (X, f) p X,f X (q,f) Ũ f p U and let us write (X, f 1,..., f n ) etc. for the obvious iterated construction. 9

Models of type theories (cont.) Now let B n be the set of sequences (f 1,..., f n ) where f 1 : pt U and f i+1 : (pt, f 1,..., f i ) U and let B n be the set of sequences (f 1,..., f n, g) where (f 1,..., f n ) is as before and g : (pt, f 1,..., f n ) W. One easily constructs a B-system structure on these sets which is determined up to a canonical isomorphism by the equivalence class of (C, p). Let us denote this B-structure as BB(C, p). 10

Models of type theories (cont.) Finally, when C is a locally cartesian closed category, various additional type-theoretic structures of the B-sets corresponding to (C, p) can in all the interesting cases we know of be obtained from natural structures on the morphism p : W W. For example the standard group of structures which correspond to the introduction-elimination rules of the dependent products are generated on BB(C, p) from a pair of morphisms P and P such that the following square is pull-back: Hom U (Ũ, U Ũ Hom U (Ũ,Id U p) P Hom U (Ũ, U U) P Ũ p U 11

Univalent model The current construction of the univalent model for type theory such as that of Coq which assumes an infinite sequence of universes U i : U i+1 is based on C being the category of simplicial sets relative to ZFC with ω + 2 universes. The largest universe is used to define the set of objects of the category of simplicial sets. The next smaller one is used to define p : Ũ U 12

Univalent model (cont.) The formal definition of p : Ũ U is as follows. The set U n of n- simplexes of U is the set of isomorphism classes of Kan fibrations X n given together with well-orderings on the sets X n and such that all X n belongs to one of the universes U 0,..., U i,.... It is easy to see that p itself is a Kan fibration. A much less trivial fact is that U is a Kan simplicial set and that p is a univalent fibration. 13

Univalent model (cont.) In the univalent model a sentence x 1 : T 1,..., x n : T n T interpreted as a tower of fibrations of (Kan) simplicial sets type is [T 1,..., T n, T ] [T 1,..., T n ]... [T 1 ] [pt] and a sentence x 1 : T 1,..., x n : T n t : T as a section of the first fibration in this tower. [t] : [T 1,..., T n ] [T 1,..., T n, T ] 14

Univalent model (cont.) In particular a type expression in the empty context T type is interpreted as a Kan simplicial set and an object of a type in the empty context t : T as a point of the Kan simplicial set corresponding to T. The standard constructors are interpreted as follows: 1. [ x : T, T ] = the simplicial set of sections of the fibration [T, T ] [T ] 2. [ x : T, T ] = [T, T ] 3. [Id T o 1 o 2 ] = simplicial paths from [o 1 ] to [o 2 ] in [T ] 4. [nat] - the usual set of natural numbers considered as a simplicial set. 15

Univalent model (cont.) Most importantly for a universe U i of the type theory the interpretation [U i ] is the simplicial subset of U such that the set of n-simplxes (U i ) n is the set of fibrations X n such that for each m the set of m-simplexes X m of X is in the set-theoretic universe number i. If we define Ũi as the sentence X : U i X type then the obvious projection [Ũi] [U i ] is the universal Kan fibration with fibers in the i-th universe. 16

Univalent model (cont.) One verifies relatively easily that the univalent model maps h-levels of types to levels of homotopy types as follows: 1. types of h-level 0 map to contractible simplicial sets 2. types of h-level 1 map to simplicial sets which are homotopy equivalent to either a point or to the empty set 3. types of h-level 2 map to simplicial sets which are homotopy equivalent to sets 4. types of h-level n+2 map to simplicial sets representing homotopy n-types. 17

Current developments Currently we are developing new type theories more complicated than the standard Martin-Lof type theory and at the same time more convenient for practical formalization of complex mathematics. Such type theories may easily have over a hundred derivation rules. Thus a careful and formalizable approach is needed to show that the newly constructed type theory is at least as consistent as ZFC with a given structure of universes. More precisely we need to be able to formally show that the univalent model extends to these new theories. 18

Current developments (cont.) The first step in the development of the machinery which one needs to be able to verify such statements is Initiality Theorem. The theorem should state that the B-sets of a type system with given set of derivation rules form the initial model of an extension of the quasi-algebraic theory of B-systems extended by operations and equations which are formally read from the derivation rules. So far we do not have even a proper formulation of such a result but all our experience shows that it is possible and that we are moving in the direction where we will be able to state and prove it. 19

Current developments (cont.) The second step in the development of such a machinery should be Operations Theorem which shows how to obtain operations of the kind considered in the Initiality Theorem on B-systems BB(C, p) for locally Cartesian closed categories from structures on p formulated in the internal language of locally Cartesian closed categories. This step is also becoming intuitively more clear. In this step in particular the ideas and language of LF (Logical Framework) appear in a very suggestive way. 20

Conclusion In my vision the more and more complex homotopy type theories will become the languages in which practical unified formalization of all mathematics is done. The set theory will remain the most important benchmark of consistency. The theory of interpretations of type theories in set-theoretic objects will be formalized in relatively simple type theories and each new addition to the practical language will require formal certification by showing, through formally constructed interpretation, that it is at least as consistent as ZFC. 21