Topology I - Exercises and Solutions

Size: px
Start display at page:

Download "Topology I - Exercises and Solutions"

Transcription

1 Topology I - Exercises and Solutions July 25, Metric spaces 1. Let p be a prime number, and d: Z Z [0, + ) be a function defined by d p (x, y) = p max{m N : pm x y}. Prove that d p is a metric on Z and that d p (x, y) max{d p (x, z), d p (z, y)} for every x, y, z Z. Proof. The symmetry condition is trivial. By p > 0 and m N, we have p m > 0 for every m N with 0 as the limit. Indeed, d(x, y) can only be zero, if p m x y for all natural numbers m. This can only happen if x y = 0, thus d(x, y) = 0 x = y. For the triangle inequality condition, assume wlog that m x,z := log p (d(x, z)) is not larger than m y,z (i.e. d(x, z) d(y, z)). Then p mx,z divides both x z and z y and therefore also x z + z y = x y, which means that m x,y m x,z or equivalently d(x, y) d(x, z) = max{d(x, z), d(y, z)}, so in particular d(x, y) d(x, z) + d(y, z) holds. 2. Let X be a set and F the family of all finite subsets of X. Prove that the function d: F F [0, + ) defined by d(a, B) = #((A\B) (B\A)) is a metric on X. Proof. d(a, B) = 0 implies that both A\B and B\A must be empty, thus the sets A and B must coincide. Conversely d(a, A) = 0. Looking at the Venn diagram for sets A, B, C, it can be seen that A C B C contains A B (where denotes the symmetric difference). 3. Let (X, d) be a metric space and F X be a finite subset. Prove that F is closed in X. Proof. Let x X \ F and define r := min{d(x, y) : y F }. As F is finite the minimum exists. The open ball B(x, r) around x does not contain any point of F, thus X \ F is open and F closed. 4. Let (X, d) be a metric space and = Y X be a subset. The distance of a point x X from the subset Y is a function X [0, + ) defined by: d(x, Y ) = inf{d(x, y) : y Y }. Verify that the distance function is well defined. Prove that Y = {x X : d(x, Y ) = 0}. Proof. The fact that d is bounded from below ensures that for each x X the infimum exists. If the infimum exists, it is unique, so the function is well-defined. The claim directly follows from Lemma 1.5 in the lecture: Take an x / Y and r > 0 such that B r (x) Y =. Then all points outside the ball, in particular the points of Y, must have distance at least r, so x / {x X : d(x, Y ) = 0}. Now let x / {x X : d(x, Y ) = 0}. Then by the triangle inequality any ball B(x, r) with 0 < r < d(x, Y ) will be an open neighbourhood of x that doesn t intersect {x X : d(x, Y ) = 0}. Hence it is closed and because it contains Y, it is a superset of Y. 1

2 5. Let X be the set of all sequences x: N R converging to zero. Prove that the function d: X X [0, + ) defined by d(x n, y n ) = sup x n y n n N is a metric on X. Show that the metric space (X, d) is separable. Proof. Symmetry and coincidence with zero are obvious. For the triangle inequality in this metric, use the triangle inequality for the Euclidean metric. For each n N, we have x n y n = x n z n + z n y n x n z n + z n y n d(x, z) + d(y, z). Then by the definition of the supremum, this also holds for d(x, y). To prove that X is separable we need to find a countable set Q such that Q = X. Let Q be the set of sequences r : N Q converging to zero. Cantors diagonal argument shows that Q is countable and for every x X, x(i) can be approximated by a sequence of rationals r n (i), so r n x. 6. Let (X, d) be a metric space and Y X be a subspace. Then U Y is open (closed) in Y if and only if there exist V X open (closed) in X such that U = V Y. Proof. By definition a set U Y is open in Y if for all points x U there exists an r x > 0 such that B d (x, r x ) lies in U, where d := d Y Y. Thus U can be expressed as x U B d (x, r x). One direction of the claim can be shown by setting V := x U B d(x, r x ). Intersecting each ball B d (x, r x ) with Y, we obtain the corresponding ball with respect to the induced metric d and deduce Y V = U. The converse direction is straight forward. If there is an open V with the above mentioned properties, it must contain an open ball B d (z, r z ) for every point z V which gives us balls which are open in Y and which all lie in U. 7. Let (X, d) be a metric space, and Y X. Prove that the function X R defined by x d(x, Y ) is a continuous function. Proof. It suffices to show that the preimage of any open set U R is open in X. Take an arbitrary x f 1 (U). U is open, so there exists an ε > 0 with the property that (z ε, z + ε) U where z := d(x, Y ). Every point x B(x, ε) satisfies d(x, Y ) d(x, x) + d(x, Y ) < ε + z by the triangle inequality. Conversely, we also have z = d(x, Y ) d(x, x )+d(x, Y ) < ε+d(x, Y )which rearranges to z ε < d(x, Y ). We deduce that x f 1 (U) which yields the claim. 8. Let (X, d) be a metric space and U X be an open subset in X. Consider a function d U : U U [0, + ) defined by d U (x, y) = d(x, y) + 1 d(x,x\u) 1 d(y,x\u). Prove that d U is a metric on U and that it is equivalent to the induced metric d U U. Proof. Again, symmetry and coincidence with zero are obvious. Using the triangle inequality first for the metric d and then for the absolute value function, we obtain d U (x, y) = d(x, y) + 1 d(x,x\u) 1 d(y,x\u) d(x, z) + d(y, z) + 1 d(x,x\u) 1 d(z,x\u) + 1 d(z,x\u) 1 d(y,x\u) d(x, z) + d(y, z) + 1 d(x,x\u) 1 d(z,x\u) + 1 d(z,x\u) 1 d(y,x\u) = d U (x, z) + d U (y, z). To show the equivalence of the metrics, take a set V U that is open with respect to d. This set contains an open r x -ball contained in V for every element x V. The open ball with radius r x with respect to d U is a subset of B d (x, r x ) and therefore lies in V. Conversely, take a set W that is open with respect to metric d U and a point x W. There exists a radius R x such that B du (x, R x ) W. For every point y in B d (x, r x ) for some r x that is yet to 2

3 determine, the distance d(y, X \ U) differs from D x := d(x, X \ U) by at most r x. Without loss of generality, assume that D x > r x, otherwise scale r x accordingly. Now 1 d(x,x\u) 1 d(y,x\u) = d(y,x\u) d(x,x\u) d(x,x\u) d(y,x\u) r x D =: N x (D x r x) x Thus d U (x, y) d(x, y) + N x < r x + N x. Setting r x such that r x + N x < R x, ensures that B d (x, r x ) B du (x, R x ) and therefore lies in W. 9. Let S be a set and (X, d) a complete metric space. Prove that the metric space of all bounded functions B(S, X) equipped with the metric D(f, g) = sup s S d(f(s), g(s)) is also complete. Proof. Take a Cauchy sequence (f n ) B(S, X) in the sup-metric. For every ε > 0 there exists an n ε N so that d(f n (s), f m (s)) D(f n, f m ) < ε 3 for all n, m n ε. From the definition of D we know that (f n (s)) is a Cauchy sequence in X for every s S. Since X is complete, for every s S there exists a f(s) X so that f n (s) f(s). Define the function f : S X so that s f(s) (well defined due to the uniqueness of the limit). To check that (f n ) converges to f, fix s S. Now there exists n s N so that d(f n (s), f(s)) < ε 3 for all n n s. Define N := max{n ε, n s }. Then for every n n ε we have d(f n (s), f(s)) d(f n (s), f N (s)) + d(f N (s), f(s)) < ε 3 + ε 3 = 2ε 3. In other words, for every s S the difference d(f n (s), f(s)) is bounded by 2ε 3. Hence by taking supremum over all s S, we have D(f n, f) 2ε 3 < ε for all n n ε. To show that f is bounded, i.e. sup r,s S d(f(s), f(r)) <, use the triangle inequality twice and the fact that f N is bounded. d(f(s), f(r)) d(f(s), f N (s)) + d(f N (s), f N (r)) + d(f N (r), f(r)) 2ε 3 + d(f N (s), f N (r)) < 10. Prove that a discrete metric space is compact if and only if its underlying set is finite. Proof. One direction is obvious, as each subset of a finite set is finite. For the other direction, take a compact space (X, d) with the discrete metric, suppose the underlying set X were infinite and look at the open cover C = {{x} : x X}. As C is infinite, any finite subcover C would yield an element y X that is not covered by C which contradicts the compactness of (X, d). 11. Let (X, d) be a metric space and lim x n = x 0 in X. Show that the set K = {x 0, x 1,... } is compact. Proof. As x 0 lies in K, there must be one open set U 0 in any open covering C that contains it. This U 0 must contain an open ball B(x 0, ε). As the sequence (x n ) converges to x 0, there is a n 0 such that for all n n 0, we have d(x n, x 0 ) < ε which leaves only finitely many points outside the ball. The (finite) subset of those, that aren t contained in U 0 can be covered by finitely many open sets from C. 12. Let (X, d) be a metric space, and let F X be a closed subset and K X a compact subset of X. Prove that F K inf{d(x, y) : x F, y K} = 0. Proof. The one direction is straight forward. A point x F K satisfies d(x, x) = 0. For the other direction, take sequences (x n ) F, (y n ) K that satisfy inf n N d(x n, y n ) = 0. For all ε > 0 we have an n 1 N s.t. for all n n 1, d(x n, y n ) < ε 2. K is compact, so (y n) has a converging subsequence (y ni ) with limit y K. In particular, we find an n 2 N such that for all n n 2, d(y ni, y) < ε 2. With the triangle inequality, we get d(y, x ni ) d(y, y ni ) + d(y ni, x ni ) < ε. Thus y is a limit point of F and since F is closed, ist must be contained in F. 13. Let (X 1, d 1 ),..., (X n, d n ) be compact metric spaces, and let X := X 1 X n be equipped with either the D 1 or D metric. Prove that X is also compact. 3

4 Proof. Take a sequence (x k ) in X and look at the sequences (x k 1),..., (x k n) in X 1,..., X n. Since (X 1, d 1 ) is compact, it has a convergent subsequence (x k l 1 ) with index set I 1. The induced sequence (x k l 2 ) in X 2 has a converging subsequence (x k lm 2 ) for an index set I 2 I 1. Iterating gives us an index set I n such that the sequences x K j for K I n converge for all j = 1,..., n. Thus, with both metrics, the corresponding subsequence of (x k ) converges. From the lecture we know that this implies compactness (Chapter 1.9, Lemma). 14. Let E be a normed space and A and B two compact subspaces. Then the Minkowski sum is also compact. A + B := {a + b : a A, b B} Proof. This can again be shown using sequential compactness. Another approach is the following. Let C be an open cover of A+B. Then the families C A := {U B : U C} and C B := {U A : U C} are covers of A and B respectively. Those sets are compact, so there exist finite subcovers. Both families (translated by A or B) together yield a finite subcover of A + B. 15. Let (X, d) be a metric space. Define a function d : X X [0, + ) by d (x, y) := min{d(x, y), 1} for every (x, y) X X. Show that d is a metric on X, and moreover is equivalent to d, i.e., induces the same topology as d. Proof. Checking the metric properties is straight forward. To see that the topologies coincide, use that for ε < 1, B d (x, ε) = B d (x, ε). 2 Topological spaces and Continuous Functions 1. Let X be a set and T = {U X : U = or X\U is countable}. Prove that T is a topology on X. Proof. Obviously and X are contained in T. For the second criterion, look at a subfamily {U α : α A} of T. Without loss of generality, assume that all U α have a countable complement. Then X \ α A U α = α A X \ U α is the intersection of countable sets and therefore countable. Also, the finite union of countable sets is countable which yields the third criterion. 2. Let X be a set and B be a basis for a topology on X. Prove that the topology generated by B is indeed a topology. Proof. Denote the topology generated by B with T. The empty set is trivially contained in it. For the whole space X, the first property of a basis ensures that C T. The second criterion is obvious, as any point x in the union of open sets must lie in one of them. Thus we find a basis set B containing x and also contained in that set and therefore also in the union. If we take a finite subfamily {U 1,..., U n }, then any x i=1,...,n U i has basis sets B i such that x B i U i. The second base property reformulates as n : x i=1,...,n B i B B : x B i=1,...,n B i (by repeatedly applying the property). Thus there exists a basis set B such that x B i=1,...,n U i. 3. Let X = R and K = { 1 n : n N}. Prove that the following families are bases for a topology on X: B = {(a, b) : a, b R, a < b}, B = {[a, b) : a, b R, a < b}, B = {(a, b) : a, b R, a < b} {(a, b)\k : a, b R, a < b}. Furthermore, let T, T and T denote the topologies on X generated by B, B and B, respectively. Prove that T and T are finer than T, and that T and T are not comparable. 4

5 Proof. Remark: T is called the lower limit topology or right half-open interval topology; the topological space is called Sorgenfrey line. T is called K-topology. First, check the two basis properties for the three families. This is straightforward. The only thing one has to watch out for is the second property for B. There one needs to do a (simple) case analysis. T T : Let U T. Then x U (a x, b x ) U : x (a x, b x ). We can rewrite any interval (a, b) as a<c<b [c, b), so (a x, b x ) T, thus for all y (a x, b x ), so in particular for the previous x, there exist B y B : y B y (a x, b x ). Thus U T. T T : Obvious. T T : Use R \ K. It is open in T but has nonempty intersection with every open set in T that also contains zero. T T : Take for instance [2, ). It is open in T but any basis set in B that contains 2 will also contain numbers smaller than Let X = R and B = {(a, b) : a, b Q, a < b}. Prove that B is a basis for a topology on X, and that it generates the standard topology on X. Proof. Let x R. Let n be some integer larger than x. Then n < x < n. Now let (a, b) and (c, d) be basis sets that contain x. Then (max(a, c), min(b, d)) lies in B because max(a, c) < x and x < min(b, d). Finally we need to check that the generated topology coincides with the standard topology. The one inclusion is obvious. For the other one, take a set U that is open in the standard topology. Then there are real numbers a < b such that x (a, b) for all x U. There exists an N such that N > 1 x a M between an and xn. This again can be rearranged to a < M N. which can be rearranged to 1 < xn an, so there must be another integer < x. Doing the same thing for x and b, we get x ( M N, M N ) (a, b). Hence U is open in the topology generated by B. 5. Let A be a subspace of X and let B be a subspace of Y. We equip A and B with the subspace topologies. Prove that the product topology on A B is the same as the topology A B inherits as a subspace of X Y. Proof. Denote with T A B,prod the product topology on A B and with T A B,sub the subspace topology induced by X Y. T A B,prod T A B,sub : Let U A U B T A T B. The open sets in A and B respectively give us open sets V A and V B in the spaces X and Y by the definition of the subspace topology and if we intersect V A V B with A B, we obtain U A U B. Thus the basis of T A B,prod is contained in T A B,sub, and the same holds for the topology generated by it. T A B,sub T A B,prod : Let U T A B,sub. Then there exists a set V T X Y such that V A B = U. By the construction of the product topology, for all v V we have a basis set V X V Y T X T Y with v V X V Y V. In particular this holds for all v U with v U A U B := V X V Y A B U, so U T A B,prod. 6. Let Y be a subspace of X. Prove that if A is closed in Y, and Y is closed in X, then A is closed in X. Proof. Denote by U Z (x) the family of sets which contain x and are open in Z and by A Z Z the closure of A in Z. Recall the following criterion from the lecture (a theorem from Chapter 2.3): x Z lies in A Z U U Z (x) : U A. Let x A X, then every element of U X (x) must have non-empty intersection with Y, because A Y. This means that x Y X which equals Y because Y is closed in X. Also, all sets in U Y (x) originate from a set in U X (x), so they all have non-empty intersection with A. Thus x A Y which coincides with A because A is closed in Y. A A X is trivial, so we deduce A = A X. 7. Let X be a Hausdorff space. Prove that a sequence in X converges to at most one point in X. Proof. Denote by U(x) the family of open sets which contain x. Assume we have a converging sequence (x n ) with distinct limit points x and y. Then by definition for all U U(x), V U(y) there exist n U, n V N such that for all n n U, n V, we have x n U and x n V respectively. 5

6 X is Hausdorff, so there exist disjoint neighbourhoods U U(x) and V U(y) and for n max{n U, n V } we have x n U V =. Contradiction. 8. Show that if A is closed in X, and B is closed in Y, then A B is closed in X Y. Proof. X \ A and Y \ B are open and so is (X \ A) Y and X (Y \ B). Thus (X Y ) \ (A B) = ((X \ A) Y ) (X (Y \ B)) is also open. Alternatively, use A B = A B from exercise Show that if U is open in X and A is closed in X, then U\A is open in X, and A\U is closed in X. Proof. U \ A = U (X \ U) and X \ (A \ U) = (X \ A) U are the finite intersection resp. union of open sets and therefore open. 10. Let A X and B Y. Show that A B = A B in X Y. Proof. Wlog only look at the limit points (for isolated points there is no problem). Let (a n, b n ) be a convergent sequence in A B with limit point (a, b). Let V T X and W T Y with a V and b W, then V W T X Y and (a, b) V W. Thus there exists an n V,W N such that all subsequent elements (a n, b n ) lie in V W. In particular a n V, b n W for all n n V,W which makes a and b limit points. A and B are closed, therefore a A and b B. Let a n a in A and b n b in B. Take an arbitrary U T X Y with (a, b) U. Then for all u U there is a basis set V W T X Y such that u V W U. The open sets V and W give us numbers n V, n W N such that a n V, b n W for all subsequent n. Define n U := max(n v, n W ), then n n U : (a n.b n ) U. We deduce that (a, b) is a limit point. 11. Show that the product of two Hausdorff spaces is Hausdorff. Proof. Let (a, b) (c, d) be points in X Y, where X, Y are Hausdorff spaces. Then a c or b d. Wlog assume a c. Then there exist disjoint open neighbourhoods A and C for a and c in X. This gives us disjoint open neighbourhoods A Y and C Y of (a, b) and (c, d). 12. Show that X is Hausdorff if and only if the diagonal := {(x, x) : x X} is closed in X X. Proof. X is Hausdorff. For every pair a, b X with a b there there exist disjoint open neighbourhoods A a and B b. Every element (a, b) of X \ has a basis set A B with (a, b) A B X \. X \ is open. is closed. 13. If A X, let us define the boundary of A by the equation: A := A X\A. Show that: (a) A A = and A = A A; (b) A = if and only if A is both open and closed; (c) A is open if and only if A = A\A. Proof. (a) x A. There is an open neighbourhood U A of x. There is an open neighbourhood U of x with U X \ A =. x / X \ A. This means A = X \ X \ A. From this we deduce two things: Firstly, A X \ A = and therefore A A = and secondly A = A (X \ A) and therefore A A = A (X \ A) A = A. (b) A is open and closed if and only if A = A = A and using (a), this corresponds to A =. (c) A is open if and only if A = A. Subtracting A from the second equation (and using the first statement) of (a), we get that A = A \ A. Inserting A = A yields the claim. A = A (A \ A) = A \ (A \ A), so A \ A =. 6

7 14. Let f : X Y be a continuous map, A X and A denotes the set of all limit points of A. If x A is it true that f(x) f(a), i.e., is f(x) a limit point of f(a)? Proof. No, in general this is not true. Isolated points can cause a problem. Consider for instance the constant map f : R [0, 1] {2} given by f(x) = 2. It is obviously continuous but 2 is no limit point. 15. Let f : A B and g : C D be continuous functions. Consider the map f g : A C B D defined by (f g)(a, c) := (f(a), g(c)) for every (a, c) A C. Prove that f g is also continuous. Proof. Let U T B D. Then for all u U there is a set B u D u T B T D with u B u D u U. Define A u := f 1 (B u ) and C u := g 1 (D u ). A u C u is an open neighbourhood for any v (f g) 1 (u) due to the fact that f and g are continuous. Thus for every v (f g) 1 (U) there is a set A (f g)(v) A (f g)(v) T A T C with v A (f g)(v) C (f g)(v) (f g) 1 (U) which proves our claim. 16. Let X and Y be topological spaces with Y being Hausdorff. Let A X and f : A Y be a continuous map. Prove that if f can be extended to a continuous function g : A Y, then g is uniquely determined by f. Proof. From exercise 2.14 we know that a convergent sequence a n in A with limit point a yields a convergent sequence g(a n ) with limit point g(a). In exercise 2.7 we learned that the limit of a convergent sequence is unique in Hausdorff spaces, so g(a) = lim n f(a n ) is uniquely defined. 17. Let {X α } α J be an indexed family of topological spaces. Assume that the topology on each X α is given by a basis B α. Prove that the family { } B α : B α B α α J is a basis for the box topology on α J X α, while { B α : B α B α and B α = X α for all but finitely many α J } α J is a basis for the product topology on α J X α. Proof. Let U T box, then for all u U there exists a set α J U α with the property that u α J U α U. For all α, we have u α U α and a basis set B α such that u α B α U α, so u α J B α α J U α U. The same line of reasoning works for the product topology. 18. Let {X α } α J be an indexed family of Hausdorff spaces. Prove that α J X α is a Hausdorff space in both the box and product topology. Proof. If two points (x α ) and (y α ) are different, then there must be an index α J such that x α y α. Use the same argument as in 11. to prove that the claim (for both topologies). 19. Let p: X Y be a continuous map. Show that if there is a continuous map f : Y X such that p f = id Y, then p is a quotient map. Proof. For every y Y the element x := f(y) is in p 1 (y), so p is surjective. Now let p 1 (U) T X. Then U = (p f) 1 (U) = f 1 p 1 (U) is open because f is continuous. Together with the fact that p is continuous, this yields the claim. 20. Let X be a topological space and A X a subspace. A continuous map r : X A is a retraction if r A = id A, i.e., r(a) = a for every a A. Show that a retraction is a quotient map. Proof. Use the previous exercise with p := r and f : A X, the embedding of A into X. 7

8 3 Connectedness and Compactness 1. Let {C n } be a sequence of connected subspaces of X with the property that C n C n+1 for every n N. Show that n N C n is connected. Proof. Assume there exist non-empty open sets U, V such that n N C n is the disjoint union of the two. For every n N we know that either U C n or V C n must be empty because C n is connected. So we have that C n U or C n V (This is also a lemma in Chapter 3). Using induction and the fact that for all n N the subspaces C n and C n+1 have non-empty intersection, we deduce that all C n must lie in the same set U or V which contradicts our assumption. 2. Let {C α } be a sequence of connected subspaces of X. Let moreover C be a connected subspace of X with the property that C C α for every α. Show that C ( α C α) is connected. Proof. Assume U and V form a separation of C ( α N C n). Very much like in the previous exercise, we deduce that C α and C lie either in U or in V. Wlog say C U, then U C α U and therefore C α U for all α. Contradiction. 3. Let X be an infinite set. Show that if X is equipped with the finite complement topology then X is connected. Proof. For every pair of sets U, V with the property that X = U V, i.e. U = X \ V, we have the following. If one of them, say U, is open, then its complement V must be finite by the definition of the topology. But this means that U itself must be infinite (as X is infinite) and therefore V cannot be open. 4. Let A X. Show that if C is a connected subspace of X that intersects both A and X\A, then C intersects A. Proof. We can write X as the disjoint union of A, A and (X \ A). If C A is empty, then C = C ( A A (X \ A)) = (C A) (C (X \ A)). These two sets are open in the subspace topology which contradicts the connectedness assumption. 5. Let A X and B Y. If X and Y are connected, show that (X Y )\(A B) is also connected. Proof. A and B don t coincide with X and Y, so we find points x X \ A and y Y \ B and can construct sets {x} Y and X {y} that are disjoint from A B. The union ({x} Y ) (X {y}) is connected as it is the union of connected sets with a point (x, y) in common (see Exercise 3.1). 6. Let p: X Y be a quotient map, p 1 ({y}) be connected for every y Y, and Y be connected. Show that X is connected. Proof. Assume U and V form a separation of X. We know that p(u) p(u) = Y because p is surjective. Assume there exists a y p(u) p(v ). Denote the fibre p 1 ({y}) with C. C is connected and the sets C U and C V are open in C and C = (C U) (C V ) which gives us a contradiction. This means that p(u) and p(v ) are disjoint but also that p 1 (p(u)) = U. p is a quotient map, so if p 1 (p(u)) is open, then so is p(u). The same holds for p(v ). Thus p(u) and p(v ) form a separation of Y, which cannot be true. 7. Let Y be a subspace of X, and both connected. Show that if A and B form a separation of X\Y, then Y A and Y B are connected Proof. Let us work with the definition of connectedness using limit points, which was introduced in Lemma 1 of the third chapter. Assume that Y A is not connected. Then we find non-empty U, V with the property that U V =, U V = and Y A = U V. Y is connected, so by the second lemma of Chapter 3 either Y U or Y V. Say Y U. Then V A A, hence V B = and V B =. If we now look at the union U B, we see that V (U B) = V (U B ) = and V (U B) =. So V and U B form a separation of X = Y A B = V U B. Contradiction. The same line of reasoning proves that Y B must be connected. 8. Show that R d and R are not homeomorphic if d > 1. 8

9 Proof. Assume there is a homeomorphism f : R n R. Define f : R n \ {f 1 (0)} R \ {0} to be the restriction of f. It is easy to see that this is again a homeomorphism. But R n \ {h 1 (0)} is connected (consider 0 as {0} {0} and see Exercise 3.5) and R \ {0} is not. The theorem which states that the image of a connected space under a continuous map is connected gives us the desired contradiction. 9. Let f : S 1 R be a continuous map. Show that there exists a point x S 1 such that f(x) = f( x). Proof. Assume there is no such point. Then we can construct the (well-defined) map g : S 1 S 0 given by g(x) := f(x) f( x) f(x) f( x). It is continuous and therefore its image should be connected, because S 1 is connected. g(x) and g( x) differ in sign for any x S 1, so { 1, 1} is the image of g and disconnected which gives us a contradiction. Remark: This statement generalizes to the Borsuk-Ulam theorem. 10. Let f : [0, 1] [0, 1] be a continuous map. Show that there exists a point x [0, 1] such that f(x) = x. Proof. Analogously to the previous exercise, assume there is no such point and define g : [0, 1] { 1, 1} given by g(x) := f(x) x f(x) x. This map is well-defined and continuous. It is also surjective because f(1) < 1 and f(0) > 0 and hence g(1) = 1 and g(0) = 1, which as before gives us a contradiction. Remark: This is a special case of the Brouwer fixed-point theorem. 11. Show that the finite union of compact subspaces of X is compact. Proof. Let U be an open covering of X = n i=1 X i. It is also an open covering of the X i. Compactness gives us a finite subcollection Ũ for every i. Then the union of these families is a finite subcover of X. 12. Show that every compact subspace Y of a metric space X is bounded with respect to the metric and is closed. Proof. Fix an y Y. Then {B(y, ε) X : ε > 0} is an open cover of Y. From the compactness property we know that there exists a finite subcover with say N sets and ε max the radius of the largest ball. Then the diameter of Y is at most 2ε max. The fact that Y is also closed was proved in Chapter Let A and B be disjoint compact subspaces of the Hausdorff space X. Show that there exist disjoint open sets U and V in X such that A U and B V. Proof. Recall that in the lecture we extracted the following property from the proof of the claim that every compact subspace of a Hausdorff space is closed: If Y is a compact subspace of a Hausdorff space X and x 0 Y, then there exist disjoint open sets U and V of X containing Y and x 0, respectively. Apply this to the compact set A and all points b in B. Then {V b } is an open cover of B with finite subcover {V b1,..., V bn }. The sets n i=1 U b i and n i=1 V b i are disjoint and open with A n i=1 U b i and b n i=1 V b i 14. Let X be compact and Y be a Hausdorff space. If f : X Y is a continuous map then f is a closed map. Proof. Let Z be a closed subset of X. From the lecture we know that it must be compact too. Images of compact spaces under continuous maps are again compact, so f(z) is compact. But that means it is also closed, because Y is Hausdorff. 15. Show that if Y is compact, then the projection π 1 : X Y X is a closed map. Proof. Let Z X Y be closed and x X \ π(z). For every y Y, we have that (x, y) / Z. The set X \ Z is open, so we find basis sets U y V y X Y \ Z that contain (x, y). The sets V y cover the compact space Y, so there is a finite subfamily, say V y1,..., V yn such that Y = n i=1 V y i. Every set U yi V yi lies in X Y \ Z, thus U yi π(z) =. Hence the intersection n i=1 U y i is an open neighbourhood of x that does not intersect π(z), so π(z) is closed. 9

10 16. Let f : X Y be a continuous map with Y compact Hausdorff. Show that f is continuous if and only if the graph of f G f := {(x, f(x)) : x X} is a closed subset of X Y. Proof. Let (x, y) (X Y ) \ G f. Then y f(x) and therefore we can find disjoint open neighbourhoods U y, V f(x). Define W := f 1 (V ). Then f(w ) V Y \ U and thus W U G f =. W U is open, so we found an open neighbourhood of (x, y) in (X Y )\G f. Now let G f be closed and let V be an open set in Y. Then the intersection G f X (Y \ V ) is also closed. If we apply Exercise 3.15, we can deduce that π 1 (G f X (Y \ V )) = {x X : f(x) / V } = X \ f 1 (V ) is closed and equivalently, that f 1 (V ) is open. 10

Introduction to Topology

Introduction to Topology Introduction to Topology Tomoo Matsumura November 30, 2010 Contents 1 Topological spaces 3 1.1 Basis of a Topology......................................... 3 1.2 Comparing Topologies.......................................

More information

Metric Spaces. Chapter 7. 7.1. Metrics

Metric Spaces. Chapter 7. 7.1. Metrics Chapter 7 Metric Spaces A metric space is a set X that has a notion of the distance d(x, y) between every pair of points x, y X. The purpose of this chapter is to introduce metric spaces and give some

More information

Metric Spaces Joseph Muscat 2003 (Last revised May 2009)

Metric Spaces Joseph Muscat 2003 (Last revised May 2009) 1 Distance J Muscat 1 Metric Spaces Joseph Muscat 2003 (Last revised May 2009) (A revised and expanded version of these notes are now published by Springer.) 1 Distance A metric space can be thought of

More information

1. Prove that the empty set is a subset of every set.

1. Prove that the empty set is a subset of every set. 1. Prove that the empty set is a subset of every set. Basic Topology Written by Men-Gen Tsai email: b89902089@ntu.edu.tw Proof: For any element x of the empty set, x is also an element of every set since

More information

Basic Concepts of Point Set Topology Notes for OU course Math 4853 Spring 2011

Basic Concepts of Point Set Topology Notes for OU course Math 4853 Spring 2011 Basic Concepts of Point Set Topology Notes for OU course Math 4853 Spring 2011 A. Miller 1. Introduction. The definitions of metric space and topological space were developed in the early 1900 s, largely

More information

Notes on metric spaces

Notes on metric spaces Notes on metric spaces 1 Introduction The purpose of these notes is to quickly review some of the basic concepts from Real Analysis, Metric Spaces and some related results that will be used in this course.

More information

Metric Spaces. Chapter 1

Metric Spaces. Chapter 1 Chapter 1 Metric Spaces Many of the arguments you have seen in several variable calculus are almost identical to the corresponding arguments in one variable calculus, especially arguments concerning convergence

More information

SOLUTIONS TO EXERCISES FOR. MATHEMATICS 205A Part 3. Spaces with special properties

SOLUTIONS TO EXERCISES FOR. MATHEMATICS 205A Part 3. Spaces with special properties SOLUTIONS TO EXERCISES FOR MATHEMATICS 205A Part 3 Fall 2008 III. Spaces with special properties III.1 : Compact spaces I Problems from Munkres, 26, pp. 170 172 3. Show that a finite union of compact subspaces

More information

THE BANACH CONTRACTION PRINCIPLE. Contents

THE BANACH CONTRACTION PRINCIPLE. Contents THE BANACH CONTRACTION PRINCIPLE ALEX PONIECKI Abstract. This paper will study contractions of metric spaces. To do this, we will mainly use tools from topology. We will give some examples of contractions,

More information

Mathematical Methods of Engineering Analysis

Mathematical Methods of Engineering Analysis Mathematical Methods of Engineering Analysis Erhan Çinlar Robert J. Vanderbei February 2, 2000 Contents Sets and Functions 1 1 Sets................................... 1 Subsets.............................

More information

SOLUTIONS TO ASSIGNMENT 1 MATH 576

SOLUTIONS TO ASSIGNMENT 1 MATH 576 SOLUTIONS TO ASSIGNMENT 1 MATH 576 SOLUTIONS BY OLIVIER MARTIN 13 #5. Let T be the topology generated by A on X. We want to show T = J B J where B is the set of all topologies J on X with A J. This amounts

More information

MA651 Topology. Lecture 6. Separation Axioms.

MA651 Topology. Lecture 6. Separation Axioms. MA651 Topology. Lecture 6. Separation Axioms. This text is based on the following books: Fundamental concepts of topology by Peter O Neil Elements of Mathematics: General Topology by Nicolas Bourbaki Counterexamples

More information

Point Set Topology. A. Topological Spaces and Continuous Maps

Point Set Topology. A. Topological Spaces and Continuous Maps Point Set Topology A. Topological Spaces and Continuous Maps Definition 1.1 A topology on a set X is a collection T of subsets of X satisfying the following axioms: T 1.,X T. T2. {O α α I} T = α IO α T.

More information

INTRODUCTION TO TOPOLOGY

INTRODUCTION TO TOPOLOGY INTRODUCTION TO TOPOLOGY ALEX KÜRONYA In preparation January 24, 2010 Contents 1. Basic concepts 1 2. Constructing topologies 13 2.1. Subspace topology 13 2.2. Local properties 18 2.3. Product topology

More information

FUNCTIONAL ANALYSIS LECTURE NOTES: QUOTIENT SPACES

FUNCTIONAL ANALYSIS LECTURE NOTES: QUOTIENT SPACES FUNCTIONAL ANALYSIS LECTURE NOTES: QUOTIENT SPACES CHRISTOPHER HEIL 1. Cosets and the Quotient Space Any vector space is an abelian group under the operation of vector addition. So, if you are have studied

More information

CHAPTER 1 BASIC TOPOLOGY

CHAPTER 1 BASIC TOPOLOGY CHAPTER 1 BASIC TOPOLOGY Topology, sometimes referred to as the mathematics of continuity, or rubber sheet geometry, or the theory of abstract topological spaces, is all of these, but, above all, it is

More information

Undergraduate Notes in Mathematics. Arkansas Tech University Department of Mathematics

Undergraduate Notes in Mathematics. Arkansas Tech University Department of Mathematics Undergraduate Notes in Mathematics Arkansas Tech University Department of Mathematics An Introductory Single Variable Real Analysis: A Learning Approach through Problem Solving Marcel B. Finan c All Rights

More information

1 if 1 x 0 1 if 0 x 1

1 if 1 x 0 1 if 0 x 1 Chapter 3 Continuity In this chapter we begin by defining the fundamental notion of continuity for real valued functions of a single real variable. When trying to decide whether a given function is or

More information

Math 104: Introduction to Analysis

Math 104: Introduction to Analysis Math 104: Introduction to Analysis Evan Chen UC Berkeley Notes for the course MATH 104, instructed by Charles Pugh. 1 1 August 29, 2013 Hard: #22 in Chapter 1. Consider a pile of sand principle. You wish

More information

Follow links for Class Use and other Permissions. For more information send email to: permissions@pupress.princeton.edu

Follow links for Class Use and other Permissions. For more information send email to: permissions@pupress.princeton.edu COPYRIGHT NOTICE: Ariel Rubinstein: Lecture Notes in Microeconomic Theory is published by Princeton University Press and copyrighted, c 2006, by Princeton University Press. All rights reserved. No part

More information

No: 10 04. Bilkent University. Monotonic Extension. Farhad Husseinov. Discussion Papers. Department of Economics

No: 10 04. Bilkent University. Monotonic Extension. Farhad Husseinov. Discussion Papers. Department of Economics No: 10 04 Bilkent University Monotonic Extension Farhad Husseinov Discussion Papers Department of Economics The Discussion Papers of the Department of Economics are intended to make the initial results

More information

THE FUNDAMENTAL THEOREM OF ALGEBRA VIA PROPER MAPS

THE FUNDAMENTAL THEOREM OF ALGEBRA VIA PROPER MAPS THE FUNDAMENTAL THEOREM OF ALGEBRA VIA PROPER MAPS KEITH CONRAD 1. Introduction The Fundamental Theorem of Algebra says every nonconstant polynomial with complex coefficients can be factored into linear

More information

CHAPTER II THE LIMIT OF A SEQUENCE OF NUMBERS DEFINITION OF THE NUMBER e.

CHAPTER II THE LIMIT OF A SEQUENCE OF NUMBERS DEFINITION OF THE NUMBER e. CHAPTER II THE LIMIT OF A SEQUENCE OF NUMBERS DEFINITION OF THE NUMBER e. This chapter contains the beginnings of the most important, and probably the most subtle, notion in mathematical analysis, i.e.,

More information

MEASURE AND INTEGRATION. Dietmar A. Salamon ETH Zürich

MEASURE AND INTEGRATION. Dietmar A. Salamon ETH Zürich MEASURE AND INTEGRATION Dietmar A. Salamon ETH Zürich 12 May 2016 ii Preface This book is based on notes for the lecture course Measure and Integration held at ETH Zürich in the spring semester 2014. Prerequisites

More information

4. Expanding dynamical systems

4. Expanding dynamical systems 4.1. Metric definition. 4. Expanding dynamical systems Definition 4.1. Let X be a compact metric space. A map f : X X is said to be expanding if there exist ɛ > 0 and L > 1 such that d(f(x), f(y)) Ld(x,

More information

0 <β 1 let u(x) u(y) kuk u := sup u(x) and [u] β := sup

0 <β 1 let u(x) u(y) kuk u := sup u(x) and [u] β := sup 456 BRUCE K. DRIVER 24. Hölder Spaces Notation 24.1. Let Ω be an open subset of R d,bc(ω) and BC( Ω) be the bounded continuous functions on Ω and Ω respectively. By identifying f BC( Ω) with f Ω BC(Ω),

More information

Lecture Notes on Topology for MAT3500/4500 following J. R. Munkres textbook. John Rognes

Lecture Notes on Topology for MAT3500/4500 following J. R. Munkres textbook. John Rognes Lecture Notes on Topology for MAT3500/4500 following J. R. Munkres textbook John Rognes November 29th 2010 Contents Introduction v 1 Set Theory and Logic 1 1.1 ( 1) Fundamental Concepts..............................

More information

BANACH AND HILBERT SPACE REVIEW

BANACH AND HILBERT SPACE REVIEW BANACH AND HILBET SPACE EVIEW CHISTOPHE HEIL These notes will briefly review some basic concepts related to the theory of Banach and Hilbert spaces. We are not trying to give a complete development, but

More information

x a x 2 (1 + x 2 ) n.

x a x 2 (1 + x 2 ) n. Limits and continuity Suppose that we have a function f : R R. Let a R. We say that f(x) tends to the limit l as x tends to a; lim f(x) = l ; x a if, given any real number ɛ > 0, there exists a real number

More information

ON SEQUENTIAL CONTINUITY OF COMPOSITION MAPPING. 0. Introduction

ON SEQUENTIAL CONTINUITY OF COMPOSITION MAPPING. 0. Introduction ON SEQUENTIAL CONTINUITY OF COMPOSITION MAPPING Abstract. In [1] there was proved a theorem concerning the continuity of the composition mapping, and there was announced a theorem on sequential continuity

More information

INTRODUCTORY SET THEORY

INTRODUCTORY SET THEORY M.Sc. program in mathematics INTRODUCTORY SET THEORY Katalin Károlyi Department of Applied Analysis, Eötvös Loránd University H-1088 Budapest, Múzeum krt. 6-8. CONTENTS 1. SETS Set, equal sets, subset,

More information

Finite dimensional topological vector spaces

Finite dimensional topological vector spaces Chapter 3 Finite dimensional topological vector spaces 3.1 Finite dimensional Hausdorff t.v.s. Let X be a vector space over the field K of real or complex numbers. We know from linear algebra that the

More information

Chapter 4, Arithmetic in F [x] Polynomial arithmetic and the division algorithm.

Chapter 4, Arithmetic in F [x] Polynomial arithmetic and the division algorithm. Chapter 4, Arithmetic in F [x] Polynomial arithmetic and the division algorithm. We begin by defining the ring of polynomials with coefficients in a ring R. After some preliminary results, we specialize

More information

1. Let X and Y be normed spaces and let T B(X, Y ).

1. Let X and Y be normed spaces and let T B(X, Y ). Uppsala Universitet Matematiska Institutionen Andreas Strömbergsson Prov i matematik Funktionalanalys Kurs: NVP, Frist. 2005-03-14 Skrivtid: 9 11.30 Tillåtna hjälpmedel: Manuella skrivdon, Kreyszigs bok

More information

Metric Spaces. Lecture Notes and Exercises, Fall 2015. M.van den Berg

Metric Spaces. Lecture Notes and Exercises, Fall 2015. M.van den Berg Metric Spaces Lecture Notes and Exercises, Fall 2015 M.van den Berg School of Mathematics University of Bristol BS8 1TW Bristol, UK mamvdb@bristol.ac.uk 1 Definition of a metric space. Let X be a set,

More information

PUTNAM TRAINING POLYNOMIALS. Exercises 1. Find a polynomial with integral coefficients whose zeros include 2 + 5.

PUTNAM TRAINING POLYNOMIALS. Exercises 1. Find a polynomial with integral coefficients whose zeros include 2 + 5. PUTNAM TRAINING POLYNOMIALS (Last updated: November 17, 2015) Remark. This is a list of exercises on polynomials. Miguel A. Lerma Exercises 1. Find a polynomial with integral coefficients whose zeros include

More information

I. GROUPS: BASIC DEFINITIONS AND EXAMPLES

I. GROUPS: BASIC DEFINITIONS AND EXAMPLES I GROUPS: BASIC DEFINITIONS AND EXAMPLES Definition 1: An operation on a set G is a function : G G G Definition 2: A group is a set G which is equipped with an operation and a special element e G, called

More information

Quotient Rings and Field Extensions

Quotient Rings and Field Extensions Chapter 5 Quotient Rings and Field Extensions In this chapter we describe a method for producing field extension of a given field. If F is a field, then a field extension is a field K that contains F.

More information

How To Prove The Dirichlet Unit Theorem

How To Prove The Dirichlet Unit Theorem Chapter 6 The Dirichlet Unit Theorem As usual, we will be working in the ring B of algebraic integers of a number field L. Two factorizations of an element of B are regarded as essentially the same if

More information

Practice with Proofs

Practice with Proofs Practice with Proofs October 6, 2014 Recall the following Definition 0.1. A function f is increasing if for every x, y in the domain of f, x < y = f(x) < f(y) 1. Prove that h(x) = x 3 is increasing, using

More information

ON FIBER DIAMETERS OF CONTINUOUS MAPS

ON FIBER DIAMETERS OF CONTINUOUS MAPS ON FIBER DIAMETERS OF CONTINUOUS MAPS PETER S. LANDWEBER, EMANUEL A. LAZAR, AND NEEL PATEL Abstract. We present a surprisingly short proof that for any continuous map f : R n R m, if n > m, then there

More information

Mathematics Review for MS Finance Students

Mathematics Review for MS Finance Students Mathematics Review for MS Finance Students Anthony M. Marino Department of Finance and Business Economics Marshall School of Business Lecture 1: Introductory Material Sets The Real Number System Functions,

More information

Fixed Point Theorems

Fixed Point Theorems Fixed Point Theorems Definition: Let X be a set and let T : X X be a function that maps X into itself. (Such a function is often called an operator, a transformation, or a transform on X, and the notation

More information

1 Norms and Vector Spaces

1 Norms and Vector Spaces 008.10.07.01 1 Norms and Vector Spaces Suppose we have a complex vector space V. A norm is a function f : V R which satisfies (i) f(x) 0 for all x V (ii) f(x + y) f(x) + f(y) for all x,y V (iii) f(λx)

More information

PSEUDOARCS, PSEUDOCIRCLES, LAKES OF WADA AND GENERIC MAPS ON S 2

PSEUDOARCS, PSEUDOCIRCLES, LAKES OF WADA AND GENERIC MAPS ON S 2 PSEUDOARCS, PSEUDOCIRCLES, LAKES OF WADA AND GENERIC MAPS ON S 2 Abstract. We prove a Bruckner-Garg type theorem for the fiber structure of a generic map from a continuum X into the unit interval I. We

More information

Solutions to Homework 10

Solutions to Homework 10 Solutions to Homework 1 Section 7., exercise # 1 (b,d): (b) Compute the value of R f dv, where f(x, y) = y/x and R = [1, 3] [, 4]. Solution: Since f is continuous over R, f is integrable over R. Let x

More information

9 More on differentiation

9 More on differentiation Tel Aviv University, 2013 Measure and category 75 9 More on differentiation 9a Finite Taylor expansion............... 75 9b Continuous and nowhere differentiable..... 78 9c Differentiable and nowhere monotone......

More information

INTRODUCTION TO DESCRIPTIVE SET THEORY

INTRODUCTION TO DESCRIPTIVE SET THEORY INTRODUCTION TO DESCRIPTIVE SET THEORY ANUSH TSERUNYAN Mathematicians in the early 20 th century discovered that the Axiom of Choice implied the existence of pathological subsets of the real line lacking

More information

3. INNER PRODUCT SPACES

3. INNER PRODUCT SPACES . INNER PRODUCT SPACES.. Definition So far we have studied abstract vector spaces. These are a generalisation of the geometric spaces R and R. But these have more structure than just that of a vector space.

More information

HOMEWORK 5 SOLUTIONS. n!f n (1) lim. ln x n! + xn x. 1 = G n 1 (x). (2) k + 1 n. (n 1)!

HOMEWORK 5 SOLUTIONS. n!f n (1) lim. ln x n! + xn x. 1 = G n 1 (x). (2) k + 1 n. (n 1)! Math 7 Fall 205 HOMEWORK 5 SOLUTIONS Problem. 2008 B2 Let F 0 x = ln x. For n 0 and x > 0, let F n+ x = 0 F ntdt. Evaluate n!f n lim n ln n. By directly computing F n x for small n s, we obtain the following

More information

3. Prime and maximal ideals. 3.1. Definitions and Examples.

3. Prime and maximal ideals. 3.1. Definitions and Examples. COMMUTATIVE ALGEBRA 5 3.1. Definitions and Examples. 3. Prime and maximal ideals Definition. An ideal P in a ring A is called prime if P A and if for every pair x, y of elements in A\P we have xy P. Equivalently,

More information

Numerical Analysis Lecture Notes

Numerical Analysis Lecture Notes Numerical Analysis Lecture Notes Peter J. Olver 5. Inner Products and Norms The norm of a vector is a measure of its size. Besides the familiar Euclidean norm based on the dot product, there are a number

More information

Separation Properties for Locally Convex Cones

Separation Properties for Locally Convex Cones Journal of Convex Analysis Volume 9 (2002), No. 1, 301 307 Separation Properties for Locally Convex Cones Walter Roth Department of Mathematics, Universiti Brunei Darussalam, Gadong BE1410, Brunei Darussalam

More information

Fixed Point Theorems in Topology and Geometry

Fixed Point Theorems in Topology and Geometry Fixed Point Theorems in Topology and Geometry A Senior Thesis Submitted to the Department of Mathematics In Partial Fulfillment of the Requirements for the Departmental Honors Baccalaureate By Morgan Schreffler

More information

DEGREES OF ORDERS ON TORSION-FREE ABELIAN GROUPS

DEGREES OF ORDERS ON TORSION-FREE ABELIAN GROUPS DEGREES OF ORDERS ON TORSION-FREE ABELIAN GROUPS ASHER M. KACH, KAREN LANGE, AND REED SOLOMON Abstract. We construct two computable presentations of computable torsion-free abelian groups, one of isomorphism

More information

Large induced subgraphs with all degrees odd

Large induced subgraphs with all degrees odd Large induced subgraphs with all degrees odd A.D. Scott Department of Pure Mathematics and Mathematical Statistics, University of Cambridge, England Abstract: We prove that every connected graph of order

More information

TOPOLOGY: THE JOURNEY INTO SEPARATION AXIOMS

TOPOLOGY: THE JOURNEY INTO SEPARATION AXIOMS TOPOLOGY: THE JOURNEY INTO SEPARATION AXIOMS VIPUL NAIK Abstract. In this journey, we are going to explore the so called separation axioms in greater detail. We shall try to understand how these axioms

More information

1 Local Brouwer degree

1 Local Brouwer degree 1 Local Brouwer degree Let D R n be an open set and f : S R n be continuous, D S and c R n. Suppose that the set f 1 (c) D is compact. (1) Then the local Brouwer degree of f at c in the set D is defined.

More information

MATHEMATICAL INDUCTION. Mathematical Induction. This is a powerful method to prove properties of positive integers.

MATHEMATICAL INDUCTION. Mathematical Induction. This is a powerful method to prove properties of positive integers. MATHEMATICAL INDUCTION MIGUEL A LERMA (Last updated: February 8, 003) Mathematical Induction This is a powerful method to prove properties of positive integers Principle of Mathematical Induction Let P

More information

CS 103X: Discrete Structures Homework Assignment 3 Solutions

CS 103X: Discrete Structures Homework Assignment 3 Solutions CS 103X: Discrete Structures Homework Assignment 3 s Exercise 1 (20 points). On well-ordering and induction: (a) Prove the induction principle from the well-ordering principle. (b) Prove the well-ordering

More information

3. Mathematical Induction

3. Mathematical Induction 3. MATHEMATICAL INDUCTION 83 3. Mathematical Induction 3.1. First Principle of Mathematical Induction. Let P (n) be a predicate with domain of discourse (over) the natural numbers N = {0, 1,,...}. If (1)

More information

How To Find Out How To Calculate A Premeasure On A Set Of Two-Dimensional Algebra

How To Find Out How To Calculate A Premeasure On A Set Of Two-Dimensional Algebra 54 CHAPTER 5 Product Measures Given two measure spaces, we may construct a natural measure on their Cartesian product; the prototype is the construction of Lebesgue measure on R 2 as the product of Lebesgue

More information

God created the integers and the rest is the work of man. (Leopold Kronecker, in an after-dinner speech at a conference, Berlin, 1886)

God created the integers and the rest is the work of man. (Leopold Kronecker, in an after-dinner speech at a conference, Berlin, 1886) Chapter 2 Numbers God created the integers and the rest is the work of man. (Leopold Kronecker, in an after-dinner speech at a conference, Berlin, 1886) God created the integers and the rest is the work

More information

n k=1 k=0 1/k! = e. Example 6.4. The series 1/k 2 converges in R. Indeed, if s n = n then k=1 1/k, then s 2n s n = 1 n + 1 +...

n k=1 k=0 1/k! = e. Example 6.4. The series 1/k 2 converges in R. Indeed, if s n = n then k=1 1/k, then s 2n s n = 1 n + 1 +... 6 Series We call a normed space (X, ) a Banach space provided that every Cauchy sequence (x n ) in X converges. For example, R with the norm = is an example of Banach space. Now let (x n ) be a sequence

More information

Ideal Class Group and Units

Ideal Class Group and Units Chapter 4 Ideal Class Group and Units We are now interested in understanding two aspects of ring of integers of number fields: how principal they are (that is, what is the proportion of principal ideals

More information

MASSACHUSETTS INSTITUTE OF TECHNOLOGY 6.436J/15.085J Fall 2008 Lecture 5 9/17/2008 RANDOM VARIABLES

MASSACHUSETTS INSTITUTE OF TECHNOLOGY 6.436J/15.085J Fall 2008 Lecture 5 9/17/2008 RANDOM VARIABLES MASSACHUSETTS INSTITUTE OF TECHNOLOGY 6.436J/15.085J Fall 2008 Lecture 5 9/17/2008 RANDOM VARIABLES Contents 1. Random variables and measurable functions 2. Cumulative distribution functions 3. Discrete

More information

TOPIC 4: DERIVATIVES

TOPIC 4: DERIVATIVES TOPIC 4: DERIVATIVES 1. The derivative of a function. Differentiation rules 1.1. The slope of a curve. The slope of a curve at a point P is a measure of the steepness of the curve. If Q is a point on the

More information

INDISTINGUISHABILITY OF ABSOLUTELY CONTINUOUS AND SINGULAR DISTRIBUTIONS

INDISTINGUISHABILITY OF ABSOLUTELY CONTINUOUS AND SINGULAR DISTRIBUTIONS INDISTINGUISHABILITY OF ABSOLUTELY CONTINUOUS AND SINGULAR DISTRIBUTIONS STEVEN P. LALLEY AND ANDREW NOBEL Abstract. It is shown that there are no consistent decision rules for the hypothesis testing problem

More information

The Henstock-Kurzweil-Stieltjes type integral for real functions on a fractal subset of the real line

The Henstock-Kurzweil-Stieltjes type integral for real functions on a fractal subset of the real line The Henstock-Kurzweil-Stieltjes type integral for real functions on a fractal subset of the real line D. Bongiorno, G. Corrao Dipartimento di Ingegneria lettrica, lettronica e delle Telecomunicazioni,

More information

LEARNING OBJECTIVES FOR THIS CHAPTER

LEARNING OBJECTIVES FOR THIS CHAPTER CHAPTER 2 American mathematician Paul Halmos (1916 2006), who in 1942 published the first modern linear algebra book. The title of Halmos s book was the same as the title of this chapter. Finite-Dimensional

More information

A Topology Primer. Preface. Lecture Notes 2001/2002. Klaus Wirthmüller. http://www.mathematik.uni-kl.de/ wirthm/de/top.html

A Topology Primer. Preface. Lecture Notes 2001/2002. Klaus Wirthmüller. http://www.mathematik.uni-kl.de/ wirthm/de/top.html A Topology Primer Lecture Notes 2001/2002 Klaus Wirthmüller http://www.mathematik.uni-kl.de/ wirthm/de/top.html Preface These lecture notes were written to accompany my introductory courses of topology

More information

The sample space for a pair of die rolls is the set. The sample space for a random number between 0 and 1 is the interval [0, 1].

The sample space for a pair of die rolls is the set. The sample space for a random number between 0 and 1 is the interval [0, 1]. Probability Theory Probability Spaces and Events Consider a random experiment with several possible outcomes. For example, we might roll a pair of dice, flip a coin three times, or choose a random real

More information

MATH PROBLEMS, WITH SOLUTIONS

MATH PROBLEMS, WITH SOLUTIONS MATH PROBLEMS, WITH SOLUTIONS OVIDIU MUNTEANU These are free online notes that I wrote to assist students that wish to test their math skills with some problems that go beyond the usual curriculum. These

More information

Math 312 Homework 1 Solutions

Math 312 Homework 1 Solutions Math 31 Homework 1 Solutions Last modified: July 15, 01 This homework is due on Thursday, July 1th, 01 at 1:10pm Please turn it in during class, or in my mailbox in the main math office (next to 4W1) Please

More information

Mathematics for Computer Science/Software Engineering. Notes for the course MSM1F3 Dr. R. A. Wilson

Mathematics for Computer Science/Software Engineering. Notes for the course MSM1F3 Dr. R. A. Wilson Mathematics for Computer Science/Software Engineering Notes for the course MSM1F3 Dr. R. A. Wilson October 1996 Chapter 1 Logic Lecture no. 1. We introduce the concept of a proposition, which is a statement

More information

MATH 304 Linear Algebra Lecture 20: Inner product spaces. Orthogonal sets.

MATH 304 Linear Algebra Lecture 20: Inner product spaces. Orthogonal sets. MATH 304 Linear Algebra Lecture 20: Inner product spaces. Orthogonal sets. Norm The notion of norm generalizes the notion of length of a vector in R n. Definition. Let V be a vector space. A function α

More information

MATH 425, PRACTICE FINAL EXAM SOLUTIONS.

MATH 425, PRACTICE FINAL EXAM SOLUTIONS. MATH 45, PRACTICE FINAL EXAM SOLUTIONS. Exercise. a Is the operator L defined on smooth functions of x, y by L u := u xx + cosu linear? b Does the answer change if we replace the operator L by the operator

More information

Chapter 7. Continuity

Chapter 7. Continuity Chapter 7 Continuity There are many processes and eects that depends on certain set of variables in such a way that a small change in these variables acts as small change in the process. Changes of this

More information

Mathematics for Econometrics, Fourth Edition

Mathematics for Econometrics, Fourth Edition Mathematics for Econometrics, Fourth Edition Phoebus J. Dhrymes 1 July 2012 1 c Phoebus J. Dhrymes, 2012. Preliminary material; not to be cited or disseminated without the author s permission. 2 Contents

More information

ALMOST COMMON PRIORS 1. INTRODUCTION

ALMOST COMMON PRIORS 1. INTRODUCTION ALMOST COMMON PRIORS ZIV HELLMAN ABSTRACT. What happens when priors are not common? We introduce a measure for how far a type space is from having a common prior, which we term prior distance. If a type

More information

THIN GROUPS OF FRACTIONS

THIN GROUPS OF FRACTIONS Contemporary Mathematics THIN GROUPS OF FRACTIONS Patrick DEHORNOY Abstract. A number of properties of spherical Artin Tits groups extend to Garside groups, defined as the groups of fractions of monoids

More information

(Basic definitions and properties; Separation theorems; Characterizations) 1.1 Definition, examples, inner description, algebraic properties

(Basic definitions and properties; Separation theorems; Characterizations) 1.1 Definition, examples, inner description, algebraic properties Lecture 1 Convex Sets (Basic definitions and properties; Separation theorems; Characterizations) 1.1 Definition, examples, inner description, algebraic properties 1.1.1 A convex set In the school geometry

More information

An example of a computable

An example of a computable An example of a computable absolutely normal number Verónica Becher Santiago Figueira Abstract The first example of an absolutely normal number was given by Sierpinski in 96, twenty years before the concept

More information

WHAT ARE MATHEMATICAL PROOFS AND WHY THEY ARE IMPORTANT?

WHAT ARE MATHEMATICAL PROOFS AND WHY THEY ARE IMPORTANT? WHAT ARE MATHEMATICAL PROOFS AND WHY THEY ARE IMPORTANT? introduction Many students seem to have trouble with the notion of a mathematical proof. People that come to a course like Math 216, who certainly

More information

FIRST YEAR CALCULUS. Chapter 7 CONTINUITY. It is a parabola, and we can draw this parabola without lifting our pencil from the paper.

FIRST YEAR CALCULUS. Chapter 7 CONTINUITY. It is a parabola, and we can draw this parabola without lifting our pencil from the paper. FIRST YEAR CALCULUS WWLCHENW L c WWWL W L Chen, 1982, 2008. 2006. This chapter originates from material used by the author at Imperial College, University of London, between 1981 and 1990. It It is is

More information

RANDOM INTERVAL HOMEOMORPHISMS. MICHA L MISIUREWICZ Indiana University Purdue University Indianapolis

RANDOM INTERVAL HOMEOMORPHISMS. MICHA L MISIUREWICZ Indiana University Purdue University Indianapolis RANDOM INTERVAL HOMEOMORPHISMS MICHA L MISIUREWICZ Indiana University Purdue University Indianapolis This is a joint work with Lluís Alsedà Motivation: A talk by Yulij Ilyashenko. Two interval maps, applied

More information

Cartesian Products and Relations

Cartesian Products and Relations Cartesian Products and Relations Definition (Cartesian product) If A and B are sets, the Cartesian product of A and B is the set A B = {(a, b) :(a A) and (b B)}. The following points are worth special

More information

Mathematics Course 111: Algebra I Part IV: Vector Spaces

Mathematics Course 111: Algebra I Part IV: Vector Spaces Mathematics Course 111: Algebra I Part IV: Vector Spaces D. R. Wilkins Academic Year 1996-7 9 Vector Spaces A vector space over some field K is an algebraic structure consisting of a set V on which are

More information

Math 4310 Handout - Quotient Vector Spaces

Math 4310 Handout - Quotient Vector Spaces Math 4310 Handout - Quotient Vector Spaces Dan Collins The textbook defines a subspace of a vector space in Chapter 4, but it avoids ever discussing the notion of a quotient space. This is understandable

More information

A domain of spacetime intervals in general relativity

A domain of spacetime intervals in general relativity A domain of spacetime intervals in general relativity Keye Martin Department of Mathematics Tulane University New Orleans, LA 70118 United States of America martin@math.tulane.edu Prakash Panangaden School

More information

8 Divisibility and prime numbers

8 Divisibility and prime numbers 8 Divisibility and prime numbers 8.1 Divisibility In this short section we extend the concept of a multiple from the natural numbers to the integers. We also summarize several other terms that express

More information

Duality of linear conic problems

Duality of linear conic problems Duality of linear conic problems Alexander Shapiro and Arkadi Nemirovski Abstract It is well known that the optimal values of a linear programming problem and its dual are equal to each other if at least

More information

On Integer Additive Set-Indexers of Graphs

On Integer Additive Set-Indexers of Graphs On Integer Additive Set-Indexers of Graphs arxiv:1312.7672v4 [math.co] 2 Mar 2014 N K Sudev and K A Germina Abstract A set-indexer of a graph G is an injective set-valued function f : V (G) 2 X such that

More information

POLYNOMIAL RINGS AND UNIQUE FACTORIZATION DOMAINS

POLYNOMIAL RINGS AND UNIQUE FACTORIZATION DOMAINS POLYNOMIAL RINGS AND UNIQUE FACTORIZATION DOMAINS RUSS WOODROOFE 1. Unique Factorization Domains Throughout the following, we think of R as sitting inside R[x] as the constant polynomials (of degree 0).

More information

Fixed Point Theorems For Set-Valued Maps

Fixed Point Theorems For Set-Valued Maps Fixed Point Theorems For Set-Valued Maps Bachelor s thesis in functional analysis Institute for Analysis and Scientific Computing Vienna University of Technology Andreas Widder, July 2009. Preface In this

More information

So let us begin our quest to find the holy grail of real analysis.

So let us begin our quest to find the holy grail of real analysis. 1 Section 5.2 The Complete Ordered Field: Purpose of Section We present an axiomatic description of the real numbers as a complete ordered field. The axioms which describe the arithmetic of the real numbers

More information

The Banach-Tarski Paradox

The Banach-Tarski Paradox University of Oslo MAT2 Project The Banach-Tarski Paradox Author: Fredrik Meyer Supervisor: Nadia S. Larsen Abstract In its weak form, the Banach-Tarski paradox states that for any ball in R, it is possible

More information

GROUPS ACTING ON A SET

GROUPS ACTING ON A SET GROUPS ACTING ON A SET MATH 435 SPRING 2012 NOTES FROM FEBRUARY 27TH, 2012 1. Left group actions Definition 1.1. Suppose that G is a group and S is a set. A left (group) action of G on S is a rule for

More information

MATH 304 Linear Algebra Lecture 9: Subspaces of vector spaces (continued). Span. Spanning set.

MATH 304 Linear Algebra Lecture 9: Subspaces of vector spaces (continued). Span. Spanning set. MATH 304 Linear Algebra Lecture 9: Subspaces of vector spaces (continued). Span. Spanning set. Vector space A vector space is a set V equipped with two operations, addition V V (x,y) x + y V and scalar

More information

Tree-representation of set families and applications to combinatorial decompositions

Tree-representation of set families and applications to combinatorial decompositions Tree-representation of set families and applications to combinatorial decompositions Binh-Minh Bui-Xuan a, Michel Habib b Michaël Rao c a Department of Informatics, University of Bergen, Norway. buixuan@ii.uib.no

More information