6.2 Convergence of Sequences

Total Page:16

File Type:pdf, Size:1020Kb

6.2 Convergence of Sequences 124 CHAPTER 6. METRIC SPACES 6.2 Convergence of Sequences You are familiar with the notion of a convergent sequence of real numbers. It is defined as follows. The sequence x1, x2, . , xn,... of real numbers is said to converge to the real number x if given any ε > 0 there exists an integer n0 such that for all n ≥ n0, |xn − x| < ε. It is obvious how this definition can be extended from R with the euclidean metric to any metric space. 6.2.1 Definitions. Let (X, d) be a metric space and x1, . , xn,... a sequence of points in X. Then the sequence is said to converge to x ∈ X if given any ε > 0 there exists an integer n0 such that for all n ≥ n0, d(x, xn) < ε. This is denoted by xn → x. The sequence y1, y2, . , yn,... of points in (X, d) is said to be convergent if there exist a point y ∈ X such that yn → y. The next Proposition is easily proved, so its proof is left as an exercise. 6.2.2 Proposition. Let x1, x2, . , xn,... be a sequence of points in a metric space (X, d). Further, let x and y be points in (X, d) such that xn → x and xn → y. Then x = y. For convenience we say that a subset A of a metric space (X, d) is closed (respectively, open) in the metric space (X, d) if it is closed (respectively, open) in the topology τ induced on X by the metric d. 6.2. CONVERGENCE OF SEQUENCES 125 The following proposition tells us the surprising fact that the topology of a metric space can be described entirely in terms of its convergent sequences. 6.2.3 Proposition. Let (X, d) be a metric space. A subset A of X is closed in (X, d) if and only if every convergent sequence of points in A converges to a point in A. (In other words, A is closed in (X, d) if and only if an → x, where x ∈ X and an ∈ A for all n, implies x ∈ A.) Proof. Assume that A is closed in (X, d) and let an → x, where an ∈ A for all positive integers n. Suppose that x ∈ X \ A. Then, as X \ A is an open set containing x, there exists an open ball Bε(x) such that x ∈ Bε(x) ⊆ X \ A. Noting that each an ∈ A, this implies that d(x, an) > ε for each n. Hence the sequence a1, a2, . , an,... does not converge to x. This is a contradiction. So x ∈ A, as required. Conversely, assume that every convergent sequence of points in A converges to a point of A. Suppose that X \ A is not open. Then there exists a point y ∈ X \ A such that for each ε > 0, Bε(y) ∩ A =6 Ø. For each positive integer n, let xn be any point in B1/n(y) ∩ A. Then we claim that xn → y. To see this let ε be any positive real number, and n0 any integer greater than 1/ε. Then for each n ≥ n0, xn ∈ B1/n(y) ⊆ B1/n0 (y) ⊆ Bε(y). So xn → y and, by our assumption, y∈ / A. This is a contradiction and so X \ A is open and thus A is closed in (X, d). 126 CHAPTER 6. METRIC SPACES Having seen that the topology of a metric space can be described in terms of convergent sequences, we should not be surprised that continuous functions can also be so described. 6.2.4 Proposition. Let (X, d) and (Y, d1) be metric spaces and f a mapping of X into Y . Let τ and τ 1 be the topologies determined by d and d1, respectively. Then f :(X, τ ) → (Y, τ 1) is continuous if and only if xn → x ⇒ f(xn) → f(x); that is, if x1, x2, . , xn,... is a sequence of points in (X, d) converging to x, then the sequence of points f(x1), f(x2), . , f(xn),... in (Y, d1) converges to f(x). Proof. Assume that xn → x ⇒ f(xn) → f(x). To verify that f is continuous it suffices to show that the inverse image of every closed set in (Y, τ 1) is closed in (X, τ ). So let A be closed in (Y, τ 1). Let x1, x2, . , xn,... be a sequence of points in −1 f (A) convergent to a point x ∈ X. As xn → x, f(xn) → f(x). But since each f(xn) ∈ A and A is closed, Proposition 6.2.3 then implies that f(x) ∈ A. Thus x ∈ f −1(A). So we have shown that every convergent sequence of points from f −1(A) converges to a point of f −1(A). Thus f −1(A) is closed, and hence f is continuous. Conversely, let f be continuous and xn → x. Let ε be any positive real number. −1 Then the open ball Bε(f(x)) is an open set in (Y, τ 1). As f is continuous, f (Bε(f(x)) is an open set in (X, τ ) and it contains x. Therefore there exists a δ > 0 such that −1 x ∈ Bδ(x) ⊆ f (Bε(f(x))). As xn → x, there exists a positive integer n0 such that for all n ≥ n0, xn ∈ Bδ(x). Therefore f(xn) ∈ f(Bδ(x)) ⊆ Bε(f(x)), for all n ≥ n0. Thus f(xn) → f(x). The Corollary below is easily deduced from Proposition 6.2.4. 6.2. CONVERGENCE OF SEQUENCES 127 6.2.5 Corollary. Let (X, d) and (Y, d1) be metric spaces, f a mapping of X into Y , and τ and τ 1 the topologies determined by d and d1, respectively. Then f :(X, τ ) → (Y, τ 1) is continuous if and only if for each x0 ∈ X and ε > 0, there exists a δ > 0 such that x ∈ X and d(x, x0) < δ ⇒ d1(f(x), f(x0)) < ε. Exercises 6.2 1. Let C[0, 1] and d be as in Example 6.1.5. Define a sequence of functions f1, f2, . , fn,... in (C[0, 1], d) by sin(nx) f (x) = , n = 1, 2, . , x ∈ [0, 1]. n n Verify that fn → f0, where f0(x) = 0, for all x ∈ [0, 1]. 2. Let (X, d) be a metric space and x1, x2, . , xn,... a sequence such that xn → x and xn → y. Prove that x = y. 3. (i) Let (X, d) be a metric space, τ the induced topology on X, and x1, x2, . , xn,... a sequence of points in X. Prove that xn → x if and only if for every open set U ∋ x, there exists a positive integer n0 such that xn ∈ U for all n ≥ n0. (ii) Let X be a set and d and d1 equivalent metrics on X. Deduce from (i) that if xn → x in (X, d), then xn → x in (X, d1). 4. Write a proof of Corollary 6.2.5. 5. Let (X, τ ) be a topological space and let x1, x2, . , xn,... be a sequence of points in X. We say that xn → x if for each open set U ∋ x there exists a positive integer n0, such that xn ∈ U for all n ≥ n0. Find an example of a topological space and a sequence such that xn → x and xn → y but x =6 y. 6. (i) Let (X, d) be a metric space and xn → x where each xn ∈ X and x ∈ X. Let A be the subset of X which consists of x and all of the points xn. Prove that A is closed in (X, d). 1 R (ii) Deduce from (i) that the set {2} ∪ {2 − n : n = 1, 2,... } is closed in . 1 R (iii) Verify that the set {2 − n : n = 1, 2,... } is not closed in . 128 CHAPTER 6. METRIC SPACES 7. (i) Let d1, d2, . , dm be metrics on a set X and a1, a2, . am positive real numbers. Prove that d is a metric on X, where d is defined by m d(x, y) = X aidi(x, y), for all x, y ∈ X. i=1 (ii) If x ∈ X and x1, x2, . , xn,... is a sequence of points in X such that xn → x in each metric space (X, di) prove that xn → x in the metric space (X, d). 8. Let X, Y, d1, d2 and d be as in Exercises 6.1 #4. If xn → x in (X, d1) and yn → y in (Y, d2), prove that hxn, yni → hx, yi in (X × Y, d). 9. Let A and B be non-empty sets in a metric space (X, d). Define ρ(A, B) = inf{d(a, b): a ∈ A, b ∈ B}. [ρ(A, B) is referred to as the distance between the sets A and B.] (i) If S is any non-empty subset of (X, d), prove that S = {x : x ∈ X and ρ({x},S) = 0}. (ii) If S is any non-empty subset of (X, d) prove that the function f :(X, d) → R defined by f(x) = ρ({x},S), x ∈ X is continuous. 10. (i) For each positive integer n let fn be a continuous function of [0, 1] into itself and let a ∈ [0, 1] be such that fn(a) = a, for all n. Further let f be a ∗ ∗ continuous function of [0, 1] into itself. If fn → f in (C[0, 1], d ) where d is the metric of Example 6.1.6, prove that a is also a fixed point of f.
Recommended publications
  • FUNCTIONAL ANALYSIS 1. Metric and Topological Spaces A
    FUNCTIONAL ANALYSIS CHRISTIAN REMLING 1. Metric and topological spaces A metric space is a set on which we can measure distances. More precisely, we proceed as follows: let X 6= ; be a set, and let d : X×X ! [0; 1) be a map. Definition 1.1. (X; d) is called a metric space if d has the following properties, for arbitrary x; y; z 2 X: (1) d(x; y) = 0 () x = y (2) d(x; y) = d(y; x) (3) d(x; y) ≤ d(x; z) + d(z; y) Property 3 is called the triangle inequality. It says that a detour via z will not give a shortcut when going from x to y. The notion of a metric space is very flexible and general, and there are many different examples. We now compile a preliminary list of metric spaces. Example 1.1. If X 6= ; is an arbitrary set, then ( 0 x = y d(x; y) = 1 x 6= y defines a metric on X. Exercise 1.1. Check this. This example does not look particularly interesting, but it does sat- isfy the requirements from Definition 1.1. Example 1.2. X = C with the metric d(x; y) = jx−yj is a metric space. X can also be an arbitrary non-empty subset of C, for example X = R. In fact, this works in complete generality: If (X; d) is a metric space and Y ⊆ X, then Y with the same metric is a metric space also. Example 1.3. Let X = Cn or X = Rn. For each p ≥ 1, n !1=p X p dp(x; y) = jxj − yjj j=1 1 2 CHRISTIAN REMLING defines a metric on X.
    [Show full text]
  • Cantor Groups
    Integre Technical Publishing Co., Inc. College Mathematics Journal 42:1 November 11, 2010 10:58 a.m. classroom.tex page 60 Cantor Groups Ben Mathes ([email protected]), Colby College, Waterville ME 04901; Chris Dow ([email protected]), University of Chicago, Chicago IL 60637; and Leo Livshits ([email protected]), Colby College, Waterville ME 04901 The Cantor set C is simultaneously small and large. Its cardinality is the same as the cardinality of all real numbers, and every element of C is a limit of other elements of C (it is perfect), but C is nowhere dense and it is a nullset. Being nowhere dense is a kind of topological smallness, meaning that there is no interval in which the set is dense, or equivalently, that its complement is a dense open subset of [0, 1]. Being a nullset is a measure theoretic concept of smallness, meaning that, for every >0, it is possible to cover the set with a sequence of intervals In whose lengths add to a sum less than . It is possible to tweak the construction of C that results in a set H that remains per- fect (and consequently has the cardinality of the continuum), is still nowhere dense, but the measure can be made to attain any number α in the interval [0, 1). The con- struction is a special case of Hewitt and Stromberg’s Cantor-like set [1,p.70],which goes like this: let E0 denote [0, 1],letE1 denote what is left after deleting an open interval from the center of E0.IfEn−1 has been constructed, obtain En by deleting open intervals of the same length from the center of each of the disjoint closed inter- vals that comprise En−1.
    [Show full text]
  • 1. Definition. Let I Be the Unit Interval. If I, G Are Maps on I Then 1 and G Are Conjugate Iff There Is a Homeomorphism H of I Such That 1 = H -I Gh
    TRANSACTIONS OF THE AMERICAN MATHEMATICAL SOCIETY Volume 319. Number I. May 1990 A COMPLETE CLASSIFICATION OF THE PIECEWISE MONOTONE FUNCTIONS ON THE INTERVAL STEWART BALDWIN ABSTRACT. We define two functions f and g on the unit interval [0, I] to be strongly conjugate iff there is an order-preserving homeomorphism h of [0, I] such that g = h-1 fh (a minor variation of the more common term "conjugate", in which h need not be order-preserving). We provide a complete set of invariants for each continuous (strictly) piecewise monotone function such that two such functions have the same invariants if and only if they are strongly conjugate, thus providing a complete classification of all such strong conjugacy classes. In addition, we provide a criterion which decides whether or not a potential invariant is actually realized by some 'piecewise monotone continuous function. INTRODUCTION 1. Definition. Let I be the unit interval. If I, g are maps on I then 1 and g are conjugate iff there is a homeomorphism h of I such that 1 = h -I gh. A more convenient term for our purposes will be: I, g are strongly conjugate (written 1 ~ g) iff there is an order preserving homeomorphism h as above. Given a map 1 on I, define the map j by I*(x) = 1 - 1(1 - x) (essentially a 1800 rotation of the graph). The main result of this paper will be to give a complete set of invariants for the strong conjugacy classes of the piecewise monotone continuous functions on the unit interval I = [0, I].
    [Show full text]
  • Course 221: Michaelmas Term 2006 Section 3: Complete Metric Spaces, Normed Vector Spaces and Banach Spaces
    Course 221: Michaelmas Term 2006 Section 3: Complete Metric Spaces, Normed Vector Spaces and Banach Spaces David R. Wilkins Copyright c David R. Wilkins 1997–2006 Contents 3 Complete Metric Spaces, Normed Vector Spaces and Banach Spaces 2 3.1 The Least Upper Bound Principle . 2 3.2 Monotonic Sequences of Real Numbers . 2 3.3 Upper and Lower Limits of Bounded Sequences of Real Numbers 3 3.4 Convergence of Sequences in Euclidean Space . 5 3.5 Cauchy’s Criterion for Convergence . 5 3.6 The Bolzano-Weierstrass Theorem . 7 3.7 Complete Metric Spaces . 9 3.8 Normed Vector Spaces . 11 3.9 Bounded Linear Transformations . 15 3.10 Spaces of Bounded Continuous Functions on a Metric Space . 19 3.11 The Contraction Mapping Theorem and Picard’s Theorem . 20 3.12 The Completion of a Metric Space . 23 1 3 Complete Metric Spaces, Normed Vector Spaces and Banach Spaces 3.1 The Least Upper Bound Principle A set S of real numbers is said to be bounded above if there exists some real number B such x ≤ B for all x ∈ S. Similarly a set S of real numbers is said to be bounded below if there exists some real number A such that x ≥ A for all x ∈ S. A set S of real numbers is said to be bounded if it is bounded above and below. Thus a set S of real numbers is bounded if and only if there exist real numbers A and B such that A ≤ x ≤ B for all x ∈ S.
    [Show full text]
  • General Topology
    General Topology Tom Leinster 2014{15 Contents A Topological spaces2 A1 Review of metric spaces.......................2 A2 The definition of topological space.................8 A3 Metrics versus topologies....................... 13 A4 Continuous maps........................... 17 A5 When are two spaces homeomorphic?................ 22 A6 Topological properties........................ 26 A7 Bases................................. 28 A8 Closure and interior......................... 31 A9 Subspaces (new spaces from old, 1)................. 35 A10 Products (new spaces from old, 2)................. 39 A11 Quotients (new spaces from old, 3)................. 43 A12 Review of ChapterA......................... 48 B Compactness 51 B1 The definition of compactness.................... 51 B2 Closed bounded intervals are compact............... 55 B3 Compactness and subspaces..................... 56 B4 Compactness and products..................... 58 B5 The compact subsets of Rn ..................... 59 B6 Compactness and quotients (and images)............. 61 B7 Compact metric spaces........................ 64 C Connectedness 68 C1 The definition of connectedness................... 68 C2 Connected subsets of the real line.................. 72 C3 Path-connectedness.......................... 76 C4 Connected-components and path-components........... 80 1 Chapter A Topological spaces A1 Review of metric spaces For the lecture of Thursday, 18 September 2014 Almost everything in this section should have been covered in Honours Analysis, with the possible exception of some of the examples. For that reason, this lecture is longer than usual. Definition A1.1 Let X be a set. A metric on X is a function d: X × X ! [0; 1) with the following three properties: • d(x; y) = 0 () x = y, for x; y 2 X; • d(x; y) + d(y; z) ≥ d(x; z) for all x; y; z 2 X (triangle inequality); • d(x; y) = d(y; x) for all x; y 2 X (symmetry).
    [Show full text]
  • Be a Metric Space
    2 The University of Sydney show that Z is closed in R. The complement of Z in R is the union of all the Pure Mathematics 3901 open intervals (n, n + 1), where n runs through all of Z, and this is open since every union of open sets is open. So Z is closed. Metric Spaces 2000 Alternatively, let (an) be a Cauchy sequence in Z. Choose an integer N such that d(xn, xm) < 1 for all n ≥ N. Put x = xN . Then for all n ≥ N we have Tutorial 5 |xn − x| = d(xn, xN ) < 1. But xn, x ∈ Z, and since two distinct integers always differ by at least 1 it follows that xn = x. This holds for all n > N. 1. Let X = (X, d) be a metric space. Let (xn) and (yn) be two sequences in X So xn → x as n → ∞ (since for all ε > 0 we have 0 = d(xn, x) < ε for all such that (yn) is a Cauchy sequence and d(xn, yn) → 0 as n → ∞. Prove that n > N). (i)(xn) is a Cauchy sequence in X, and 4. (i) Show that if D is a metric on the set X and f: Y → X is an injective (ii)(xn) converges to a limit x if and only if (yn) also converges to x. function then the formula d(a, b) = D(f(a), f(b)) defines a metric d on Y , and use this to show that d(m, n) = |m−1 − n−1| defines a metric Solution.
    [Show full text]
  • Semisimplicial Unital Groups
    International Journal of Theoretical Physics, Vol. 43, Nos. 7/8, August 2004 (C 2004) Semisimplicial Unital Groups David J. Foulis1 and Richard J. Greechie2 If there is an order-preserving group isomorphism from a directed abelian group G with a finitely generated positive cone G+ onto a simplicial group, then G is called a semisimplicial group. By factoring out the torsion subgroup of a unital group having a finite unit interval, one obtains a semisimplicial unital group. We exhibit a represen- tation for the base-normed space associated with a semisimplicial unital group G as the Banach dual space of a finite dimensional order-unit space that contains G as an additive subgroup. In terms of this representation, we formulate necessary and sufficient conditions for G to be archimedean. KEY WORDS: partially ordered abelian group; directed group; unital group; sim- plicial group; semisimplicial unital group; effect algebra; state; base-normed space, order-unit space. 1. INTRODUCTION If H is a Hilbert space, then the set G of all bounded self-adjoint operators on H is organized in the usual way into a partially ordered real linear space (in fact, an order-unit Banach space), and the operators belonging to the interval E :={A ∈ G | 0 ≤ A ≤ 1} are called the effect operators on H. The set E, organized into a partial algebra under the restriction ⊕ of addition on G to E, is called the algebra of effect operators on H. In the contemporary theory of quantum measurement (Busch et al., 1991), an observable is represented by a positive-operator-valued (POV) measure defined on a σ-field of sets and taking on values in the effect algebra E.
    [Show full text]
  • Chapter 1: Interval Analysis, Fuzzy Set Theory and Possibility Theory In
    Draft 1.0 November 4, 2010 CHAPTER 1 of the book Lodwick, Weldon A. (2011). Flexible and Un- certainty Optimization (to be published) Interval Analysis, Fuzzy Set Theory and Possibility Theory in Optimization Weldon A. Lodwick University of Colorado Denver Department of Mathematical and Statistical Sciences, Campus Box 170 P.O. Box 173364 Denver, CO 80217-3364, U.S.A. Email: [email protected] Abstract: This study explores the interconnections between interval analysis, fuzzy interval analysis, and interval, fuzzy, and possibility optimization. The key ideas considered are: (1) Fuzzy and possibility optimization are impor- tant methods in applied optimization problems, (2) Fuzzy sets and possibility distributions are distinct which in the context of optimization lead to ‡exible optimization on one hand and optimization under uncertainty on the other, (3) There are two ways to view possibility analysis leading to two distinct types of possibility optimization under uncertainty, single and dual distribu- tion optimization, and (4) The semantic (meaning) of constraint set in the presence of fuzziness and possibility needs to be known a-priori in order to determine what the constraint set is and how to compute its elements. The thesis of this exposition is that optimization problems that intend to model real problems are very (most) often satis…cing and epistemic and that the math- ematical language of fuzzy sets and possibility theory are well-suited theories for stating and solving a wide classes of optimization problems. Keywords: Fuzzy optimization, possibility optimization, interval analysis, constraint fuzzy interval arithmetic 1 Introduction This exposition explores interval analysis, fuzzy interval analysis, fuzzy set theory, and possibility theory as they relate to optimization which is both a synthesis of the author’s previous work bringing together, transforming, 1 and updating many ideas found in [49],[50], [51], [52], [58], [63], [64], [118], [116], and [117] as well as some new material dealing with the computation of constraint sets.
    [Show full text]
  • WHY a DEDEKIND CUT DOES NOT PRODUCE IRRATIONAL NUMBERS And, Open Intervals Are Not Sets
    WHY A DEDEKIND CUT DOES NOT PRODUCE IRRATIONAL NUMBERS And, Open Intervals are not Sets Pravin K. Johri The theory of mathematics claims that the set of real numbers is uncountable while the set of rational numbers is countable. Almost all real numbers are supposed to be irrational but there are few examples of irrational numbers relative to the rational numbers. The reality does not match the theory. Real numbers satisfy the field axioms but the simple arithmetic in these axioms can only result in rational numbers. The Dedekind cut is one of the ways mathematics rationalizes the existence of irrational numbers. Excerpts from the Wikipedia page “Dedekind cut” A Dedekind cut is а method of construction of the real numbers. It is a partition of the rational numbers into two non-empty sets A and B, such that all elements of A are less than all elements of B, and A contains no greatest element. If B has a smallest element among the rationals, the cut corresponds to that rational. Otherwise, that cut defines a unique irrational number which, loosely speaking, fills the "gap" between A and B. The countable partitions of the rational numbers cannot result in uncountable irrational numbers. Moreover, a known irrational number, or any real number for that matter, defines a Dedekind cut but it is not possible to go in the other direction and create a Dedekind cut which then produces an unknown irrational number. 1 Irrational Numbers There is an endless sequence of finite natural numbers 1, 2, 3 … based on the Peano axiom that if n is a natural number then so is n+1.
    [Show full text]
  • Topological Properties
    CHAPTER 4 Topological properties 1. Connectedness • Definitions and examples • Basic properties • Connected components • Connected versus path connected, again 2. Compactness • Definition and first examples • Topological properties of compact spaces • Compactness of products, and compactness in Rn • Compactness and continuous functions • Embeddings of compact manifolds • Sequential compactness • More about the metric case 3. Local compactness and the one-point compactification • Local compactness • The one-point compactification 4. More exercises 63 64 4. TOPOLOGICAL PROPERTIES 1. Connectedness 1.1. Definitions and examples. Definition 4.1. We say that a topological space (X, T ) is connected if X cannot be written as the union of two disjoint non-empty opens U, V ⊂ X. We say that a topological space (X, T ) is path connected if for any x, y ∈ X, there exists a path γ connecting x and y, i.e. a continuous map γ : [0, 1] → X such that γ(0) = x, γ(1) = y. Given (X, T ), we say that a subset A ⊂ X is connected (or path connected) if A, together with the induced topology, is connected (path connected). As we shall soon see, path connectedness implies connectedness. This is good news since, unlike connectedness, path connectedness can be checked more directly (see the examples below). Example 4.2. (1) X = {0, 1} with the discrete topology is not connected. Indeed, U = {0}, V = {1} are disjoint non-empty opens (in X) whose union is X. (2) Similarly, X = [0, 1) ∪ [2, 3] is not connected (take U = [0, 1), V = [2, 3]). More generally, if X ⊂ R is connected, then X must be an interval.
    [Show full text]
  • DEFINITIONS and THEOREMS in GENERAL TOPOLOGY 1. Basic
    DEFINITIONS AND THEOREMS IN GENERAL TOPOLOGY 1. Basic definitions. A topology on a set X is defined by a family O of subsets of X, the open sets of the topology, satisfying the axioms: (i) ; and X are in O; (ii) the intersection of finitely many sets in O is in O; (iii) arbitrary unions of sets in O are in O. Alternatively, a topology may be defined by the neighborhoods U(p) of an arbitrary point p 2 X, where p 2 U(p) and, in addition: (i) If U1;U2 are neighborhoods of p, there exists U3 neighborhood of p, such that U3 ⊂ U1 \ U2; (ii) If U is a neighborhood of p and q 2 U, there exists a neighborhood V of q so that V ⊂ U. A topology is Hausdorff if any distinct points p 6= q admit disjoint neigh- borhoods. This is almost always assumed. A set C ⊂ X is closed if its complement is open. The closure A¯ of a set A ⊂ X is the intersection of all closed sets containing X. A subset A ⊂ X is dense in X if A¯ = X. A point x 2 X is a cluster point of a subset A ⊂ X if any neighborhood of x contains a point of A distinct from x. If A0 denotes the set of cluster points, then A¯ = A [ A0: A map f : X ! Y of topological spaces is continuous at p 2 X if for any open neighborhood V ⊂ Y of f(p), there exists an open neighborhood U ⊂ X of p so that f(U) ⊂ V .
    [Show full text]
  • Interval Analysis and Constructive Mathematics
    16w5099—INTERVAL ANALYSIS AND CONSTRUCTIVE MATHEMATICS Douglas Bridges (University of Canterbury), Hannes Diener (University of Canterbury), Baker Kearfott (University of Louisiana at Lafayette), Vladik Kreinovich (University of Texas at El Paso), Patricia Melin (Tijuana Institute of Technology), Raazesh Sainudiin (University of Canterbury), Helmut Schwichtenberg (University of Munich) 13–18 November 2016 1 Overview of the Field 1.1 Constructive Mathematics In this case, we have two fields to overview—constructive mathematics and interval analysis—one of the main objectives of the workshop being to foster joint research across the two. By ‘constructive mathematics’ we mean ‘mathematics using intuitionistic logic and an appropriate set­ or type­theoretic foundation’. Although the origins of the field go back to Brouwer, over 100 years ago, it was the publication, in 1967, of Errett Bishop’s Foundations of Constructive Analysis [16, 17] that began the modern revival of the field. Bishop adopted the high­level viewpoint of the working mathematical analyst (he was already famous for his work in classical functional analysis and several complex variables), and devel­ oped constructively analysis across a wide swathe of the discipline: real, complex, and functional analysis, as well as abstract integration/measure theory. The significant aspect of his work is that the exclusive use of intuitionistic logic guaranteed that each proof embodied algorithms that could be extracted, encoded, and machine­implemented. For a rather simple example, Bishop’s proof of the fundamental theorem of algebra is, in effect, an algorithm enabling one to find the roots of a given complex polynomial; contrast this with the standard undergraduate proofs, such as the reductio ad absurdum one using Liouville’s theorem.
    [Show full text]