Topic 7: Using identity types

Size: px
Start display at page:

Download "Topic 7: Using identity types"

Transcription

1 Toic 7: Using identity tyes June 10, 2014 Now we would like to learn how to use identity tyes and how to do some actual mathematics with them. By now we have essentially introduced all inference rules of HoTT; the main missing ingredient is the univalence axiom. At this stage it is ossible to do a substantial amount of mathematics, and some of this we will do here. Throughout A, B U are fixed tyes. Examle: Proositional uniqueness rinciles Recall the uniqueness rincile for functions, which is an inference rule stating that f λx.f(x) for any (deendent) function f. For other tyes, we did not have such uniqueness rinciles; for examle for u 1, such a uniqueness rincile would assert that u, but we have not ostulated this and it is not derivable. However, at this oint we can show that such a uniqueness rincile holds with roositional equality in lace of judgemental equality: Theorem 1. u 1 u =. The roof of this is exemlative of many other roofs in HoTT. It is a good examle of how one can derive non-trivial equations in HoTT, although the only way to rove an equation is to reduce it in some way to reflexivity. Proof. In order to find an element w u 1 u =, we use induction on u. This reduces the roblem to finding w( ) =, which we can define to be w( ) refl. The same theorem and roof in Coq: Theorem ro_unique : forall u : unit, u = tt. Proof. intro u. induction u. reflexivity. Defined. Analogous roositional uniqueness rinciles can now be derived for many other tyes as well: Theorem 2. x A B x = (r 1 (x), r 2 (x)). Proof. In order to find an element of the tye x A B x = (r 1 (x), r 2 (x)), we use induction on x. This reduces the roblem to finding an element v (a, b) = (r 1 ((a, b)), r 2 ((a, b))). a A b B 1

2 Since r 1 ((a, b)) a and r 2 ((a, b)) b, we can take v λa.λb.refl (a,b). Theorem ro_unique_roduct ( A B : Tye ) : forall x : A * B, x = ( fst x, snd x). Proof. intro x. induction x. siml. reflexivity. Defined. One can generalize this to the deendent air tye: for any deendent tye P A U, one can similarly derive x = (r 1 (x), r 2 (x)) for any x a A P (a). We will rove a more general statement later on, when we characterize the identity tye = q for, q a A P (a). Functions acting on aths If we have x, y A together with x = y and a function f A B, does this yield an element of f(x) = f(y)? In other words, does function alication reserve roositional equality? In terms of the toological interretation, one can say that we now analyse how functions act on aths. Lemma 3. For any function f A B and x, y A, there is a function a f (x = A y) (f(x) = B f(y)) defined such that for all x A, a f (refl x ) refl f(x). Strictly seaking, we also need to consider the two elements x, y A as arguments of the function a f, whose tye therefore should be a f (x = A y) (f(x) = B f(y)). x,y A But since the first two arguments x and y are determined by the third argument x = y, we consider x and y to be imlicit arguments which are not written down exlicitly, excet for in the following roof. Proof. For any x, y A and any x = A y, we want to find a f (x, y, ) f(x) = B f(y). By induction on as an element of the (say, unbased) identity tye, it is sufficient to do so in the case that y x and refl x. But in this case, we can ut a f (x, x, refl x ) refl f(x) f(x) = B f(x). In Coq, the statement and roof look as follows: Lemma a { A B : Tye } ( f : A B) : forall x y : A, ( x = y) ( f( x) = f( y)). Proof. intros x y. induction. reflexivity. Defined. We interret Lemma 3 as saying that every function f is automatically continuous, since it mas aths to aths! So in HoTT, it is imossible to construct a function that is not continuous. 2

3 Examle: commutativity of addition As the ossibly first examle of actual mathematics in HoTT, let us revisit the natural numbers and rove that addition is commutative. The following roof structure coincides exactly with how one would rove commutativity of addition in conventional foundations! This is true for many other things as well. Lemma 4. x,y N succ(y + x) = y + succ(x). Recall that we had defined addition x+y add(x, y) by induction over the first argument, using the definitions add(0, y) y and add(succ(x), y) succ(add(x, y)). Proof. In order to find an element of the tye succ(y + x) = y + succ(x) for any x, y N, we can use induction on y. For y 0, we have refl succ(x) succ(x) = succ(x), and by the definition of + we also have judgemental equalities succ(0 + x) succ(x) and 0 + succ(x) succ(x). Therefore, we also have refl succ(x) succ(0 + x) = 0 + succ(x). For the induction ste, we need to show that one can construct an element of the identity tye succ(succ(y) + x) = succ(y) + succ(x) from any given element v succ(y + x) = y + succ(x). Since a succ (v) succ(succ(y + x)) = succ(y + succ(x)) and we have judgemental equalities succ(succ(y) + x) succ(succ(y + x)), succ(y) + succ(x) succ(y + succ(x)) by the definition of +, we also have a succ (v) succ(succ(y) + x) = succ(y) + succ(x). Let us write add succ x,y N y + succ(x) = succ(y + x) for the element constructed in the roof. The same statement and roof in Coq: Lemma add_succ : forall x y : nat, x + S y = S ( x + y). Proof. intros x y. induction x. siml. reflexivity. Defined. siml. aly (a S). exact IHx. Theorem 5. x,y N x + y = y + x. Proof. In order to find an element of the tye x + y = y + x for any x and y, we can use induction on x. This reduces the roblem to finding elements of the following two tyes: 0 + y = y + 0, (x + y = y + x) (succ(x) + y = y + succ(x)) We start with the first. Since + was defined by induction over the first argument, we have 0 + y y, so it remains to show that y = y + 0. This in turn can be shown by induction on y as follows. For y 0, we have again by definition of +, and hence we have a judgemental equality of tyes 3

4 (0 = 0) (0 = 0 + 0), and therefore refl 0 0 = Concerning the induction ste, if we have an equality witness w y = y + 0, then we obtain a succ (w) succ(y) = succ(y + 0). Since succ(y) + 0 succ(y + 0) by the inductive definition of +, we also have a succ (w) succ(y) = succ(y) + 0. Now for the main induction ste. Suose that we have v x + y = y + x, and we want to find an element of succ(x) + y = y + succ(x). For every y, we have a succ (v) succ(x) + y = succ(y + x), where we have used succ(x + y) succ(x) + y by the inductive definition of +, and add succ(x, y) succ(y + x) = y + succ(x) thanks to Lemma 4. The claim now follows from transitivity of equality; this is what we get to next. Concatenating aths Last time, we already saw that roositional equality is symmetric, in the sense that there exists a canonical function (x = y) (y = x) which mas any ath x = y to its inverse 1 y = x. In the ath interretation, this corresonds to the fact that every ath can be traversed forwards or backwards. Recall that taking the inverse is a function 1 (x = y) (y = x) x,y A which can be defined by (based or unbased) ath induction, which reduces the roblem to defining the function on y x and refl x, in which case we define the function value to be refl x itself. Although x and y (and even A) should formally also be considered as arguments of this function, we omit them for brevity; if one knows, one can deduce x and y from the tye of, and then A as the tye of x and y. To summarize, the function 1 is defined by ath induction on, together with the stiulation that refl 1 x refl x for every x A. Similarly, it is ossible to concatenate aths: if is a ath from x to y and q is a ath from y to z, then there is a concatenated ath q from x to z. This is indeed the case: for any A U, one can construct a function (x = y) (y = z) (x = z) (1) x,y,z A as follows. By ermuting the z argument with the (x = y)-argument, it is enough to construct this function in the form (x = y) (y = z) (x = z). x,y z A Alying (unbased) ath induction lets us assume that we are dealing with the case y x and refl x x = x, in which case we simly need to construct an element of the tye (x = z) (x = z), z A for which we could simly take the identity function for every z. However, it turns out to be better to not use the identity function here, but rather to define such a function again through ath 4

5 induction, which allows us to ut z x and assume refl x x = x, in which case we take the value of the function to again be refl x x = x. The reason for not using the identity function, but instead using another ath induction, is mainly aesthetics: with the identity function, the resulting comutation rule for is, refl x q q for all q y = z, while with a second ath induction, the comutation rule is merely refl x refl x refl x, which we refer, since it makes both arguments behave in the same way. In logical terms, one can interret (1) as the transitivity of equality: if x is equal to y and y is equal to z, then x is also equal to z. The function (1) can be interreted as converting any two roofs x = y and q y = z into q x = z. Generally seaking, thinking in terms of aths between oints in a sace rather than roofs of equalities is the referred intuition, and so we stick with this one from now on. Theorem 6. Concatenation of aths is associative: for any w, x, y, z A and w = x, q x = y, r y = z, (q r) = ( q) r. Strictly seaking, what me mean by this theorem is that we claim to be able to construct an element of the tye (q r) = ( q) r, (2) w=x q x=y r y=z A U w,x,y,z A and this is what will be done in the roof. Proof. We use similar arguments as in the construction of : ermuting some of the arameters w, x, y, z and, q, r and then alying ath induction. Indeed, ath induction over allows us to assume x w and refl w, in which case we have q w = y and r y = z and need to rove refl w (q r) = (refl w q) r. We show this by another ath induction, this time on q, which gives y w and q refl w, so that we have reduced the roblem to finding an element of refl w (refl w r) = (refl w refl w ) r. Using the same kind of ath induction for r and alying the comutation rule refl w refl w refl w results in the assertion refl w = refl w, which has a trivial roof given by refl reflw. This result is our first coherence law. Generally seaking, a coherence law states that any two ways to construct a new object from given data are equal. In this case, it states that the concatenation of a sequence of aths does not deend on the order in which these aths are concatenated at least u to roositional equality. The element of the above tye (2) can be shown to satisfy its own coherence law! There is also a sense in which the reflexivity elements are unit elements for the concatenation of aths, in the sense that concatenating with them gives the other ath back of course, again u to roositional equality: 5

6 Theorem 7. For any x, y A and x = y, refl x =, refl y =. Finally, in the same sense, concatenating a ath with its inverse recovers the reflexivity elements: Theorem 8. For any x, y A and x = y, 1 = refl x, 1 = refl y. Both theorems can easily be roven by ath induction on. The concatenation of aths is an algebraic structure on all the identity tyes over any tye A which turns A into a so-called grouoid. Can similar things also be done with higher aths, i.e. with elements of identity tyes between aths, identities between those, and so on? Before getting to this, we briefly study how the algebraic structure on aths interacts with the a function from Lemma 3. Theorem 9. The function a has the following roerties: 1. a f ( q) = a f () a f (q), 2. a f ( 1 ) = a f () 1, 3. For f A B and g B C, we have a g f () = a g (a f ()). 4. a ida () =. Proof. All these roerties follow from ath induction on (and q). Concerning the latter two items, it would be helful to have the stronger statements that a g f = a g a f, and likewise a ida = id x=y. However, roving these statements would require to be able to conclude that two functions are equal as soon as they take on equal values on all oints; this is something which we cannot rove yet! A natural question now is, what haens if instead of f A B we consider a deendent function f x A B(x)? In this case, things are a bit more comlicated: if we have x = A y, then f(x) B(x) and f(y) B(y), so that it does not actually make sense to assert that f(x) = f(y). So, before solving this uzzle, we need to understand deendent tyes a little better; we consider this below. Tyes as higher grouoids For aths, q x = y, we can also consider a ath between these aths, α = q. More rigorously, we should indicate the base tye over which the identity tye = q is formed, and then we have to write α = x=a y q. We will also call such a ath between aths a 2-ath. Suose that we have, in addition to this data, also another ath r y = z. Geometrically, the situation looks like this: x q α y r z 6

7 Using ath induction on r, we can concatenate this data to a 2-ath of tye r = q r which we denote by α r, x r q r More recisely, there is a function which concatenates any 2-ath to any 1-ath in the sense of having the tye ( r) = (q r). A U x,y,z A,q x=y α =q r y=z Again, we only consider α and r as the arguments of this function, since the others can be deduced. Similarly, if we are given another w A and o w = x as in α r z w o x q α y then we can likewise use ath induction on o in order to define a new 2-ath o α o = o q. What oerations can we construct which concatenate two 2-aths to a new 2-ath? For one, if we have r,, q x = y and α = q and β q = r like this, x q r α β y then we already know that we can form the concatenation α β = r. Since this is only one kind of concatenation of 2-aths, it is usually called the vertical concatenation, due to how the α and β are arranged in the diagram above. On the other hand, if we have this situation, x q α y r s β z we can also construct a horizontal concatenation by defining α β (α r) (q β), which is of tye ( r) = (q s). Alternatively, it would also have been ossible to define this horizontal concatenation as ( β) (α s); the result would have been again equal, since one can find an element of the identity tye by using several consecutive ath inductions. (α r) (q β) = ( β) (α s) 7

8 Theorem 10. (Exchange law) In a situation like this, o r x q α β y s t γ δ z we have (α β) (γ δ) = (α γ) (β δ). Proof. As usual, we aly ath induction, this time on α, β, γ and δ, which reduces the roblem to this case: s x refl refl y s s refl s refl s z In this case, the desired equality is (refl refl ) (refl s refl s ) = (refl refl s ) (refl refl s ). Since we have refl refl refl, and similar for refl s and (refl refl s ), this simlifies to refl refl s = refl refl s, which is true again by reflexivity. There are many more oerations on higher-dimensional aths which can be constructed by ath induction. We will sto our short discussion of this asect by noting that all these higher oerations can be regarded as one ossible definition of an algebraic structure called an -grouoid. Deendent tyes as fibrations We already learnt that we can think of a tye A as a sace with elements x A as oints and equalities x = y as aths. We also just realized that a function f A B can be interreted as a continuous ma from the sace A to the sace B. Now suose that we aly this in the case B U. So, the universe U is itself a gigantic sace whose elements are themselves other saces. (Such a sace of saces is often also called a moduli sace.) So, a deendent tye over A or tye family over A is a function D A U; intuitively, this means that D assigns to every x A another sace D(x) U in a way which deends continuously on x. Conventionally, such a deendent sace is known as a fibration; so, a tye family is the HoTT analogue of the notion of fibration. As an examle, if we start with the base sace A being a circle, and attach to each x A a coy of the interval, such that as we go once around the circle, the interval comes back with a twist, then we obtain the Möbius stri of Figure 1. What is deicted is not the function D A U, but rather the total sace x A D(x), which is the union of 8

9 Figure 1: A Möbius stri all the individual D(x). One can identify the circle S 1 with the central line that winds around the stri; for every x, the sace D(x) then consists of the interval erendicular to that circle. Higher inductive tyes will let us ermit the definition of a tye modelling the circle and a tye modelling the interval, and then the Möbius stri will be an actual tye family that we can construct. Until then, it is nothing but an illustration. So, the deendent sum x A D(x) corresonds to the total sace of the fibration D A U; but what about the deendent roduct x A D(x)? Intuitively, an element s x A D(x) corresonds to an assignment x s(x) with s(x) D(x) such that the deendence on x is continuous. Under the corresondence to fibrations, such an s is conventionally known as a section. The Möbius stri is very secial in that it ermits a section which embeds the circle as the base into the total sace x A D(x); in general, this is not the case. With this intuition in mind, we can now move on to discussing the behavior of aths with resect to such fibrations. Theorem 11. Given a tye family D A U over A and a ath x = A y, there exists a function transort D () D(x) D(y). Proof. Path induction on, using the definition transort D (refl x ) id D(x). Whenever the tye family D is clear, then we also use the shorthand notation D(x) D(y) in lace of transort D (). If D A U is interreted as a roosition deending on x A, then we can say that x A has roerty D if D(x) is inhabited. Therefore, the theorem tells us that if x is equal to y, and x has roerty D, then so does y. More recisely, any witness or roof of the statement x has roerty D can be transorted into a witness or roof of the statement y has roerty D. In the toological theory of fibrations, the transort function can be interreted as a connection, which is a fundamental structure in differential geometry. In this sense, a tye family is more than just a fibration: it is a fibration equied with a connection. Imortant roerties of the transort function are the following, which are all easily roven by the usual ath induction: 9

10 Theorem 12. If q y = z is another ath, then for all t D(x). ( q) (t) = q ( (t)) So the transort ma has the exected behaviour uon concatenation of aths; note the similarity to the revious theorem a f (q ) = a f (q) a f (). Using transort, we can not only transort elements around, we can also transort aths themselves, a transort D (s = t) ( (s) = (t)). (3) s,t D(x) The behaviour of transort with resect to changing the base tye A is like this: Theorem 13. If f B A is a function, then D f B U is again a tye family, and for all x = B y with x, y B, and t D(f(x)). transort D f (, t) = transort D (a f (), t). Finally, we also note the behaviour of transort with resect to changing the tye family, while keeing the base A fixed: Theorem 14. Given any two tye families D, E A U and a family of deendent functions f x A D(x) E(x) and any x = A y and t D(x), we have transort E (, f(x, t)) = f(y, transort D (, t)). We can exress this as saying that transort commutes with the alication of a deendent function. In terms of category theory, f is a transformation between functors, and the theorem shows that this transformation is automatically natural. This is similar to how Lemma 3 shows that every function is automatically continuous. If we aly transort in the case of a non-deendent tye, it acts trivially: Theorem 15. If D λx.b A U for some fixed B U, then for any x, y A and x = A y there is a family of aths transortconst B () transort λx.b (, t) = t t B We are now in a situation to generalize the function a (x = y) (f(x) = f(y)) to the case in which f is a deendent function, by simly transorting f(x) from D(x) to D(y) before comaring it to f(y): Theorem 16. Given any deendent function f x A D(x), there exists a function ad f (f(x)) = D(y) f(y). x=y Again we consider the elements x, y A to be imlicit arguments of ad f for which we omit mention. The roof of the theorem is again straightforward by ath induction on. While the revious a was a function (x = y) (f(x) = f(y)), the new ad f for deendent f is itself a deendent function. Also ad f has the exected behaviour with resect to concatenation of aths, and more generally there are more comlicated analogues of Theorem 9, but we omit these. When f is a non-deendent function, we would exect ad f to reduce to a f, assuming that we identify f A B with the corresonding element of x A B. This is indeed the case: 10

11 Theorem 17. For all f A B and x = A y, we have ad f () = transortconst B (, f(x)) a f (). The is well-tyed since the ath on the left goes from transort λx.b (, f(x)) to f(y), while the one on the right is a concatenation of a ath from transort λx.b (, f(x)) to f(x) and a ath from f(x) to f(y). As usual, the roof is by ath induction on, in which case both sides reduce to refl f(x). Path lifting The revious considerations involving transort were about turning a ath x = y on the base A into a function transort D () D(x) D(y). But can we also lift a ath in the base to a ath in D? In order to make sense of this, we need to consider aths in the total sace x A D(x), and then we have: Theorem 18 (Path lifting roerty). For any x A and t D(x), every ath x = A y gives a ath and this ath lies over in the sense that lift(t, ) (x, t) = x A D(x) (y, (t)), a r1 (lift(t, )) =. Proof. Using ath induction on reduces the roof of both statements to the case y x and refl x, for which they are trivial. Omniotent ath induction? The revious results may suggest that ath induction is a roof method with which one can rove almost anything, since it always reduces the roof to a trivial case. However, this is by no means the case: for examle, the statement = refl x (4) x A x=x is not derivable by ath induction. In fact, ath induction does not aly here since it would require at least one endoint of to be free based ath induction alies to statements of the form x A x=y C(x, y, ) only! We will see soon that together with the univalence axiom, one can show (4) to be false. Actually, (4) is closely related to Axiom K, which is a commonly imosed axiom resulting in so-called extensional tye theory, in which two things can be equal in at most one way. Due to the incomatibility with the univalence axiom, and the realization that univalence is a more owerful rincile resulting in a foundation of mathematics close to mathematical ractice, we do not imose Axiom K. 11

12 Examle: discriminating the elements of Bool In order to illustrate the use of the results derived here, we show that the two canonical elements of Bool are not equal: Theorem 19. (0 = 1) 0. Proof. Define the tye family D Bool U by induction over Bool using the values D(0) 0, D(1) 1 on the base cases. We know that D(1) is inhabited by D(1). Hence for any utative equation 0 = 1, we have ( 1 ) ( ) D(0), which is an element of 0 since D(0) 0. 12

SECTION 5: FIBRATIONS AND HOMOTOPY FIBERS

SECTION 5: FIBRATIONS AND HOMOTOPY FIBERS SECTION 5: FIBRATIONS AND HOMOTOPY FIBERS In this section we will introduce two imortant classes of mas of saces, namely the Hurewicz fibrations and the more general Serre fibrations, which are both obtained

More information

MATH 2710: NOTES FOR ANALYSIS

MATH 2710: NOTES FOR ANALYSIS MATH 270: NOTES FOR ANALYSIS The main ideas we will learn from analysis center around the idea of a limit. Limits occurs in several settings. We will start with finite limits of sequences, then cover infinite

More information

Various Proofs for the Decrease Monotonicity of the Schatten s Power Norm, Various Families of R n Norms and Some Open Problems

Various Proofs for the Decrease Monotonicity of the Schatten s Power Norm, Various Families of R n Norms and Some Open Problems Int. J. Oen Problems Comt. Math., Vol. 3, No. 2, June 2010 ISSN 1998-6262; Coyright c ICSRS Publication, 2010 www.i-csrs.org Various Proofs for the Decrease Monotonicity of the Schatten s Power Norm, Various

More information

HENSEL S LEMMA KEITH CONRAD

HENSEL S LEMMA KEITH CONRAD HENSEL S LEMMA KEITH CONRAD 1. Introduction In the -adic integers, congruences are aroximations: for a and b in Z, a b mod n is the same as a b 1/ n. Turning information modulo one ower of into similar

More information

DIFFERENTIAL GEOMETRY. LECTURES 9-10,

DIFFERENTIAL GEOMETRY. LECTURES 9-10, DIFFERENTIAL GEOMETRY. LECTURES 9-10, 23-26.06.08 Let us rovide some more details to the definintion of the de Rham differential. Let V, W be two vector bundles and assume we want to define an oerator

More information

δ(xy) = φ(x)δ(y) + y p δ(x). (1)

δ(xy) = φ(x)δ(y) + y p δ(x). (1) LECTURE II: δ-rings Fix a rime. In this lecture, we discuss some asects of the theory of δ-rings. This theory rovides a good language to talk about rings with a lift of Frobenius modulo. Some of the material

More information

Why Proofs? Proof Techniques. Theorems. Other True Things. Proper Proof Technique. How To Construct A Proof. By Chuck Cusack

Why Proofs? Proof Techniques. Theorems. Other True Things. Proper Proof Technique. How To Construct A Proof. By Chuck Cusack Proof Techniques By Chuck Cusack Why Proofs? Writing roofs is not most student s favorite activity. To make matters worse, most students do not understand why it is imortant to rove things. Here are just

More information

Quaternionic Projective Space (Lecture 34)

Quaternionic Projective Space (Lecture 34) Quaternionic Projective Sace (Lecture 34) July 11, 2008 The three-shere S 3 can be identified with SU(2), and therefore has the structure of a toological grou. In this lecture, we will address the question

More information

Sets of Real Numbers

Sets of Real Numbers Chater 4 Sets of Real Numbers 4. The Integers Z and their Proerties In our revious discussions about sets and functions the set of integers Z served as a key examle. Its ubiquitousness comes from the fact

More information

Mobius Functions, Legendre Symbols, and Discriminants

Mobius Functions, Legendre Symbols, and Discriminants Mobius Functions, Legendre Symbols, and Discriminants 1 Introduction Zev Chonoles, Erick Knight, Tim Kunisky Over the integers, there are two key number-theoretic functions that take on values of 1, 1,

More information

Section 0.10: Complex Numbers from Precalculus Prerequisites a.k.a. Chapter 0 by Carl Stitz, PhD, and Jeff Zeager, PhD, is available under a Creative

Section 0.10: Complex Numbers from Precalculus Prerequisites a.k.a. Chapter 0 by Carl Stitz, PhD, and Jeff Zeager, PhD, is available under a Creative Section 0.0: Comlex Numbers from Precalculus Prerequisites a.k.a. Chater 0 by Carl Stitz, PhD, and Jeff Zeager, PhD, is available under a Creative Commons Attribution-NonCommercial-ShareAlike.0 license.

More information

DRAFT - do not circulate

DRAFT - do not circulate An Introduction to Proofs about Concurrent Programs K. V. S. Prasad (for the course TDA383/DIT390) Deartment of Comuter Science Chalmers University Setember 26, 2016 Rough sketch of notes released since

More information

MA3H1 TOPICS IN NUMBER THEORY PART III

MA3H1 TOPICS IN NUMBER THEORY PART III MA3H1 TOPICS IN NUMBER THEORY PART III SAMIR SIKSEK 1. Congruences Modulo m In quadratic recirocity we studied congruences of the form x 2 a (mod ). We now turn our attention to situations where is relaced

More information

An Overview of Witt Vectors

An Overview of Witt Vectors An Overview of Witt Vectors Daniel Finkel December 7, 2007 Abstract This aer offers a brief overview of the basics of Witt vectors. As an alication, we summarize work of Bartolo and Falcone to rove that

More information

Elementary Analysis in Q p

Elementary Analysis in Q p Elementary Analysis in Q Hannah Hutter, May Szedlák, Phili Wirth November 17, 2011 This reort follows very closely the book of Svetlana Katok 1. 1 Sequences and Series In this section we will see some

More information

RECIPROCITY LAWS JEREMY BOOHER

RECIPROCITY LAWS JEREMY BOOHER RECIPROCITY LAWS JEREMY BOOHER 1 Introduction The law of uadratic recirocity gives a beautiful descrition of which rimes are suares modulo Secial cases of this law going back to Fermat, and Euler and Legendre

More information

THE 2D CASE OF THE BOURGAIN-DEMETER-GUTH ARGUMENT

THE 2D CASE OF THE BOURGAIN-DEMETER-GUTH ARGUMENT THE 2D CASE OF THE BOURGAIN-DEMETER-GUTH ARGUMENT ZANE LI Let e(z) := e 2πiz and for g : [0, ] C and J [0, ], define the extension oerator E J g(x) := g(t)e(tx + t 2 x 2 ) dt. J For a ositive weight ν

More information

Feedback-error control

Feedback-error control Chater 4 Feedback-error control 4.1 Introduction This chater exlains the feedback-error (FBE) control scheme originally described by Kawato [, 87, 8]. FBE is a widely used neural network based controller

More information

Elementary theory of L p spaces

Elementary theory of L p spaces CHAPTER 3 Elementary theory of L saces 3.1 Convexity. Jensen, Hölder, Minkowski inequality. We begin with two definitions. A set A R d is said to be convex if, for any x 0, x 1 2 A x = x 0 + (x 1 x 0 )

More information

A review of the foundations of perfectoid spaces

A review of the foundations of perfectoid spaces A review of the foundations of erfectoid saces (Notes for some talks in the Fargues Fontaine curve study grou at Harvard, Oct./Nov. 2017) Matthew Morrow Abstract We give a reasonably detailed overview

More information

Real Analysis 1 Fall Homework 3. a n.

Real Analysis 1 Fall Homework 3. a n. eal Analysis Fall 06 Homework 3. Let and consider the measure sace N, P, µ, where µ is counting measure. That is, if N, then µ equals the number of elements in if is finite; µ = otherwise. One usually

More information

On the Rank of the Elliptic Curve y 2 = x(x p)(x 2)

On the Rank of the Elliptic Curve y 2 = x(x p)(x 2) On the Rank of the Ellitic Curve y = x(x )(x ) Jeffrey Hatley Aril 9, 009 Abstract An ellitic curve E defined over Q is an algebraic variety which forms a finitely generated abelian grou, and the structure

More information

p-adic Measures and Bernoulli Numbers

p-adic Measures and Bernoulli Numbers -Adic Measures and Bernoulli Numbers Adam Bowers Introduction The constants B k in the Taylor series exansion t e t = t k B k k! k=0 are known as the Bernoulli numbers. The first few are,, 6, 0, 30, 0,

More information

Math 104B: Number Theory II (Winter 2012)

Math 104B: Number Theory II (Winter 2012) Math 104B: Number Theory II (Winter 01) Alina Bucur Contents 1 Review 11 Prime numbers 1 Euclidean algorithm 13 Multilicative functions 14 Linear diohantine equations 3 15 Congruences 3 Primes as sums

More information

RANDOM WALKS AND PERCOLATION: AN ANALYSIS OF CURRENT RESEARCH ON MODELING NATURAL PROCESSES

RANDOM WALKS AND PERCOLATION: AN ANALYSIS OF CURRENT RESEARCH ON MODELING NATURAL PROCESSES RANDOM WALKS AND PERCOLATION: AN ANALYSIS OF CURRENT RESEARCH ON MODELING NATURAL PROCESSES AARON ZWIEBACH Abstract. In this aer we will analyze research that has been recently done in the field of discrete

More information

LECTURE 6: FIBER BUNDLES

LECTURE 6: FIBER BUNDLES LECTURE 6: FIBER BUNDLES In this section we will introduce the interesting class o ibrations given by iber bundles. Fiber bundles lay an imortant role in many geometric contexts. For examle, the Grassmaniann

More information

GOOD MODELS FOR CUBIC SURFACES. 1. Introduction

GOOD MODELS FOR CUBIC SURFACES. 1. Introduction GOOD MODELS FOR CUBIC SURFACES ANDREAS-STEPHAN ELSENHANS Abstract. This article describes an algorithm for finding a model of a hyersurface with small coefficients. It is shown that the aroach works in

More information

Multiplicative group law on the folium of Descartes

Multiplicative group law on the folium of Descartes Multilicative grou law on the folium of Descartes Steluţa Pricoie and Constantin Udrişte Abstract. The folium of Descartes is still studied and understood today. Not only did it rovide for the roof of

More information

On Isoperimetric Functions of Probability Measures Having Log-Concave Densities with Respect to the Standard Normal Law

On Isoperimetric Functions of Probability Measures Having Log-Concave Densities with Respect to the Standard Normal Law On Isoerimetric Functions of Probability Measures Having Log-Concave Densities with Resect to the Standard Normal Law Sergey G. Bobkov Abstract Isoerimetric inequalities are discussed for one-dimensional

More information

SECTION 12: HOMOTOPY EXTENSION AND LIFTING PROPERTY

SECTION 12: HOMOTOPY EXTENSION AND LIFTING PROPERTY SECTION 12: HOMOTOPY EXTENSION AND LIFTING PROPERTY In the revious section, we exloited the interlay between (relative) CW comlexes and fibrations to construct the Postnikov and Whitehead towers aroximating

More information

Stone Duality for Skew Boolean Algebras with Intersections

Stone Duality for Skew Boolean Algebras with Intersections Stone Duality for Skew Boolean Algebras with Intersections Andrej Bauer Faculty of Mathematics and Physics University of Ljubljana Andrej.Bauer@andrej.com Karin Cvetko-Vah Faculty of Mathematics and Physics

More information

4. Score normalization technical details We now discuss the technical details of the score normalization method.

4. Score normalization technical details We now discuss the technical details of the score normalization method. SMT SCORING SYSTEM This document describes the scoring system for the Stanford Math Tournament We begin by giving an overview of the changes to scoring and a non-technical descrition of the scoring rules

More information

MATH 361: NUMBER THEORY ELEVENTH LECTURE

MATH 361: NUMBER THEORY ELEVENTH LECTURE MATH 361: NUMBER THEORY ELEVENTH LECTURE The subjects of this lecture are characters, Gauss sums, Jacobi sums, and counting formulas for olynomial equations over finite fields. 1. Definitions, Basic Proerties

More information

Practice Final Solutions

Practice Final Solutions Practice Final Solutions 1. True or false: (a) If a is a sum of three squares, and b is a sum of three squares, then so is ab. False: Consider a 14, b 2. (b) No number of the form 4 m (8n + 7) can be written

More information

Chapter 6. Phillip Hall - Room 537, Huxley

Chapter 6. Phillip Hall - Room 537, Huxley Chater 6 6 Partial Derivatives.................................................... 72 6. Higher order artial derivatives...................................... 73 6.2 Matrix of artial derivatives.........................................74

More information

1 Gambler s Ruin Problem

1 Gambler s Ruin Problem Coyright c 2017 by Karl Sigman 1 Gambler s Ruin Problem Let N 2 be an integer and let 1 i N 1. Consider a gambler who starts with an initial fortune of $i and then on each successive gamble either wins

More information

CMSC 425: Lecture 4 Geometry and Geometric Programming

CMSC 425: Lecture 4 Geometry and Geometric Programming CMSC 425: Lecture 4 Geometry and Geometric Programming Geometry for Game Programming and Grahics: For the next few lectures, we will discuss some of the basic elements of geometry. There are many areas

More information

Sums of independent random variables

Sums of independent random variables 3 Sums of indeendent random variables This lecture collects a number of estimates for sums of indeendent random variables with values in a Banach sace E. We concentrate on sums of the form N γ nx n, where

More information

arxiv:math/ v4 [math.gn] 25 Nov 2006

arxiv:math/ v4 [math.gn] 25 Nov 2006 arxiv:math/0607751v4 [math.gn] 25 Nov 2006 On the uniqueness of the coincidence index on orientable differentiable manifolds P. Christoher Staecker October 12, 2006 Abstract The fixed oint index of toological

More information

A CONCRETE EXAMPLE OF PRIME BEHAVIOR IN QUADRATIC FIELDS. 1. Abstract

A CONCRETE EXAMPLE OF PRIME BEHAVIOR IN QUADRATIC FIELDS. 1. Abstract A CONCRETE EXAMPLE OF PRIME BEHAVIOR IN QUADRATIC FIELDS CASEY BRUCK 1. Abstract The goal of this aer is to rovide a concise way for undergraduate mathematics students to learn about how rime numbers behave

More information

CHAPTER 5 TANGENT VECTORS

CHAPTER 5 TANGENT VECTORS CHAPTER 5 TANGENT VECTORS In R n tangent vectors can be viewed from two ersectives (1) they cature the infinitesimal movement along a ath, the direction, and () they oerate on functions by directional

More information

2 Asymptotic density and Dirichlet density

2 Asymptotic density and Dirichlet density 8.785: Analytic Number Theory, MIT, sring 2007 (K.S. Kedlaya) Primes in arithmetic rogressions In this unit, we first rove Dirichlet s theorem on rimes in arithmetic rogressions. We then rove the rime

More information

2 Asymptotic density and Dirichlet density

2 Asymptotic density and Dirichlet density 8.785: Analytic Number Theory, MIT, sring 2007 (K.S. Kedlaya) Primes in arithmetic rogressions In this unit, we first rove Dirichlet s theorem on rimes in arithmetic rogressions. We then rove the rime

More information

Analysis of some entrance probabilities for killed birth-death processes

Analysis of some entrance probabilities for killed birth-death processes Analysis of some entrance robabilities for killed birth-death rocesses Master s Thesis O.J.G. van der Velde Suervisor: Dr. F.M. Sieksma July 5, 207 Mathematical Institute, Leiden University Contents Introduction

More information

DISCRIMINANTS IN TOWERS

DISCRIMINANTS IN TOWERS DISCRIMINANTS IN TOWERS JOSEPH RABINOFF Let A be a Dedekind domain with fraction field F, let K/F be a finite searable extension field, and let B be the integral closure of A in K. In this note, we will

More information

On the Toppling of a Sand Pile

On the Toppling of a Sand Pile Discrete Mathematics and Theoretical Comuter Science Proceedings AA (DM-CCG), 2001, 275 286 On the Toling of a Sand Pile Jean-Christohe Novelli 1 and Dominique Rossin 2 1 CNRS, LIFL, Bâtiment M3, Université

More information

Fibration of Toposes PSSL 101, Leeds

Fibration of Toposes PSSL 101, Leeds Fibration of Tooses PSSL 101, Leeds Sina Hazratour sinahazratour@gmail.com Setember 2017 AUs AUs as finitary aroximation of Grothendieck tooses Pretooses 1 finite limits 2 stable finite disjoint coroducts

More information

POINTS ON CONICS MODULO p

POINTS ON CONICS MODULO p POINTS ON CONICS MODULO TEAM 2: JONGMIN BAEK, ANAND DEOPURKAR, AND KATHERINE REDFIELD Abstract. We comute the number of integer oints on conics modulo, where is an odd rime. We extend our results to conics

More information

Lecture 6. 2 Recurrence/transience, harmonic functions and martingales

Lecture 6. 2 Recurrence/transience, harmonic functions and martingales Lecture 6 Classification of states We have shown that all states of an irreducible countable state Markov chain must of the same tye. This gives rise to the following classification. Definition. [Classification

More information

Math 4400/6400 Homework #8 solutions. 1. Let P be an odd integer (not necessarily prime). Show that modulo 2,

Math 4400/6400 Homework #8 solutions. 1. Let P be an odd integer (not necessarily prime). Show that modulo 2, MATH 4400 roblems. Math 4400/6400 Homework # solutions 1. Let P be an odd integer not necessarily rime. Show that modulo, { P 1 0 if P 1, 7 mod, 1 if P 3, mod. Proof. Suose that P 1 mod. Then we can write

More information

19th Bay Area Mathematical Olympiad. Problems and Solutions. February 28, 2017

19th Bay Area Mathematical Olympiad. Problems and Solutions. February 28, 2017 th Bay Area Mathematical Olymiad February, 07 Problems and Solutions BAMO- and BAMO- are each 5-question essay-roof exams, for middle- and high-school students, resectively. The roblems in each exam are

More information

Extension of Minimax to Infinite Matrices

Extension of Minimax to Infinite Matrices Extension of Minimax to Infinite Matrices Chris Calabro June 21, 2004 Abstract Von Neumann s minimax theorem is tyically alied to a finite ayoff matrix A R m n. Here we show that (i) if m, n are both inite,

More information

A Social Welfare Optimal Sequential Allocation Procedure

A Social Welfare Optimal Sequential Allocation Procedure A Social Welfare Otimal Sequential Allocation Procedure Thomas Kalinowsi Universität Rostoc, Germany Nina Narodytsa and Toby Walsh NICTA and UNSW, Australia May 2, 201 Abstract We consider a simle sequential

More information

Almost 4000 years ago, Babylonians had discovered the following approximation to. x 2 dy 2 =1, (5.0.2)

Almost 4000 years ago, Babylonians had discovered the following approximation to. x 2 dy 2 =1, (5.0.2) Chater 5 Pell s Equation One of the earliest issues graled with in number theory is the fact that geometric quantities are often not rational. For instance, if we take a right triangle with two side lengths

More information

ALGEBRAIC TOPOLOGY MASTERMATH (FALL 2014) Written exam, 21/01/2015, 3 hours Outline of solutions

ALGEBRAIC TOPOLOGY MASTERMATH (FALL 2014) Written exam, 21/01/2015, 3 hours Outline of solutions ALGERAIC TOPOLOGY MASTERMATH FALL 014) Written exam, 1/01/015, 3 hours Outline of solutions Exercise 1. i) There are various definitions in the literature. ased on the discussion on. 5 of Lecture 3, as

More information

B8.1 Martingales Through Measure Theory. Concept of independence

B8.1 Martingales Through Measure Theory. Concept of independence B8.1 Martingales Through Measure Theory Concet of indeendence Motivated by the notion of indeendent events in relims robability, we have generalized the concet of indeendence to families of σ-algebras.

More information

1. INTRODUCTION. Fn 2 = F j F j+1 (1.1)

1. INTRODUCTION. Fn 2 = F j F j+1 (1.1) CERTAIN CLASSES OF FINITE SUMS THAT INVOLVE GENERALIZED FIBONACCI AND LUCAS NUMBERS The beautiful identity R.S. Melham Deartment of Mathematical Sciences, University of Technology, Sydney PO Box 23, Broadway,

More information

Chapter 7 Rational and Irrational Numbers

Chapter 7 Rational and Irrational Numbers Chater 7 Rational and Irrational Numbers In this chater we first review the real line model for numbers, as discussed in Chater 2 of seventh grade, by recalling how the integers and then the rational numbers

More information

Homotopy Type Theory Lecture Notes

Homotopy Type Theory Lecture Notes 15-819 Homotopy Type Theory Lecture Notes Nathan Fulton October 9 and 11, 2013 1 Contents These notes summarize and extend two lectures from Bob Harper s Homotopy Type Theory course. The cumulative hierarchy

More information

0.6 Factoring 73. As always, the reader is encouraged to multiply out (3

0.6 Factoring 73. As always, the reader is encouraged to multiply out (3 0.6 Factoring 7 5. The G.C.F. of the terms in 81 16t is just 1 so there is nothing of substance to factor out from both terms. With just a difference of two terms, we are limited to fitting this olynomial

More information

Commutators on l. D. Dosev and W. B. Johnson

Commutators on l. D. Dosev and W. B. Johnson Submitted exclusively to the London Mathematical Society doi:10.1112/0000/000000 Commutators on l D. Dosev and W. B. Johnson Abstract The oerators on l which are commutators are those not of the form λi

More information

ANALYTIC NUMBER THEORY AND DIRICHLET S THEOREM

ANALYTIC NUMBER THEORY AND DIRICHLET S THEOREM ANALYTIC NUMBER THEORY AND DIRICHLET S THEOREM JOHN BINDER Abstract. In this aer, we rove Dirichlet s theorem that, given any air h, k with h, k) =, there are infinitely many rime numbers congruent to

More information

[Ch 3, 4] Logic and Proofs (2) 1. Valid and Invalid Arguments ( 2.3, 3.4) 400 lecture note #2. 1) Basics

[Ch 3, 4] Logic and Proofs (2) 1. Valid and Invalid Arguments ( 2.3, 3.4) 400 lecture note #2. 1) Basics 400 lecture note #2 [Ch 3, 4] Logic and Proofs (2) 1. Valid and Invalid Arguments ( 2.3, 3.4) 1) Basics An argument is a sequence of statements ( s1, s2,, sn). All statements in an argument, excet for

More information

ON FREIMAN S 2.4-THEOREM

ON FREIMAN S 2.4-THEOREM ON FREIMAN S 2.4-THEOREM ØYSTEIN J. RØDSETH Abstract. Gregory Freiman s celebrated 2.4-Theorem says that if A is a set of residue classes modulo a rime satisfying 2A 2.4 A 3 and A < /35, then A is contained

More information

Outline. CS21 Decidability and Tractability. Regular expressions and FA. Regular expressions and FA. Regular expressions and FA

Outline. CS21 Decidability and Tractability. Regular expressions and FA. Regular expressions and FA. Regular expressions and FA Outline CS21 Decidability and Tractability Lecture 4 January 14, 2019 FA and Regular Exressions Non-regular languages: Puming Lemma Pushdown Automata Context-Free Grammars and Languages January 14, 2019

More information

A construction of bent functions from plateaued functions

A construction of bent functions from plateaued functions A construction of bent functions from lateaued functions Ayça Çeşmelioğlu, Wilfried Meidl Sabancı University, MDBF, Orhanlı, 34956 Tuzla, İstanbul, Turkey. Abstract In this resentation, a technique for

More information

Topic 30 Notes Jeremy Orloff

Topic 30 Notes Jeremy Orloff Toic 30 Notes Jeremy Orloff 30 Alications to oulation biology 30.1 Modeling examles 30.1.1 Volterra redator-rey model The Volterra redator-rey system models the oulations of two secies with a redatorrey

More information

ON THE NORM OF AN IDEMPOTENT SCHUR MULTIPLIER ON THE SCHATTEN CLASS

ON THE NORM OF AN IDEMPOTENT SCHUR MULTIPLIER ON THE SCHATTEN CLASS PROCEEDINGS OF THE AMERICAN MATHEMATICAL SOCIETY Volume 00, Number 0, Pages 000 000 S 000-9939XX)0000-0 ON THE NORM OF AN IDEMPOTENT SCHUR MULTIPLIER ON THE SCHATTEN CLASS WILLIAM D. BANKS AND ASMA HARCHARRAS

More information

A Note on Guaranteed Sparse Recovery via l 1 -Minimization

A Note on Guaranteed Sparse Recovery via l 1 -Minimization A Note on Guaranteed Sarse Recovery via l -Minimization Simon Foucart, Université Pierre et Marie Curie Abstract It is roved that every s-sarse vector x C N can be recovered from the measurement vector

More information

arxiv: v1 [physics.data-an] 26 Oct 2012

arxiv: v1 [physics.data-an] 26 Oct 2012 Constraints on Yield Parameters in Extended Maximum Likelihood Fits Till Moritz Karbach a, Maximilian Schlu b a TU Dortmund, Germany, moritz.karbach@cern.ch b TU Dortmund, Germany, maximilian.schlu@cern.ch

More information

7.2 Inference for comparing means of two populations where the samples are independent

7.2 Inference for comparing means of two populations where the samples are independent Objectives 7.2 Inference for comaring means of two oulations where the samles are indeendent Two-samle t significance test (we give three examles) Two-samle t confidence interval htt://onlinestatbook.com/2/tests_of_means/difference_means.ht

More information

Network Configuration Control Via Connectivity Graph Processes

Network Configuration Control Via Connectivity Graph Processes Network Configuration Control Via Connectivity Grah Processes Abubakr Muhammad Deartment of Electrical and Systems Engineering University of Pennsylvania Philadelhia, PA 90 abubakr@seas.uenn.edu Magnus

More information

18.312: Algebraic Combinatorics Lionel Levine. Lecture 12

18.312: Algebraic Combinatorics Lionel Levine. Lecture 12 8.3: Algebraic Combinatorics Lionel Levine Lecture date: March 7, Lecture Notes by: Lou Odette This lecture: A continuation of the last lecture: comutation of µ Πn, the Möbius function over the incidence

More information

Advanced Calculus I. Part A, for both Section 200 and Section 501

Advanced Calculus I. Part A, for both Section 200 and Section 501 Sring 2 Instructions Please write your solutions on your own aer. These roblems should be treated as essay questions. A roblem that says give an examle requires a suorting exlanation. In all roblems, you

More information

Lilian Markenzon 1, Nair Maria Maia de Abreu 2* and Luciana Lee 3

Lilian Markenzon 1, Nair Maria Maia de Abreu 2* and Luciana Lee 3 Pesquisa Oeracional (2013) 33(1): 123-132 2013 Brazilian Oerations Research Society Printed version ISSN 0101-7438 / Online version ISSN 1678-5142 www.scielo.br/oe SOME RESULTS ABOUT THE CONNECTIVITY OF

More information

Cryptanalysis of Pseudorandom Generators

Cryptanalysis of Pseudorandom Generators CSE 206A: Lattice Algorithms and Alications Fall 2017 Crytanalysis of Pseudorandom Generators Instructor: Daniele Micciancio UCSD CSE As a motivating alication for the study of lattice in crytograhy we

More information

9 The Theory of Special Relativity

9 The Theory of Special Relativity 9 The Theory of Secial Relativity Assign: Read Chater 4 of Carrol and Ostlie (2006) Newtonian hysics is a quantitative descrition of Nature excet under three circumstances: 1. In the realm of the very

More information

Topic: Lower Bounds on Randomized Algorithms Date: September 22, 2004 Scribe: Srinath Sridhar

Topic: Lower Bounds on Randomized Algorithms Date: September 22, 2004 Scribe: Srinath Sridhar 15-859(M): Randomized Algorithms Lecturer: Anuam Guta Toic: Lower Bounds on Randomized Algorithms Date: Setember 22, 2004 Scribe: Srinath Sridhar 4.1 Introduction In this lecture, we will first consider

More information

ε i (E j )=δj i = 0, if i j, form a basis for V, called the dual basis to (E i ). Therefore, dim V =dim V.

ε i (E j )=δj i = 0, if i j, form a basis for V, called the dual basis to (E i ). Therefore, dim V =dim V. Covectors Definition. Let V be a finite-dimensional vector sace. A covector on V is real-valued linear functional on V, that is, a linear ma ω : V R. The sace of all covectors on V is itself a real vector

More information

MATH 361: NUMBER THEORY EIGHTH LECTURE

MATH 361: NUMBER THEORY EIGHTH LECTURE MATH 361: NUMBER THEORY EIGHTH LECTURE 1. Quadratic Recirocity: Introduction Quadratic recirocity is the first result of modern number theory. Lagrange conjectured it in the late 1700 s, but it was first

More information

MAS 4203 Number Theory. M. Yotov

MAS 4203 Number Theory. M. Yotov MAS 4203 Number Theory M. Yotov June 15, 2017 These Notes were comiled by the author with the intent to be used by his students as a main text for the course MAS 4203 Number Theory taught at the Deartment

More information

Math 751 Lecture Notes Week 3

Math 751 Lecture Notes Week 3 Math 751 Lecture Notes Week 3 Setember 25, 2014 1 Fundamental grou of a circle Theorem 1. Let φ : Z π 1 (S 1 ) be given by n [ω n ], where ω n : I S 1 R 2 is the loo ω n (s) = (cos(2πns), sin(2πns)). Then

More information

Lecture 10: Hypercontractivity

Lecture 10: Hypercontractivity CS 880: Advanced Comlexity Theory /15/008 Lecture 10: Hyercontractivity Instructor: Dieter van Melkebeek Scribe: Baris Aydinlioglu This is a technical lecture throughout which we rove the hyercontractivity

More information

Lecture 6 : Dimensionality Reduction

Lecture 6 : Dimensionality Reduction CPS290: Algorithmic Founations of Data Science February 3, 207 Lecture 6 : Dimensionality Reuction Lecturer: Kamesh Munagala Scribe: Kamesh Munagala In this lecture, we will consier the roblem of maing

More information

HASSE INVARIANTS FOR THE CLAUSEN ELLIPTIC CURVES

HASSE INVARIANTS FOR THE CLAUSEN ELLIPTIC CURVES HASSE INVARIANTS FOR THE CLAUSEN ELLIPTIC CURVES AHMAD EL-GUINDY AND KEN ONO Astract. Gauss s F x hyergeometric function gives eriods of ellitic curves in Legendre normal form. Certain truncations of this

More information

IMPROVED BOUNDS IN THE SCALED ENFLO TYPE INEQUALITY FOR BANACH SPACES

IMPROVED BOUNDS IN THE SCALED ENFLO TYPE INEQUALITY FOR BANACH SPACES IMPROVED BOUNDS IN THE SCALED ENFLO TYPE INEQUALITY FOR BANACH SPACES OHAD GILADI AND ASSAF NAOR Abstract. It is shown that if (, ) is a Banach sace with Rademacher tye 1 then for every n N there exists

More information

Stochastic integration II: the Itô integral

Stochastic integration II: the Itô integral 13 Stochastic integration II: the Itô integral We have seen in Lecture 6 how to integrate functions Φ : (, ) L (H, E) with resect to an H-cylindrical Brownian motion W H. In this lecture we address the

More information

DIRICHLET S THEOREM ON PRIMES IN ARITHMETIC PROGRESSIONS. 1. Introduction

DIRICHLET S THEOREM ON PRIMES IN ARITHMETIC PROGRESSIONS. 1. Introduction DIRICHLET S THEOREM ON PRIMES IN ARITHMETIC PROGRESSIONS INNA ZAKHAREVICH. Introduction It is a well-known fact that there are infinitely many rimes. However, it is less clear how the rimes are distributed

More information

MATH 371 Class notes/outline October 15, 2013

MATH 371 Class notes/outline October 15, 2013 MATH 371 Class notes/outline October 15, 2013 More on olynomials We now consider olynomials with coefficients in rings (not just fields) other than R and C. (Our rings continue to be commutative and have

More information

8 STOCHASTIC PROCESSES

8 STOCHASTIC PROCESSES 8 STOCHASTIC PROCESSES The word stochastic is derived from the Greek στoχαστικoς, meaning to aim at a target. Stochastic rocesses involve state which changes in a random way. A Markov rocess is a articular

More information

UNIVALENT UNIVERSES FOR ELEGANT MODELS OF HOMOTOPY TYPES. Denis-Charles Cisinski

UNIVALENT UNIVERSES FOR ELEGANT MODELS OF HOMOTOPY TYPES. Denis-Charles Cisinski UNIVALENT UNIVERSES FOR ELEGANT MODELS OF HOMOTOP TPES by Denis-Charles Cisinski Abstract. We construct a univalent universe in the sense of Voevodsky in some suitable model categories for homotoy tyes

More information

On Wald-Type Optimal Stopping for Brownian Motion

On Wald-Type Optimal Stopping for Brownian Motion J Al Probab Vol 34, No 1, 1997, (66-73) Prerint Ser No 1, 1994, Math Inst Aarhus On Wald-Tye Otimal Stoing for Brownian Motion S RAVRSN and PSKIR The solution is resented to all otimal stoing roblems of

More information

STA 250: Statistics. Notes 7. Bayesian Approach to Statistics. Book chapters: 7.2

STA 250: Statistics. Notes 7. Bayesian Approach to Statistics. Book chapters: 7.2 STA 25: Statistics Notes 7. Bayesian Aroach to Statistics Book chaters: 7.2 1 From calibrating a rocedure to quantifying uncertainty We saw that the central idea of classical testing is to rovide a rigorous

More information

MATHEMATICAL MODELLING OF THE WIRELESS COMMUNICATION NETWORK

MATHEMATICAL MODELLING OF THE WIRELESS COMMUNICATION NETWORK Comuter Modelling and ew Technologies, 5, Vol.9, o., 3-39 Transort and Telecommunication Institute, Lomonosov, LV-9, Riga, Latvia MATHEMATICAL MODELLIG OF THE WIRELESS COMMUICATIO ETWORK M. KOPEETSK Deartment

More information

dn i where we have used the Gibbs equation for the Gibbs energy and the definition of chemical potential

dn i where we have used the Gibbs equation for the Gibbs energy and the definition of chemical potential Chem 467 Sulement to Lectures 33 Phase Equilibrium Chemical Potential Revisited We introduced the chemical otential as the conjugate variable to amount. Briefly reviewing, the total Gibbs energy of a system

More information

c Copyright by Helen J. Elwood December, 2011

c Copyright by Helen J. Elwood December, 2011 c Coyright by Helen J. Elwood December, 2011 CONSTRUCTING COMPLEX EQUIANGULAR PARSEVAL FRAMES A Dissertation Presented to the Faculty of the Deartment of Mathematics University of Houston In Partial Fulfillment

More information

Frobenius Elements, the Chebotarev Density Theorem, and Reciprocity

Frobenius Elements, the Chebotarev Density Theorem, and Reciprocity Frobenius Elements, the Chebotarev Density Theorem, and Recirocity Dylan Yott July 30, 204 Motivation Recall Dirichlet s theorem from elementary number theory. Theorem.. For a, m) =, there are infinitely

More information

arxiv:cond-mat/ v2 25 Sep 2002

arxiv:cond-mat/ v2 25 Sep 2002 Energy fluctuations at the multicritical oint in two-dimensional sin glasses arxiv:cond-mat/0207694 v2 25 Se 2002 1. Introduction Hidetoshi Nishimori, Cyril Falvo and Yukiyasu Ozeki Deartment of Physics,

More information

On a Markov Game with Incomplete Information

On a Markov Game with Incomplete Information On a Markov Game with Incomlete Information Johannes Hörner, Dinah Rosenberg y, Eilon Solan z and Nicolas Vieille x{ January 24, 26 Abstract We consider an examle of a Markov game with lack of information

More information

Radial Basis Function Networks: Algorithms

Radial Basis Function Networks: Algorithms Radial Basis Function Networks: Algorithms Introduction to Neural Networks : Lecture 13 John A. Bullinaria, 2004 1. The RBF Maing 2. The RBF Network Architecture 3. Comutational Power of RBF Networks 4.

More information