| author | wenzelm | 
| Mon, 06 Mar 2023 10:16:40 +0100 | |
| changeset 77534 | fc57886e37dd | 
| parent 77138 | c8597292cd41 | 
| child 77934 | 01c88cf514fc | 
| permissions | -rw-r--r-- | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 1 | (* Author: L C Paulson, University of Cambridge | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 2 | Author: Amine Chaieb, University of Cambridge | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 3 | Author: Robert Himmelmann, TU Muenchen | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 4 | Author: Brian Huffman, Portland State University | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 5 | *) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 6 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 7 | section \<open>Abstract Topology 2\<close> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 8 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 9 | theory Abstract_Topology_2 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 10 | imports | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 11 | Elementary_Topology | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 12 | Abstract_Topology | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 13 | "HOL-Library.Indicator_Function" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 14 | begin | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 15 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 16 | text \<open>Combination of Elementary and Abstract Topology\<close> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 17 | |
| 72225 | 18 | lemma approachable_lt_le2: | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 19 | "(\<exists>(d::real) > 0. \<forall>x. Q x \<longrightarrow> f x < d \<longrightarrow> P x) \<longleftrightarrow> (\<exists>d>0. \<forall>x. f x \<le> d \<longrightarrow> Q x \<longrightarrow> P x)" | 
| 76894 | 20 | by (meson dense less_eq_real_def order_le_less_trans) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 21 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 22 | lemma triangle_lemma: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 23 | fixes x y z :: real | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 24 | assumes x: "0 \<le> x" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 25 | and y: "0 \<le> y" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 26 | and z: "0 \<le> z" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 27 | and xy: "x\<^sup>2 \<le> y\<^sup>2 + z\<^sup>2" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 28 | shows "x \<le> y + z" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 29 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 30 | have "y\<^sup>2 + z\<^sup>2 \<le> y\<^sup>2 + 2 * y * z + z\<^sup>2" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 31 | using z y by simp | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 32 | with xy have th: "x\<^sup>2 \<le> (y + z)\<^sup>2" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 33 | by (simp add: power2_eq_square field_simps) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 34 | from y z have yz: "y + z \<ge> 0" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 35 | by arith | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 36 | from power2_le_imp_le[OF th yz] show ?thesis . | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 37 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 38 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 39 | lemma isCont_indicator: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 40 | fixes x :: "'a::t2_space" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 41 | shows "isCont (indicator A :: 'a \<Rightarrow> real) x = (x \<notin> frontier A)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 42 | proof auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 43 | fix x | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 44 | assume cts_at: "isCont (indicator A :: 'a \<Rightarrow> real) x" and fr: "x \<in> frontier A" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 45 | with continuous_at_open have 1: "\<forall>V::real set. open V \<and> indicator A x \<in> V \<longrightarrow> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 46 | (\<exists>U::'a set. open U \<and> x \<in> U \<and> (\<forall>y\<in>U. indicator A y \<in> V))" by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 47 | show False | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 48 | proof (cases "x \<in> A") | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 49 | assume x: "x \<in> A" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 50 |     hence "indicator A x \<in> ({0<..<2} :: real set)" by simp
 | 
| 74362 | 51 |     with 1 obtain U where U: "open U" "x \<in> U" "\<forall>y\<in>U. indicator A y \<in> ({0<..<2} :: real set)"
 | 
| 52 | using open_greaterThanLessThan by metis | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 53 | hence "\<forall>y\<in>U. indicator A y > (0::real)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 54 | unfolding greaterThanLessThan_def by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 55 | hence "U \<subseteq> A" using indicator_eq_0_iff by force | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 56 | hence "x \<in> interior A" using U interiorI by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 57 | thus ?thesis using fr unfolding frontier_def by simp | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 58 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 59 | assume x: "x \<notin> A" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 60 |     hence "indicator A x \<in> ({-1<..<1} :: real set)" by simp
 | 
| 74362 | 61 |     with 1 obtain U where U: "open U" "x \<in> U" "\<forall>y\<in>U. indicator A y \<in> ({-1<..<1} :: real set)"
 | 
| 62 | using 1 open_greaterThanLessThan by metis | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 63 | hence "\<forall>y\<in>U. indicator A y < (1::real)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 64 | unfolding greaterThanLessThan_def by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 65 | hence "U \<subseteq> -A" by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 66 | hence "x \<in> interior (-A)" using U interiorI by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 67 | thus ?thesis using fr interior_complement unfolding frontier_def by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 68 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 69 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 70 | assume nfr: "x \<notin> frontier A" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 71 | hence "x \<in> interior A \<or> x \<in> interior (-A)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 72 | by (auto simp: frontier_def closure_interior) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 73 | thus "isCont ((indicator A)::'a \<Rightarrow> real) x" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 74 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 75 | assume int: "x \<in> interior A" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 76 | then obtain U where U: "open U" "x \<in> U" "U \<subseteq> A" unfolding interior_def by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 77 | hence "\<forall>y\<in>U. indicator A y = (1::real)" unfolding indicator_def by auto | 
| 71172 | 78 | hence "continuous_on U (indicator A)" by (simp add: indicator_eq_1_iff) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 79 | thus ?thesis using U continuous_on_eq_continuous_at by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 80 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 81 | assume ext: "x \<in> interior (-A)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 82 | then obtain U where U: "open U" "x \<in> U" "U \<subseteq> -A" unfolding interior_def by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 83 | then have "continuous_on U (indicator A)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 84 | using continuous_on_topological by (auto simp: subset_iff) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 85 | thus ?thesis using U continuous_on_eq_continuous_at by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 86 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 87 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 88 | |
| 76894 | 89 | lemma islimpt_closure: | 
| 90 | "\<lbrakk>S \<subseteq> T; \<And>x. \<lbrakk>x islimpt S; x \<in> T\<rbrakk> \<Longrightarrow> x \<in> S\<rbrakk> \<Longrightarrow> S = T \<inter> closure S" | |
| 91 | using closure_def by fastforce | |
| 92 | ||
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 93 | lemma closedin_limpt: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 94 | "closedin (top_of_set T) S \<longleftrightarrow> S \<subseteq> T \<and> (\<forall>x. x islimpt S \<and> x \<in> T \<longrightarrow> x \<in> S)" | 
| 76894 | 95 | proof - | 
| 96 | have "\<And>U x. \<lbrakk>closed U; S = T \<inter> U; x islimpt S; x \<in> T\<rbrakk> \<Longrightarrow> x \<in> S" | |
| 97 | by (meson IntI closed_limpt inf_le2 islimpt_subset) | |
| 98 | then show ?thesis | |
| 99 | by (metis closed_closure closedin_closed closedin_imp_subset islimpt_closure) | |
| 100 | qed | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 101 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 102 | lemma closedin_closed_eq: "closed S \<Longrightarrow> closedin (top_of_set S) T \<longleftrightarrow> closed T \<and> T \<subseteq> S" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 103 | by (meson closedin_limpt closed_subset closedin_closed_trans) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 104 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 105 | lemma connected_closed_set: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 106 | "closed S | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 107 |     \<Longrightarrow> connected S \<longleftrightarrow> (\<nexists>A B. closed A \<and> closed B \<and> A \<noteq> {} \<and> B \<noteq> {} \<and> A \<union> B = S \<and> A \<inter> B = {})"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 108 | unfolding connected_closedin_eq closedin_closed_eq connected_closedin_eq by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 109 | |
| 76894 | 110 | text \<open>If a connnected set is written as the union of two nonempty closed sets, | 
| 111 | then these sets have to intersect.\<close> | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 112 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 113 | lemma connected_as_closed_union: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 114 |   assumes "connected C" "C = A \<union> B" "closed A" "closed B" "A \<noteq> {}" "B \<noteq> {}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 115 |   shows "A \<inter> B \<noteq> {}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 116 | by (metis assms closed_Un connected_closed_set) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 117 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 118 | lemma closedin_subset_trans: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 119 | "closedin (top_of_set U) S \<Longrightarrow> S \<subseteq> T \<Longrightarrow> T \<subseteq> U \<Longrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 120 | closedin (top_of_set T) S" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 121 | by (meson closedin_limpt subset_iff) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 122 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 123 | lemma openin_subset_trans: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 124 | "openin (top_of_set U) S \<Longrightarrow> S \<subseteq> T \<Longrightarrow> T \<subseteq> U \<Longrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 125 | openin (top_of_set T) S" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 126 | by (auto simp: openin_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 127 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 128 | lemma closedin_compact: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 129 | "\<lbrakk>compact S; closedin (top_of_set S) T\<rbrakk> \<Longrightarrow> compact T" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 130 | by (metis closedin_closed compact_Int_closed) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 131 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 132 | lemma closedin_compact_eq: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 133 | fixes S :: "'a::t2_space set" | 
| 76894 | 134 | shows "compact S \<Longrightarrow> (closedin (top_of_set S) T \<longleftrightarrow> compact T \<and> T \<subseteq> S)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 135 | by (metis closedin_imp_subset closedin_compact closed_subset compact_imp_closed) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 136 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 137 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 138 | subsection \<open>Closure\<close> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 139 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 140 | lemma euclidean_closure_of [simp]: "euclidean closure_of S = closure S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 141 | by (auto simp: closure_of_def closure_def islimpt_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 142 | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 143 | lemma closure_openin_Int_closure: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 144 | assumes ope: "openin (top_of_set U) S" and "T \<subseteq> U" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 145 | shows "closure(S \<inter> closure T) = closure(S \<inter> T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 146 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 147 | obtain V where "open V" and S: "S = U \<inter> V" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 148 | using ope using openin_open by metis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 149 | show "closure (S \<inter> closure T) \<subseteq> closure (S \<inter> T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 150 | proof (clarsimp simp: S) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 151 | fix x | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 152 | assume "x \<in> closure (U \<inter> V \<inter> closure T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 153 | then have "V \<inter> closure T \<subseteq> A \<Longrightarrow> x \<in> closure A" for A | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 154 | by (metis closure_mono subsetD inf.coboundedI2 inf_assoc) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 155 | then have "x \<in> closure (T \<inter> V)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 156 | by (metis \<open>open V\<close> closure_closure inf_commute open_Int_closure_subset) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 157 | then show "x \<in> closure (U \<inter> V \<inter> T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 158 | by (metis \<open>T \<subseteq> U\<close> inf.absorb_iff2 inf_assoc inf_commute) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 159 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 160 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 161 | show "closure (S \<inter> T) \<subseteq> closure (S \<inter> closure T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 162 | by (meson Int_mono closure_mono closure_subset order_refl) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 163 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 164 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 165 | corollary infinite_openin: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 166 | fixes S :: "'a :: t1_space set" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 167 | shows "\<lbrakk>openin (top_of_set U) S; x \<in> S; x islimpt U\<rbrakk> \<Longrightarrow> infinite S" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 168 | by (clarsimp simp add: openin_open islimpt_eq_acc_point inf_commute) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 169 | |
| 69622 | 170 | lemma closure_Int_ballI: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 171 |   assumes "\<And>U. \<lbrakk>openin (top_of_set S) U; U \<noteq> {}\<rbrakk> \<Longrightarrow> T \<inter> U \<noteq> {}"
 | 
| 69622 | 172 | shows "S \<subseteq> closure T" | 
| 173 | proof (clarsimp simp: closure_iff_nhds_not_empty) | |
| 174 | fix x and A and V | |
| 175 |   assume "x \<in> S" "V \<subseteq> A" "open V" "x \<in> V" "T \<inter> A = {}"
 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 176 | then have "openin (top_of_set S) (A \<inter> V \<inter> S)" | 
| 76894 | 177 | by (simp add: inf_absorb2 openin_subtopology_Int) | 
| 69622 | 178 |   moreover have "A \<inter> V \<inter> S \<noteq> {}" using \<open>x \<in> V\<close> \<open>V \<subseteq> A\<close> \<open>x \<in> S\<close>
 | 
| 179 | by auto | |
| 76894 | 180 | ultimately show False | 
| 181 |     using \<open>T \<inter> A = {}\<close> assms by fastforce
 | |
| 69622 | 182 | qed | 
| 183 | ||
| 184 | ||
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 185 | subsection \<open>Frontier\<close> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 186 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 187 | lemma euclidean_interior_of [simp]: "euclidean interior_of S = interior S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 188 | by (auto simp: interior_of_def interior_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 189 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 190 | lemma euclidean_frontier_of [simp]: "euclidean frontier_of S = frontier S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 191 | by (auto simp: frontier_of_def frontier_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 192 | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 193 | lemma connected_Int_frontier: | 
| 76894 | 194 |      "\<lbrakk>connected S; S \<inter> T \<noteq> {}; S - T \<noteq> {}\<rbrakk> \<Longrightarrow> S \<inter> frontier T \<noteq> {}"
 | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 195 | apply (simp add: frontier_interiors connected_openin, safe) | 
| 76894 | 196 | apply (drule_tac x="S \<inter> interior T" in spec, safe) | 
| 197 | apply (drule_tac [2] x="S \<inter> interior (-T)" in spec) | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 198 | apply (auto simp: disjoint_eq_subset_Compl dest: interior_subset [THEN subsetD]) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 199 | done | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 200 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 201 | subsection \<open>Compactness\<close> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 202 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 203 | lemma openin_delete: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 204 | fixes a :: "'a :: t1_space" | 
| 76894 | 205 |   shows "openin (top_of_set u) S \<Longrightarrow> openin (top_of_set u) (S - {a})"
 | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 206 | by (metis Int_Diff open_delete openin_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 207 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 208 | lemma compact_eq_openin_cover: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 209 | "compact S \<longleftrightarrow> | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 210 | (\<forall>C. (\<forall>c\<in>C. openin (top_of_set S) c) \<and> S \<subseteq> \<Union>C \<longrightarrow> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 211 | (\<exists>D\<subseteq>C. finite D \<and> S \<subseteq> \<Union>D))" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 212 | proof safe | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 213 | fix C | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 214 | assume "compact S" and "\<forall>c\<in>C. openin (top_of_set S) c" and "S \<subseteq> \<Union>C" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 215 |   then have "\<forall>c\<in>{T. open T \<and> S \<inter> T \<in> C}. open c" and "S \<subseteq> \<Union>{T. open T \<and> S \<inter> T \<in> C}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 216 | unfolding openin_open by force+ | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 217 |   with \<open>compact S\<close> obtain D where "D \<subseteq> {T. open T \<and> S \<inter> T \<in> C}" and "finite D" and "S \<subseteq> \<Union>D"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 218 | by (meson compactE) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 219 | then have "image (\<lambda>T. S \<inter> T) D \<subseteq> C \<and> finite (image (\<lambda>T. S \<inter> T) D) \<and> S \<subseteq> \<Union>(image (\<lambda>T. S \<inter> T) D)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 220 | by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 221 | then show "\<exists>D\<subseteq>C. finite D \<and> S \<subseteq> \<Union>D" .. | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 222 | next | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 223 | assume 1: "\<forall>C. (\<forall>c\<in>C. openin (top_of_set S) c) \<and> S \<subseteq> \<Union>C \<longrightarrow> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 224 | (\<exists>D\<subseteq>C. finite D \<and> S \<subseteq> \<Union>D)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 225 | show "compact S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 226 | proof (rule compactI) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 227 | fix C | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 228 | let ?C = "image (\<lambda>T. S \<inter> T) C" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 229 | assume "\<forall>t\<in>C. open t" and "S \<subseteq> \<Union>C" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 230 | then have "(\<forall>c\<in>?C. openin (top_of_set S) c) \<and> S \<subseteq> \<Union>?C" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 231 | unfolding openin_open by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 232 | with 1 obtain D where "D \<subseteq> ?C" and "finite D" and "S \<subseteq> \<Union>D" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 233 | by metis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 234 | let ?D = "inv_into C (\<lambda>T. S \<inter> T) ` D" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 235 | have "?D \<subseteq> C \<and> finite ?D \<and> S \<subseteq> \<Union>?D" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 236 | proof (intro conjI) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 237 | from \<open>D \<subseteq> ?C\<close> show "?D \<subseteq> C" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 238 | by (fast intro: inv_into_into) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 239 | from \<open>finite D\<close> show "finite ?D" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 240 | by (rule finite_imageI) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 241 | from \<open>S \<subseteq> \<Union>D\<close> show "S \<subseteq> \<Union>?D" | 
| 76894 | 242 | by (metis \<open>D \<subseteq> (\<inter>) S ` C\<close> image_inv_into_cancel inf_Sup le_infE) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 243 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 244 | then show "\<exists>D\<subseteq>C. finite D \<and> S \<subseteq> \<Union>D" .. | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 245 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 246 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 247 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 248 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 249 | subsection \<open>Continuity\<close> | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 250 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 251 | lemma interior_image_subset: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 252 | assumes "inj f" "\<And>x. continuous (at x) f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 253 | shows "interior (f ` S) \<subseteq> f ` (interior S)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 254 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 255 | fix x assume "x \<in> interior (f ` S)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 256 | then obtain T where as: "open T" "x \<in> T" "T \<subseteq> f ` S" .. | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 257 | then have "x \<in> f ` S" by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 258 | then obtain y where y: "y \<in> S" "x = f y" by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 259 | have "open (f -` T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 260 | using assms \<open>open T\<close> by (simp add: continuous_at_imp_continuous_on open_vimage) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 261 | moreover have "y \<in> vimage f T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 262 | using \<open>x = f y\<close> \<open>x \<in> T\<close> by simp | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 263 | moreover have "vimage f T \<subseteq> S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 264 | using \<open>T \<subseteq> image f S\<close> \<open>inj f\<close> unfolding inj_on_def subset_eq by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 265 | ultimately have "y \<in> interior S" .. | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 266 | with \<open>x = f y\<close> show "x \<in> f ` interior S" .. | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 267 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 268 | |
| 70136 | 269 | subsection\<^marker>\<open>tag unimportant\<close> \<open>Equality of continuous functions on closure and related results\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 270 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 271 | lemma continuous_closedin_preimage_constant: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 272 | fixes f :: "_ \<Rightarrow> 'b::t1_space" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 273 |   shows "continuous_on S f \<Longrightarrow> closedin (top_of_set S) {x \<in> S. f x = a}"
 | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 274 |   using continuous_closedin_preimage[of S f "{a}"] by (simp add: vimage_def Collect_conj_eq)
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 275 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 276 | lemma continuous_closed_preimage_constant: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 277 | fixes f :: "_ \<Rightarrow> 'b::t1_space" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 278 |   shows "continuous_on S f \<Longrightarrow> closed S \<Longrightarrow> closed {x \<in> S. f x = a}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 279 |   using continuous_closed_preimage[of S f "{a}"] by (simp add: vimage_def Collect_conj_eq)
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 280 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 281 | lemma continuous_constant_on_closure: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 282 | fixes f :: "_ \<Rightarrow> 'b::t1_space" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 283 | assumes "continuous_on (closure S) f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 284 | and "\<And>x. x \<in> S \<Longrightarrow> f x = a" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 285 | and "x \<in> closure S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 286 | shows "f x = a" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 287 | using continuous_closed_preimage_constant[of "closure S" f a] | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 288 |       assms closure_minimal[of S "{x \<in> closure S. f x = a}"] closure_subset
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 289 | unfolding subset_eq | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 290 | by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 291 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 292 | lemma image_closure_subset: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 293 | assumes contf: "continuous_on (closure S) f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 294 | and "closed T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 295 | and "(f ` S) \<subseteq> T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 296 | shows "f ` (closure S) \<subseteq> T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 297 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 298 |   have "S \<subseteq> {x \<in> closure S. f x \<in> T}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 299 | using assms(3) closure_subset by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 300 | moreover have "closed (closure S \<inter> f -` T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 301 | using continuous_closed_preimage[OF contf] \<open>closed T\<close> by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 302 | ultimately have "closure S = (closure S \<inter> f -` T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 303 | using closure_minimal[of S "(closure S \<inter> f -` T)"] by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 304 | then show ?thesis by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 305 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 306 | |
| 70136 | 307 | subsection\<^marker>\<open>tag unimportant\<close> \<open>A function constant on a set\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 308 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 309 | definition constant_on (infixl "(constant'_on)" 50) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 310 | where "f constant_on A \<equiv> \<exists>y. \<forall>x\<in>A. f x = y" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 311 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 312 | lemma constant_on_subset: "\<lbrakk>f constant_on A; B \<subseteq> A\<rbrakk> \<Longrightarrow> f constant_on B" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 313 | unfolding constant_on_def by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 314 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 315 | lemma injective_not_constant: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 316 |   fixes S :: "'a::{perfect_space} set"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 317 |   shows "\<lbrakk>open S; inj_on f S; f constant_on S\<rbrakk> \<Longrightarrow> S = {}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 318 | unfolding constant_on_def | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 319 | by (metis equals0I inj_on_contraD islimpt_UNIV islimpt_def) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 320 | |
| 77138 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 321 | lemma constant_on_compose: | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 322 | assumes "f constant_on A" | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 323 | shows "g \<circ> f constant_on A" | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 324 | using assms by (auto simp: constant_on_def) | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 325 | |
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 326 | lemma not_constant_onI: | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 327 | "f x \<noteq> f y \<Longrightarrow> x \<in> A \<Longrightarrow> y \<in> A \<Longrightarrow> \<not>f constant_on A" | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 328 | unfolding constant_on_def by metis | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 329 | |
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 330 | lemma constant_onE: | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 331 | assumes "f constant_on S" and "\<And>x. x\<in>S \<Longrightarrow> f x = g x" | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 332 | shows "g constant_on S" | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 333 | using assms unfolding constant_on_def by simp | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 334 | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 335 | lemma constant_on_closureI: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 336 | fixes f :: "_ \<Rightarrow> 'b::t1_space" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 337 | assumes cof: "f constant_on S" and contf: "continuous_on (closure S) f" | 
| 77138 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 338 | shows "f constant_on (closure S)" | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 339 | using continuous_constant_on_closure [OF contf] cof unfolding constant_on_def | 
| 
c8597292cd41
Moved in a large number of highly useful library lemmas, mostly due to Manuel Eberl
 paulson <lp15@cam.ac.uk> parents: 
76894diff
changeset | 340 | by metis | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 341 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 342 | |
| 70136 | 343 | subsection\<^marker>\<open>tag unimportant\<close> \<open>Continuity relative to a union.\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 344 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 345 | lemma continuous_on_Un_local: | 
| 76894 | 346 | "\<lbrakk>closedin (top_of_set (S \<union> T)) S; closedin (top_of_set (S \<union> T)) T; | 
| 347 | continuous_on S f; continuous_on T f\<rbrakk> | |
| 348 | \<Longrightarrow> continuous_on (S \<union> T) f" | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 349 | unfolding continuous_on closedin_limpt | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 350 | by (metis Lim_trivial_limit Lim_within_union Un_iff trivial_limit_within) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 351 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 352 | lemma continuous_on_cases_local: | 
| 76894 | 353 | "\<lbrakk>closedin (top_of_set (S \<union> T)) S; closedin (top_of_set (S \<union> T)) T; | 
| 354 | continuous_on S f; continuous_on T g; | |
| 355 | \<And>x. \<lbrakk>x \<in> S \<and> \<not>P x \<or> x \<in> T \<and> P x\<rbrakk> \<Longrightarrow> f x = g x\<rbrakk> | |
| 356 | \<Longrightarrow> continuous_on (S \<union> T) (\<lambda>x. if P x then f x else g x)" | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 357 | by (rule continuous_on_Un_local) (auto intro: continuous_on_eq) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 358 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 359 | lemma continuous_on_cases_le: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 360 | fixes h :: "'a :: topological_space \<Rightarrow> real" | 
| 76894 | 361 |   assumes "continuous_on {x \<in> S. h x \<le> a} f"
 | 
| 362 |       and "continuous_on {x \<in> S. a \<le> h x} g"
 | |
| 363 | and h: "continuous_on S h" | |
| 364 | and "\<And>x. \<lbrakk>x \<in> S; h x = a\<rbrakk> \<Longrightarrow> f x = g x" | |
| 365 | shows "continuous_on S (\<lambda>x. if h x \<le> a then f(x) else g(x))" | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 366 | proof - | 
| 76894 | 367 | have S: "S = (S \<inter> h -` atMost a) \<union> (S \<inter> h -` atLeast a)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 368 | by force | 
| 76894 | 369 | have 1: "closedin (top_of_set S) (S \<inter> h -` atMost a)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 370 | by (rule continuous_closedin_preimage [OF h closed_atMost]) | 
| 76894 | 371 | have 2: "closedin (top_of_set S) (S \<inter> h -` atLeast a)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 372 | by (rule continuous_closedin_preimage [OF h closed_atLeast]) | 
| 76894 | 373 |   have [simp]: "S \<inter> h -` {..a} = {x \<in> S. h x \<le> a}" "S \<inter> h -` {a..} = {x \<in> S. a \<le> h x}"
 | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 374 | by auto | 
| 76894 | 375 |   have "continuous_on (S \<inter> h -` {..a} \<union> S \<inter> h -` {a..}) (\<lambda>x. if h x \<le> a then f x else g x)"
 | 
| 376 | by (intro continuous_on_cases_local) (use 1 2 S assms in auto) | |
| 377 | then show ?thesis | |
| 378 | using S by force | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 379 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 380 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 381 | lemma continuous_on_cases_1: | 
| 76894 | 382 | fixes S :: "real set" | 
| 383 |   assumes "continuous_on {t \<in> S. t \<le> a} f"
 | |
| 384 |       and "continuous_on {t \<in> S. a \<le> t} g"
 | |
| 385 | and "a \<in> S \<Longrightarrow> f a = g a" | |
| 386 | shows "continuous_on S (\<lambda>t. if t \<le> a then f(t) else g(t))" | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 387 | using assms | 
| 71172 | 388 | by (auto intro: continuous_on_cases_le [where h = id, simplified]) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 389 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 390 | |
| 70136 | 391 | subsection\<^marker>\<open>tag unimportant\<close>\<open>Inverse function property for open/closed maps\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 392 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 393 | lemma continuous_on_inverse_open_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 394 | assumes contf: "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 395 | and imf: "f ` S = T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 396 | and injf: "\<And>x. x \<in> S \<Longrightarrow> g (f x) = x" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 397 | and oo: "\<And>U. openin (top_of_set S) U \<Longrightarrow> openin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 398 | shows "continuous_on T g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 399 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 400 | from imf injf have gTS: "g ` T = S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 401 | by force | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 402 | from imf injf have fU: "U \<subseteq> S \<Longrightarrow> (f ` U) = T \<inter> g -` U" for U | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 403 | by force | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 404 | show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 405 | by (simp add: continuous_on_open [of T g] gTS) (metis openin_imp_subset fU oo) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 406 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 407 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 408 | lemma continuous_on_inverse_closed_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 409 | assumes contf: "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 410 | and imf: "f ` S = T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 411 | and injf: "\<And>x. x \<in> S \<Longrightarrow> g(f x) = x" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 412 | and oo: "\<And>U. closedin (top_of_set S) U \<Longrightarrow> closedin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 413 | shows "continuous_on T g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 414 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 415 | from imf injf have gTS: "g ` T = S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 416 | by force | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 417 | from imf injf have fU: "U \<subseteq> S \<Longrightarrow> (f ` U) = T \<inter> g -` U" for U | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 418 | by force | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 419 | show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 420 | by (simp add: continuous_on_closed [of T g] gTS) (metis closedin_imp_subset fU oo) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 421 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 422 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 423 | lemma homeomorphism_injective_open_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 424 | assumes contf: "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 425 | and imf: "f ` S = T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 426 | and injf: "inj_on f S" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 427 | and oo: "\<And>U. openin (top_of_set S) U \<Longrightarrow> openin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 428 | obtains g where "homeomorphism S T f g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 429 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 430 | have "continuous_on T (inv_into S f)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 431 | by (metis contf continuous_on_inverse_open_map imf injf inv_into_f_f oo) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 432 | with imf injf contf show "homeomorphism S T f (inv_into S f)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 433 | by (auto simp: homeomorphism_def) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 434 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 435 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 436 | lemma homeomorphism_injective_closed_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 437 | assumes contf: "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 438 | and imf: "f ` S = T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 439 | and injf: "inj_on f S" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 440 | and oo: "\<And>U. closedin (top_of_set S) U \<Longrightarrow> closedin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 441 | obtains g where "homeomorphism S T f g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 442 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 443 | have "continuous_on T (inv_into S f)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 444 | by (metis contf continuous_on_inverse_closed_map imf injf inv_into_f_f oo) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 445 | with imf injf contf show "homeomorphism S T f (inv_into S f)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 446 | by (auto simp: homeomorphism_def) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 447 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 448 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 449 | lemma homeomorphism_imp_open_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 450 | assumes hom: "homeomorphism S T f g" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 451 | and oo: "openin (top_of_set S) U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 452 | shows "openin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 453 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 454 | from hom oo have [simp]: "f ` U = T \<inter> g -` U" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 455 | using openin_subset by (fastforce simp: homeomorphism_def rev_image_eqI) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 456 | from hom have "continuous_on T g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 457 | unfolding homeomorphism_def by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 458 | moreover have "g ` T = S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 459 | by (metis hom homeomorphism_def) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 460 | ultimately show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 461 | by (simp add: continuous_on_open oo) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 462 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 463 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 464 | lemma homeomorphism_imp_closed_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 465 | assumes hom: "homeomorphism S T f g" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 466 | and oo: "closedin (top_of_set S) U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 467 | shows "closedin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 468 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 469 | from hom oo have [simp]: "f ` U = T \<inter> g -` U" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 470 | using closedin_subset by (fastforce simp: homeomorphism_def rev_image_eqI) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 471 | from hom have "continuous_on T g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 472 | unfolding homeomorphism_def by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 473 | moreover have "g ` T = S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 474 | by (metis hom homeomorphism_def) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 475 | ultimately show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 476 | by (simp add: continuous_on_closed oo) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 477 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 478 | |
| 70136 | 479 | subsection\<^marker>\<open>tag unimportant\<close> \<open>Seperability\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 480 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 481 | lemma subset_second_countable: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 482 | obtains \<B> :: "'a:: second_countable_topology set set" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 483 | where "countable \<B>" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 484 |           "{} \<notin> \<B>"
 | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 485 | "\<And>C. C \<in> \<B> \<Longrightarrow> openin(top_of_set S) C" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 486 | "\<And>T. openin(top_of_set S) T \<Longrightarrow> \<exists>\<U>. \<U> \<subseteq> \<B> \<and> T = \<Union>\<U>" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 487 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 488 | obtain \<B> :: "'a set set" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 489 | where "countable \<B>" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 490 | and opeB: "\<And>C. C \<in> \<B> \<Longrightarrow> openin(top_of_set S) C" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 491 | and \<B>: "\<And>T. openin(top_of_set S) T \<Longrightarrow> \<exists>\<U>. \<U> \<subseteq> \<B> \<and> T = \<Union>\<U>" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 492 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 493 | obtain \<C> :: "'a set set" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 494 | where "countable \<C>" and ope: "\<And>C. C \<in> \<C> \<Longrightarrow> open C" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 495 | and \<C>: "\<And>S. open S \<Longrightarrow> \<exists>U. U \<subseteq> \<C> \<and> S = \<Union>U" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 496 | by (metis univ_second_countable that) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 497 | show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 498 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 499 | show "countable ((\<lambda>C. S \<inter> C) ` \<C>)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 500 | by (simp add: \<open>countable \<C>\<close>) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 501 | show "\<And>C. C \<in> (\<inter>) S ` \<C> \<Longrightarrow> openin (top_of_set S) C" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 502 | using ope by auto | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 503 | show "\<And>T. openin (top_of_set S) T \<Longrightarrow> \<exists>\<U>\<subseteq>(\<inter>) S ` \<C>. T = \<Union>\<U>" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 504 | by (metis \<C> image_mono inf_Sup openin_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 505 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 506 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 507 | show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 508 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 509 |     show "countable (\<B> - {{}})"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 510 | using \<open>countable \<B>\<close> by blast | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 511 |     show "\<And>C. \<lbrakk>C \<in> \<B> - {{}}\<rbrakk> \<Longrightarrow> openin (top_of_set S) C"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 512 | by (simp add: \<open>\<And>C. C \<in> \<B> \<Longrightarrow> openin (top_of_set S) C\<close>) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 513 |     show "\<exists>\<U>\<subseteq>\<B> - {{}}. T = \<Union>\<U>" if "openin (top_of_set S) T" for T
 | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 514 | using \<B> [OF that] | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 515 | apply clarify | 
| 76894 | 516 |       by (rule_tac x="\<U> - {{}}" in exI, auto)
 | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 517 | qed auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 518 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 519 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 520 | lemma Lindelof_openin: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 521 | fixes \<F> :: "'a::second_countable_topology set set" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 522 | assumes "\<And>S. S \<in> \<F> \<Longrightarrow> openin (top_of_set U) S" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 523 | obtains \<F>' where "\<F>' \<subseteq> \<F>" "countable \<F>'" "\<Union>\<F>' = \<Union>\<F>" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 524 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 525 | have "\<And>S. S \<in> \<F> \<Longrightarrow> \<exists>T. open T \<and> S = U \<inter> T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 526 | using assms by (simp add: openin_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 527 | then obtain tf where tf: "\<And>S. S \<in> \<F> \<Longrightarrow> open (tf S) \<and> (S = U \<inter> tf S)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 528 | by metis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 529 | have [simp]: "\<And>\<F>'. \<F>' \<subseteq> \<F> \<Longrightarrow> \<Union>\<F>' = U \<inter> \<Union>(tf ` \<F>')" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 530 | using tf by fastforce | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 531 | obtain \<G> where "countable \<G> \<and> \<G> \<subseteq> tf ` \<F>" "\<Union>\<G> = \<Union>(tf ` \<F>)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 532 | using tf by (force intro: Lindelof [of "tf ` \<F>"]) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 533 | then obtain \<F>' where \<F>': "\<F>' \<subseteq> \<F>" "countable \<F>'" "\<Union>\<F>' = \<Union>\<F>" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 534 | by (clarsimp simp add: countable_subset_image) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 535 | then show ?thesis .. | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 536 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 537 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 538 | |
| 70136 | 539 | subsection\<^marker>\<open>tag unimportant\<close>\<open>Closed Maps\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 540 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 541 | lemma continuous_imp_closed_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 542 | fixes f :: "'a::t2_space \<Rightarrow> 'b::t2_space" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 543 | assumes "closedin (top_of_set S) U" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 544 | "continuous_on S f" "f ` S = T" "compact S" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 545 | shows "closedin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 546 | by (metis assms closedin_compact_eq compact_continuous_image continuous_on_subset subset_image_iff) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 547 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 548 | lemma closed_map_restrict: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 549 | assumes cloU: "closedin (top_of_set (S \<inter> f -` T')) U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 550 | and cc: "\<And>U. closedin (top_of_set S) U \<Longrightarrow> closedin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 551 | and "T' \<subseteq> T" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 552 | shows "closedin (top_of_set T') (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 553 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 554 | obtain V where "closed V" "U = S \<inter> f -` T' \<inter> V" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 555 | using cloU by (auto simp: closedin_closed) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 556 | with cc [of "S \<inter> V"] \<open>T' \<subseteq> T\<close> show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 557 | by (fastforce simp add: closedin_closed) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 558 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 559 | |
| 70136 | 560 | subsection\<^marker>\<open>tag unimportant\<close>\<open>Open Maps\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 561 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 562 | lemma open_map_restrict: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 563 | assumes opeU: "openin (top_of_set (S \<inter> f -` T')) U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 564 | and oo: "\<And>U. openin (top_of_set S) U \<Longrightarrow> openin (top_of_set T) (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 565 | and "T' \<subseteq> T" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 566 | shows "openin (top_of_set T') (f ` U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 567 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 568 | obtain V where "open V" "U = S \<inter> f -` T' \<inter> V" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 569 | using opeU by (auto simp: openin_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 570 | with oo [of "S \<inter> V"] \<open>T' \<subseteq> T\<close> show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 571 | by (fastforce simp add: openin_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 572 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 573 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 574 | |
| 70136 | 575 | subsection\<^marker>\<open>tag unimportant\<close>\<open>Quotient maps\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 576 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 577 | lemma quotient_map_imp_continuous_open: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 578 | assumes T: "f ` S \<subseteq> T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 579 | and ope: "\<And>U. U \<subseteq> T | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 580 | \<Longrightarrow> (openin (top_of_set S) (S \<inter> f -` U) \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 581 | openin (top_of_set T) U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 582 | shows "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 583 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 584 | have [simp]: "S \<inter> f -` f ` S = S" by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 585 | show ?thesis | 
| 72225 | 586 | by (meson T continuous_on_open_gen ope openin_imp_subset) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 587 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 588 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 589 | lemma quotient_map_imp_continuous_closed: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 590 | assumes T: "f ` S \<subseteq> T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 591 | and ope: "\<And>U. U \<subseteq> T | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 592 | \<Longrightarrow> (closedin (top_of_set S) (S \<inter> f -` U) \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 593 | closedin (top_of_set T) U)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 594 | shows "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 595 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 596 | have [simp]: "S \<inter> f -` f ` S = S" by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 597 | show ?thesis | 
| 72225 | 598 | by (meson T closedin_imp_subset continuous_on_closed_gen ope) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 599 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 600 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 601 | lemma open_map_imp_quotient_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 602 | assumes contf: "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 603 | and T: "T \<subseteq> f ` S" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 604 | and ope: "\<And>T. openin (top_of_set S) T | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 605 | \<Longrightarrow> openin (top_of_set (f ` S)) (f ` T)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 606 | shows "openin (top_of_set S) (S \<inter> f -` T) = | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 607 | openin (top_of_set (f ` S)) T" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 608 | proof - | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 609 | have "T = f ` (S \<inter> f -` T)" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 610 | using T by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 611 | then show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 612 | using "ope" contf continuous_on_open by metis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 613 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 614 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 615 | lemma closed_map_imp_quotient_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 616 | assumes contf: "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 617 | and T: "T \<subseteq> f ` S" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 618 | and ope: "\<And>T. closedin (top_of_set S) T | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 619 | \<Longrightarrow> closedin (top_of_set (f ` S)) (f ` T)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 620 | shows "openin (top_of_set S) (S \<inter> f -` T) \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 621 | openin (top_of_set (f ` S)) T" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 622 | (is "?lhs = ?rhs") | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 623 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 624 | assume ?lhs | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 625 | then have *: "closedin (top_of_set S) (S - (S \<inter> f -` T))" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 626 | using closedin_diff by fastforce | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 627 | have [simp]: "(f ` S - f ` (S - (S \<inter> f -` T))) = T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 628 | using T by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 629 | show ?rhs | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 630 | using ope [OF *, unfolded closedin_def] by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 631 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 632 | assume ?rhs | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 633 | with contf show ?lhs | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 634 | by (auto simp: continuous_on_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 635 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 636 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 637 | lemma continuous_right_inverse_imp_quotient_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 638 | assumes contf: "continuous_on S f" and imf: "f ` S \<subseteq> T" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 639 | and contg: "continuous_on T g" and img: "g ` T \<subseteq> S" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 640 | and fg [simp]: "\<And>y. y \<in> T \<Longrightarrow> f(g y) = y" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 641 | and U: "U \<subseteq> T" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 642 | shows "openin (top_of_set S) (S \<inter> f -` U) \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 643 | openin (top_of_set T) U" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 644 | (is "?lhs = ?rhs") | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 645 | proof - | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 646 | have f: "\<And>Z. openin (top_of_set (f ` S)) Z \<Longrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 647 | openin (top_of_set S) (S \<inter> f -` Z)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 648 | and g: "\<And>Z. openin (top_of_set (g ` T)) Z \<Longrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 649 | openin (top_of_set T) (T \<inter> g -` Z)" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 650 | using contf contg by (auto simp: continuous_on_open) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 651 | show ?thesis | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 652 | proof | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 653 |     have "T \<inter> g -` (g ` T \<inter> (S \<inter> f -` U)) = {x \<in> T. f (g x) \<in> U}"
 | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 654 | using imf img by blast | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 655 | also have "... = U" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 656 | using U by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 657 | finally have eq: "T \<inter> g -` (g ` T \<inter> (S \<inter> f -` U)) = U" . | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 658 | assume ?lhs | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 659 | then have *: "openin (top_of_set (g ` T)) (g ` T \<inter> (S \<inter> f -` U))" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 660 | by (meson img openin_Int openin_subtopology_Int_subset openin_subtopology_self) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 661 | show ?rhs | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 662 | using g [OF *] eq by auto | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 663 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 664 | assume rhs: ?rhs | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 665 | show ?lhs | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 666 | by (metis f fg image_eqI image_subset_iff imf img openin_subopen openin_subtopology_self openin_trans rhs) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 667 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 668 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 669 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 670 | lemma continuous_left_inverse_imp_quotient_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 671 | assumes "continuous_on S f" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 672 | and "continuous_on (f ` S) g" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 673 | and "\<And>x. x \<in> S \<Longrightarrow> g(f x) = x" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 674 | and "U \<subseteq> f ` S" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 675 | shows "openin (top_of_set S) (S \<inter> f -` U) \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 676 | openin (top_of_set (f ` S)) U" | 
| 76894 | 677 | using assms | 
| 678 | by (intro continuous_right_inverse_imp_quotient_map) auto | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 679 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 680 | lemma continuous_imp_quotient_map: | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 681 | fixes f :: "'a::t2_space \<Rightarrow> 'b::t2_space" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 682 | assumes "continuous_on S f" "f ` S = T" "compact S" "U \<subseteq> T" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 683 | shows "openin (top_of_set S) (S \<inter> f -` U) \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 684 | openin (top_of_set T) U" | 
| 76894 | 685 | by (simp add: assms closed_map_imp_quotient_map continuous_imp_closed_map) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 686 | |
| 70136 | 687 | subsection\<^marker>\<open>tag unimportant\<close>\<open>Pasting lemmas for functions, for of casewise definitions\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 688 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 689 | subsubsection\<open>on open sets\<close> | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 690 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 691 | lemma pasting_lemma: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 692 | assumes ope: "\<And>i. i \<in> I \<Longrightarrow> openin X (T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 693 | and cont: "\<And>i. i \<in> I \<Longrightarrow> continuous_map(subtopology X (T i)) Y (f i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 694 | and f: "\<And>i j x. \<lbrakk>i \<in> I; j \<in> I; x \<in> topspace X \<inter> T i \<inter> T j\<rbrakk> \<Longrightarrow> f i x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 695 | and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 696 | shows "continuous_map X Y g" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 697 | unfolding continuous_map_openin_preimage_eq | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 698 | proof (intro conjI allI impI) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 699 | show "g ` topspace X \<subseteq> topspace Y" | 
| 71174 | 700 | using g cont continuous_map_image_subset_topspace by fastforce | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 701 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 702 | fix U | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 703 | assume Y: "openin Y U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 704 | have T: "T i \<subseteq> topspace X" if "i \<in> I" for i | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 705 | using ope by (simp add: openin_subset that) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 706 | have *: "topspace X \<inter> g -` U = (\<Union>i \<in> I. T i \<inter> f i -` U)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 707 | using f g T by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 708 | have "\<And>i. i \<in> I \<Longrightarrow> openin X (T i \<inter> f i -` U)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 709 | using cont unfolding continuous_map_openin_preimage_eq | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 710 | by (metis Y T inf.commute inf_absorb1 ope topspace_subtopology openin_trans_full) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 711 | then show "openin X (topspace X \<inter> g -` U)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 712 | by (auto simp: *) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 713 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 714 | |
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 715 | lemma pasting_lemma_exists: | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 716 | assumes X: "topspace X \<subseteq> (\<Union>i \<in> I. T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 717 | and ope: "\<And>i. i \<in> I \<Longrightarrow> openin X (T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 718 | and cont: "\<And>i. i \<in> I \<Longrightarrow> continuous_map (subtopology X (T i)) Y (f i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 719 | and f: "\<And>i j x. \<lbrakk>i \<in> I; j \<in> I; x \<in> topspace X \<inter> T i \<inter> T j\<rbrakk> \<Longrightarrow> f i x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 720 | obtains g where "continuous_map X Y g" "\<And>x i. \<lbrakk>i \<in> I; x \<in> topspace X \<inter> T i\<rbrakk> \<Longrightarrow> g x = f i x" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 721 | proof | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 722 | let ?h = "\<lambda>x. f (SOME i. i \<in> I \<and> x \<in> T i) x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 723 | show "continuous_map X Y ?h" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 724 | apply (rule pasting_lemma [OF ope cont]) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 725 | apply (blast intro: f)+ | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 726 | by (metis (no_types, lifting) UN_E X subsetD someI_ex) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 727 | show "f (SOME i. i \<in> I \<and> x \<in> T i) x = f i x" if "i \<in> I" "x \<in> topspace X \<inter> T i" for i x | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 728 | by (metis (no_types, lifting) IntD2 IntI f someI_ex that) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 729 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 730 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 731 | lemma pasting_lemma_locally_finite: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 732 |   assumes fin: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>V. openin X V \<and> x \<in> V \<and> finite {i \<in> I. T i \<inter> V \<noteq> {}}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 733 | and clo: "\<And>i. i \<in> I \<Longrightarrow> closedin X (T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 734 | and cont: "\<And>i. i \<in> I \<Longrightarrow> continuous_map(subtopology X (T i)) Y (f i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 735 | and f: "\<And>i j x. \<lbrakk>i \<in> I; j \<in> I; x \<in> topspace X \<inter> T i \<inter> T j\<rbrakk> \<Longrightarrow> f i x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 736 | and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 737 | shows "continuous_map X Y g" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 738 | unfolding continuous_map_closedin_preimage_eq | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 739 | proof (intro conjI allI impI) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 740 | show "g ` topspace X \<subseteq> topspace Y" | 
| 71174 | 741 | using g cont continuous_map_image_subset_topspace by fastforce | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 742 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 743 | fix U | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 744 | assume Y: "closedin Y U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 745 | have T: "T i \<subseteq> topspace X" if "i \<in> I" for i | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 746 | using clo by (simp add: closedin_subset that) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 747 | have *: "topspace X \<inter> g -` U = (\<Union>i \<in> I. T i \<inter> f i -` U)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 748 | using f g T by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 749 | have cTf: "\<And>i. i \<in> I \<Longrightarrow> closedin X (T i \<inter> f i -` U)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 750 | using cont unfolding continuous_map_closedin_preimage_eq topspace_subtopology | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 751 | by (simp add: Int_absorb1 T Y clo closedin_closed_subtopology) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 752 |   have sub: "{Z \<in> (\<lambda>i. T i \<inter> f i -` U) ` I. Z \<inter> V \<noteq> {}}
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 753 |            \<subseteq> (\<lambda>i. T i \<inter> f i -` U) ` {i \<in> I. T i \<inter> V \<noteq> {}}" for V
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 754 | by auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 755 | have 1: "(\<Union>i\<in>I. T i \<inter> f i -` U) \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 756 | using T by blast | 
| 76894 | 757 | then have "locally_finite_in X ((\<lambda>i. T i \<inter> f i -` U) ` I)" | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 758 | unfolding locally_finite_in_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 759 | using finite_subset [OF sub] fin by force | 
| 76894 | 760 | then show "closedin X (topspace X \<inter> g -` U)" | 
| 761 | by (smt (verit, best) * cTf closedin_locally_finite_Union image_iff) | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 762 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 763 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 764 | subsubsection\<open>Likewise on closed sets, with a finiteness assumption\<close> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 765 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 766 | lemma pasting_lemma_closed: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 767 | assumes fin: "finite I" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 768 | and clo: "\<And>i. i \<in> I \<Longrightarrow> closedin X (T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 769 | and cont: "\<And>i. i \<in> I \<Longrightarrow> continuous_map(subtopology X (T i)) Y (f i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 770 | and f: "\<And>i j x. \<lbrakk>i \<in> I; j \<in> I; x \<in> topspace X \<inter> T i \<inter> T j\<rbrakk> \<Longrightarrow> f i x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 771 | and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 772 | shows "continuous_map X Y g" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 773 | using pasting_lemma_locally_finite [OF _ clo cont f g] fin by auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 774 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 775 | lemma pasting_lemma_exists_locally_finite: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 776 |   assumes fin: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>V. openin X V \<and> x \<in> V \<and> finite {i \<in> I. T i \<inter> V \<noteq> {}}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 777 | and X: "topspace X \<subseteq> \<Union>(T ` I)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 778 | and clo: "\<And>i. i \<in> I \<Longrightarrow> closedin X (T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 779 | and cont: "\<And>i. i \<in> I \<Longrightarrow> continuous_map(subtopology X (T i)) Y (f i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 780 | and f: "\<And>i j x. \<lbrakk>i \<in> I; j \<in> I; x \<in> topspace X \<inter> T i \<inter> T j\<rbrakk> \<Longrightarrow> f i x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 781 | and g: "\<And>x. x \<in> topspace X \<Longrightarrow> \<exists>j. j \<in> I \<and> x \<in> T j \<and> g x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 782 | obtains g where "continuous_map X Y g" "\<And>x i. \<lbrakk>i \<in> I; x \<in> topspace X \<inter> T i\<rbrakk> \<Longrightarrow> g x = f i x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 783 | proof | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 784 | show "continuous_map X Y (\<lambda>x. f(@i. i \<in> I \<and> x \<in> T i) x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 785 | apply (rule pasting_lemma_locally_finite [OF fin]) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 786 | apply (blast intro: assms)+ | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 787 | by (metis (no_types, lifting) UN_E X set_rev_mp someI_ex) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 788 | next | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 789 | fix x i | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 790 | assume "i \<in> I" and "x \<in> topspace X \<inter> T i" | 
| 76894 | 791 | then show "f (SOME i. i \<in> I \<and> x \<in> T i) x = f i x" | 
| 792 | by (metis (mono_tags, lifting) IntE IntI f someI2) | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 793 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 794 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 795 | lemma pasting_lemma_exists_closed: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 796 | assumes fin: "finite I" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 797 | and X: "topspace X \<subseteq> \<Union>(T ` I)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 798 | and clo: "\<And>i. i \<in> I \<Longrightarrow> closedin X (T i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 799 | and cont: "\<And>i. i \<in> I \<Longrightarrow> continuous_map(subtopology X (T i)) Y (f i)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 800 | and f: "\<And>i j x. \<lbrakk>i \<in> I; j \<in> I; x \<in> topspace X \<inter> T i \<inter> T j\<rbrakk> \<Longrightarrow> f i x = f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 801 | obtains g where "continuous_map X Y g" "\<And>x i. \<lbrakk>i \<in> I; x \<in> topspace X \<inter> T i\<rbrakk> \<Longrightarrow> g x = f i x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 802 | proof | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 803 | show "continuous_map X Y (\<lambda>x. f (SOME i. i \<in> I \<and> x \<in> T i) x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 804 | apply (rule pasting_lemma_closed [OF \<open>finite I\<close> clo cont]) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 805 | apply (blast intro: f)+ | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 806 | by (metis (mono_tags, lifting) UN_iff X someI_ex subset_iff) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 807 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 808 | fix x i | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 809 | assume "i \<in> I" "x \<in> topspace X \<inter> T i" | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 810 | then show "f (SOME i. i \<in> I \<and> x \<in> T i) x = f i x" | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 811 | by (metis (no_types, lifting) IntD2 IntI f someI_ex) | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 812 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 813 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 814 | lemma continuous_map_cases: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 815 |   assumes f: "continuous_map (subtopology X (X closure_of {x. P x})) Y f"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 816 |       and g: "continuous_map (subtopology X (X closure_of {x. \<not> P x})) Y g"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 817 |       and fg: "\<And>x. x \<in> X frontier_of {x. P x} \<Longrightarrow> f x = g x"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 818 | shows "continuous_map X Y (\<lambda>x. if P x then f x else g x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 819 | proof (rule pasting_lemma_closed) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 820 | let ?f = "\<lambda>b. if b then f else g" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 821 | let ?g = "\<lambda>x. if P x then f x else g x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 822 |   let ?T = "\<lambda>b. if b then X closure_of {x. P x} else X closure_of {x. ~P x}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 823 |   show "finite {True,False}" by auto
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 824 |   have eq: "topspace X - Collect P = topspace X \<inter> {x. \<not> P x}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 825 | by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 826 | show "?f i x = ?f j x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 827 |     if "i \<in> {True,False}" "j \<in> {True,False}" and x: "x \<in> topspace X \<inter> ?T i \<inter> ?T j" for i j x
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 828 | proof - | 
| 76894 | 829 | have "f x = g x" if "i" "\<not> j" | 
| 830 | by (smt (verit, best) Diff_Diff_Int closure_of_interior_of closure_of_restrict eq fg | |
| 831 | frontier_of_closures interior_of_complement that x) | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 832 | moreover | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 833 | have "g x = f x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 834 |       if "x \<in> X closure_of {x. \<not> P x}" "x \<in> X closure_of Collect P" "\<not> i" "j" for x
 | 
| 76894 | 835 | by (metis IntI closure_of_restrict eq fg frontier_of_closures that) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 836 | ultimately show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 837 | using that by (auto simp flip: closure_of_restrict) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 838 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 839 |   show "\<exists>j. j \<in> {True,False} \<and> x \<in> ?T j \<and> (if P x then f x else g x) = ?f j x"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 840 | if "x \<in> topspace X" for x | 
| 76894 | 841 | by simp (metis in_closure_of mem_Collect_eq that) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 842 | qed (auto simp: f g) | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 843 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 844 | lemma continuous_map_cases_alt: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 845 |   assumes f: "continuous_map (subtopology X (X closure_of {x \<in> topspace X. P x})) Y f"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 846 |       and g: "continuous_map (subtopology X (X closure_of {x \<in> topspace X. ~P x})) Y g"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 847 |       and fg: "\<And>x. x \<in> X frontier_of {x \<in> topspace X. P x} \<Longrightarrow> f x = g x"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 848 | shows "continuous_map X Y (\<lambda>x. if P x then f x else g x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 849 | apply (rule continuous_map_cases) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 850 | using assms | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 851 | apply (simp_all add: Collect_conj_eq closure_of_restrict [symmetric] frontier_of_restrict [symmetric]) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 852 | done | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 853 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 854 | lemma continuous_map_cases_function: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 855 | assumes contp: "continuous_map X Z p" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 856 |     and contf: "continuous_map (subtopology X {x \<in> topspace X. p x \<in> Z closure_of U}) Y f"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 857 |     and contg: "continuous_map (subtopology X {x \<in> topspace X. p x \<in> Z closure_of (topspace Z - U)}) Y g"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 858 | and fg: "\<And>x. \<lbrakk>x \<in> topspace X; p x \<in> Z frontier_of U\<rbrakk> \<Longrightarrow> f x = g x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 859 | shows "continuous_map X Y (\<lambda>x. if p x \<in> U then f x else g x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 860 | proof (rule continuous_map_cases_alt) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 861 |   show "continuous_map (subtopology X (X closure_of {x \<in> topspace X. p x \<in> U})) Y f"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 862 | proof (rule continuous_map_from_subtopology_mono) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 863 |     let ?T = "{x \<in> topspace X. p x \<in> Z closure_of U}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 864 | show "continuous_map (subtopology X ?T) Y f" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 865 | by (simp add: contf) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 866 |     show "X closure_of {x \<in> topspace X. p x \<in> U} \<subseteq> ?T"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 867 | by (rule continuous_map_closure_preimage_subset [OF contp]) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 868 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 869 |   show "continuous_map (subtopology X (X closure_of {x \<in> topspace X. p x \<notin> U})) Y g"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 870 | proof (rule continuous_map_from_subtopology_mono) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 871 |     let ?T = "{x \<in> topspace X. p x \<in> Z closure_of (topspace Z - U)}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 872 | show "continuous_map (subtopology X ?T) Y g" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 873 | by (simp add: contg) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 874 |     have "X closure_of {x \<in> topspace X. p x \<notin> U} \<subseteq> X closure_of {x \<in> topspace X. p x \<in> topspace Z - U}"
 | 
| 76894 | 875 | by (smt (verit, del_insts) DiffI mem_Collect_eq subset_iff closure_of_mono continuous_map_closedin contp) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 876 |     then show "X closure_of {x \<in> topspace X. p x \<notin> U} \<subseteq> ?T"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 877 | by (rule order_trans [OF _ continuous_map_closure_preimage_subset [OF contp]]) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 878 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 879 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 880 |   show "f x = g x" if "x \<in> X frontier_of {x \<in> topspace X. p x \<in> U}" for x
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 881 | using that continuous_map_frontier_frontier_preimage_subset [OF contp, of U] fg by blast | 
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 882 | qed | 
| 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 883 | |
| 69750 | 884 | subsection \<open>Retractions\<close> | 
| 885 | ||
| 70136 | 886 | definition\<^marker>\<open>tag important\<close> retraction :: "('a::topological_space) set \<Rightarrow> 'a set \<Rightarrow> ('a \<Rightarrow> 'a) \<Rightarrow> bool"
 | 
| 69750 | 887 | where "retraction S T r \<longleftrightarrow> | 
| 888 | T \<subseteq> S \<and> continuous_on S r \<and> r ` S \<subseteq> T \<and> (\<forall>x\<in>T. r x = x)" | |
| 889 | ||
| 70136 | 890 | definition\<^marker>\<open>tag important\<close> retract_of (infixl "retract'_of" 50) where | 
| 69750 | 891 | "T retract_of S \<longleftrightarrow> (\<exists>r. retraction S T r)" | 
| 892 | ||
| 893 | lemma retraction_idempotent: "retraction S T r \<Longrightarrow> x \<in> S \<Longrightarrow> r (r x) = r x" | |
| 894 | unfolding retraction_def by auto | |
| 895 | ||
| 896 | text \<open>Preservation of fixpoints under (more general notion of) retraction\<close> | |
| 897 | ||
| 898 | lemma invertible_fixpoint_property: | |
| 899 | fixes S :: "'a::topological_space set" | |
| 900 | and T :: "'b::topological_space set" | |
| 901 | assumes contt: "continuous_on T i" | |
| 902 | and "i ` T \<subseteq> S" | |
| 903 | and contr: "continuous_on S r" | |
| 904 | and "r ` S \<subseteq> T" | |
| 905 | and ri: "\<And>y. y \<in> T \<Longrightarrow> r (i y) = y" | |
| 906 | and FP: "\<And>f. \<lbrakk>continuous_on S f; f ` S \<subseteq> S\<rbrakk> \<Longrightarrow> \<exists>x\<in>S. f x = x" | |
| 907 | and contg: "continuous_on T g" | |
| 908 | and "g ` T \<subseteq> T" | |
| 909 | obtains y where "y \<in> T" and "g y = y" | |
| 910 | proof - | |
| 911 | have "\<exists>x\<in>S. (i \<circ> g \<circ> r) x = x" | |
| 912 | proof (rule FP) | |
| 913 | show "continuous_on S (i \<circ> g \<circ> r)" | |
| 914 | by (meson contt contr assms(4) contg assms(8) continuous_on_compose continuous_on_subset) | |
| 915 | show "(i \<circ> g \<circ> r) ` S \<subseteq> S" | |
| 916 | using assms(2,4,8) by force | |
| 917 | qed | |
| 918 | then obtain x where x: "x \<in> S" "(i \<circ> g \<circ> r) x = x" .. | |
| 919 | then have *: "g (r x) \<in> T" | |
| 920 | using assms(4,8) by auto | |
| 921 | have "r ((i \<circ> g \<circ> r) x) = r x" | |
| 922 | using x by auto | |
| 923 | then show ?thesis | |
| 924 | using "*" ri that by auto | |
| 925 | qed | |
| 926 | ||
| 927 | lemma homeomorphic_fixpoint_property: | |
| 928 | fixes S :: "'a::topological_space set" | |
| 929 | and T :: "'b::topological_space set" | |
| 930 | assumes "S homeomorphic T" | |
| 931 | shows "(\<forall>f. continuous_on S f \<and> f ` S \<subseteq> S \<longrightarrow> (\<exists>x\<in>S. f x = x)) \<longleftrightarrow> | |
| 932 | (\<forall>g. continuous_on T g \<and> g ` T \<subseteq> T \<longrightarrow> (\<exists>y\<in>T. g y = y))" | |
| 933 | (is "?lhs = ?rhs") | |
| 934 | proof - | |
| 935 | obtain r i where r: | |
| 936 | "\<forall>x\<in>S. i (r x) = x" "r ` S = T" "continuous_on S r" | |
| 937 | "\<forall>y\<in>T. r (i y) = y" "i ` T = S" "continuous_on T i" | |
| 938 | using assms unfolding homeomorphic_def homeomorphism_def by blast | |
| 939 | show ?thesis | |
| 940 | proof | |
| 941 | assume ?lhs | |
| 942 | with r show ?rhs | |
| 943 | by (metis invertible_fixpoint_property[of T i S r] order_refl) | |
| 944 | next | |
| 945 | assume ?rhs | |
| 946 | with r show ?lhs | |
| 947 | by (metis invertible_fixpoint_property[of S r T i] order_refl) | |
| 948 | qed | |
| 949 | qed | |
| 950 | ||
| 951 | lemma retract_fixpoint_property: | |
| 952 | fixes f :: "'a::topological_space \<Rightarrow> 'b::topological_space" | |
| 953 | and S :: "'a set" | |
| 954 | assumes "T retract_of S" | |
| 955 | and FP: "\<And>f. \<lbrakk>continuous_on S f; f ` S \<subseteq> S\<rbrakk> \<Longrightarrow> \<exists>x\<in>S. f x = x" | |
| 956 | and contg: "continuous_on T g" | |
| 957 | and "g ` T \<subseteq> T" | |
| 958 | obtains y where "y \<in> T" and "g y = y" | |
| 959 | proof - | |
| 960 | obtain h where "retraction S T h" | |
| 961 | using assms(1) unfolding retract_of_def .. | |
| 962 | then show ?thesis | |
| 963 | unfolding retraction_def | |
| 964 | using invertible_fixpoint_property[OF continuous_on_id _ _ _ _ FP] | |
| 965 | by (metis assms(4) contg image_ident that) | |
| 966 | qed | |
| 967 | ||
| 968 | lemma retraction: | |
| 969 | "retraction S T r \<longleftrightarrow> | |
| 970 | T \<subseteq> S \<and> continuous_on S r \<and> r ` S = T \<and> (\<forall>x \<in> T. r x = x)" | |
| 971 | by (force simp: retraction_def) | |
| 972 | ||
| 69753 | 973 | lemma retractionE: \<comment> \<open>yields properties normalized wrt. simp -- less likely to loop\<close> | 
| 69750 | 974 | assumes "retraction S T r" | 
| 975 | obtains "T = r ` S" "r ` S \<subseteq> S" "continuous_on S r" "\<And>x. x \<in> S \<Longrightarrow> r (r x) = r x" | |
| 976 | proof (rule that) | |
| 977 | from retraction [of S T r] assms | |
| 978 | have "T \<subseteq> S" "continuous_on S r" "r ` S = T" and "\<forall>x \<in> T. r x = x" | |
| 979 | by simp_all | |
| 980 | then show "T = r ` S" "r ` S \<subseteq> S" "continuous_on S r" | |
| 981 | by simp_all | |
| 982 | from \<open>\<forall>x \<in> T. r x = x\<close> have "r x = x" if "x \<in> T" for x | |
| 983 | using that by simp | |
| 984 | with \<open>r ` S = T\<close> show "r (r x) = r x" if "x \<in> S" for x | |
| 985 | using that by auto | |
| 986 | qed | |
| 987 | ||
| 69753 | 988 | lemma retract_ofE: \<comment> \<open>yields properties normalized wrt. simp -- less likely to loop\<close> | 
| 69750 | 989 | assumes "T retract_of S" | 
| 990 | obtains r where "T = r ` S" "r ` S \<subseteq> S" "continuous_on S r" "\<And>x. x \<in> S \<Longrightarrow> r (r x) = r x" | |
| 991 | proof - | |
| 992 | from assms obtain r where "retraction S T r" | |
| 993 | by (auto simp add: retract_of_def) | |
| 994 | with that show thesis | |
| 995 | by (auto elim: retractionE) | |
| 996 | qed | |
| 997 | ||
| 998 | lemma retract_of_imp_extensible: | |
| 999 | assumes "S retract_of T" and "continuous_on S f" and "f ` S \<subseteq> U" | |
| 1000 | obtains g where "continuous_on T g" "g ` T \<subseteq> U" "\<And>x. x \<in> S \<Longrightarrow> g x = f x" | |
| 1001 | proof - | |
| 1002 | from \<open>S retract_of T\<close> obtain r where "retraction T S r" | |
| 1003 | by (auto simp add: retract_of_def) | |
| 1004 | show thesis | |
| 1005 | by (rule that [of "f \<circ> r"]) | |
| 1006 | (use \<open>continuous_on S f\<close> \<open>f ` S \<subseteq> U\<close> \<open>retraction T S r\<close> in \<open>auto simp: continuous_on_compose2 retraction\<close>) | |
| 1007 | qed | |
| 1008 | ||
| 1009 | lemma idempotent_imp_retraction: | |
| 1010 | assumes "continuous_on S f" and "f ` S \<subseteq> S" and "\<And>x. x \<in> S \<Longrightarrow> f(f x) = f x" | |
| 1011 | shows "retraction S (f ` S) f" | |
| 1012 | by (simp add: assms retraction) | |
| 1013 | ||
| 1014 | lemma retraction_subset: | |
| 1015 | assumes "retraction S T r" and "T \<subseteq> s'" and "s' \<subseteq> S" | |
| 1016 | shows "retraction s' T r" | |
| 1017 | unfolding retraction_def | |
| 1018 | by (metis assms continuous_on_subset image_mono retraction) | |
| 1019 | ||
| 1020 | lemma retract_of_subset: | |
| 1021 | assumes "T retract_of S" and "T \<subseteq> s'" and "s' \<subseteq> S" | |
| 1022 | shows "T retract_of s'" | |
| 1023 | by (meson assms retract_of_def retraction_subset) | |
| 1024 | ||
| 1025 | lemma retraction_refl [simp]: "retraction S S (\<lambda>x. x)" | |
| 1026 | by (simp add: retraction) | |
| 1027 | ||
| 1028 | lemma retract_of_refl [iff]: "S retract_of S" | |
| 1029 | unfolding retract_of_def retraction_def | |
| 1030 | using continuous_on_id by blast | |
| 1031 | ||
| 1032 | lemma retract_of_imp_subset: | |
| 1033 | "S retract_of T \<Longrightarrow> S \<subseteq> T" | |
| 1034 | by (simp add: retract_of_def retraction_def) | |
| 1035 | ||
| 1036 | lemma retract_of_empty [simp]: | |
| 1037 |      "({} retract_of S) \<longleftrightarrow> S = {}"  "(S retract_of {}) \<longleftrightarrow> S = {}"
 | |
| 1038 | by (auto simp: retract_of_def retraction_def) | |
| 1039 | ||
| 1040 | lemma retract_of_singleton [iff]: "({x} retract_of S) \<longleftrightarrow> x \<in> S"
 | |
| 1041 | unfolding retract_of_def retraction_def by force | |
| 1042 | ||
| 1043 | lemma retraction_comp: | |
| 76894 | 1044 | "\<lbrakk>retraction S T f; retraction T U g\<rbrakk> \<Longrightarrow> retraction S U (g \<circ> f)" | 
| 1045 | by (smt (verit, best) comp_apply continuous_on_compose image_comp retraction subset_iff) | |
| 69750 | 1046 | |
| 1047 | lemma retract_of_trans [trans]: | |
| 1048 | assumes "S retract_of T" and "T retract_of U" | |
| 1049 | shows "S retract_of U" | |
| 1050 | using assms by (auto simp: retract_of_def intro: retraction_comp) | |
| 1051 | ||
| 1052 | lemma closedin_retract: | |
| 1053 | fixes S :: "'a :: t2_space set" | |
| 1054 | assumes "S retract_of T" | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1055 | shows "closedin (top_of_set T) S" | 
| 69750 | 1056 | proof - | 
| 1057 | obtain r where r: "S \<subseteq> T" "continuous_on T r" "r ` T \<subseteq> S" "\<And>x. x \<in> S \<Longrightarrow> r x = x" | |
| 1058 | using assms by (auto simp: retract_of_def retraction_def) | |
| 1059 |   have "S = {x\<in>T. x = r x}"
 | |
| 1060 | using r by auto | |
| 1061 |   also have "\<dots> = T \<inter> ((\<lambda>x. (x, r x)) -` ({y. \<exists>x. y = (x, x)}))"
 | |
| 1062 | unfolding vimage_def mem_Times_iff fst_conv snd_conv | |
| 1063 | using r | |
| 1064 | by auto | |
| 1065 | also have "closedin (top_of_set T) \<dots>" | |
| 1066 | by (rule continuous_closedin_preimage) (auto intro!: closed_diagonal continuous_on_Pair r) | |
| 1067 | finally show ?thesis . | |
| 1068 | qed | |
| 1069 | ||
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1070 | lemma closedin_self [simp]: "closedin (top_of_set S) S" | 
| 69750 | 1071 | by simp | 
| 1072 | ||
| 1073 | lemma retract_of_closed: | |
| 1074 | fixes S :: "'a :: t2_space set" | |
| 1075 | shows "\<lbrakk>closed T; S retract_of T\<rbrakk> \<Longrightarrow> closed S" | |
| 1076 | by (metis closedin_retract closedin_closed_eq) | |
| 1077 | ||
| 1078 | lemma retract_of_compact: | |
| 1079 | "\<lbrakk>compact T; S retract_of T\<rbrakk> \<Longrightarrow> compact S" | |
| 1080 | by (metis compact_continuous_image retract_of_def retraction) | |
| 1081 | ||
| 1082 | lemma retract_of_connected: | |
| 1083 | "\<lbrakk>connected T; S retract_of T\<rbrakk> \<Longrightarrow> connected S" | |
| 1084 | by (metis Topological_Spaces.connected_continuous_image retract_of_def retraction) | |
| 1085 | ||
| 70178 
4900351361b0
Lindelöf spaces and supporting material
 paulson <lp15@cam.ac.uk> parents: 
70136diff
changeset | 1086 | lemma retraction_openin_vimage_iff: | 
| 76894 | 1087 | assumes r: "retraction S T r" and "U \<subseteq> T" | 
| 1088 | shows "openin (top_of_set S) (S \<inter> r -` U) \<longleftrightarrow> openin (top_of_set T) U" (is "?lhs = ?rhs") | |
| 1089 | proof | |
| 1090 | show "?lhs \<Longrightarrow> ?rhs" | |
| 1091 | using r retraction_def retractionE | |
| 1092 | by (smt (verit, best) continuous_right_inverse_imp_quotient_map retraction_subset \<open>U \<subseteq> T\<close>) | |
| 1093 | show "?rhs \<Longrightarrow> ?lhs" | |
| 1094 | by (meson continuous_openin_preimage r retraction_def) | |
| 1095 | qed | |
| 69750 | 1096 | |
| 1097 | lemma retract_of_Times: | |
| 1098 | "\<lbrakk>S retract_of s'; T retract_of t'\<rbrakk> \<Longrightarrow> (S \<times> T) retract_of (s' \<times> t')" | |
| 1099 | apply (simp add: retract_of_def retraction_def Sigma_mono, clarify) | |
| 1100 | apply (rename_tac f g) | |
| 1101 | apply (rule_tac x="\<lambda>z. ((f \<circ> fst) z, (g \<circ> snd) z)" in exI) | |
| 1102 | apply (rule conjI continuous_intros | erule continuous_on_subset | force)+ | |
| 1103 | done | |
| 1104 | ||
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1105 | subsection\<open>Retractions on a topological space\<close> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1106 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1107 | definition retract_of_space :: "'a set \<Rightarrow> 'a topology \<Rightarrow> bool" (infix "retract'_of'_space" 50) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1108 | where "S retract_of_space X | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1109 | \<equiv> S \<subseteq> topspace X \<and> (\<exists>r. continuous_map X (subtopology X S) r \<and> (\<forall>x \<in> S. r x = x))" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1110 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1111 | lemma retract_of_space_retraction_maps: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1112 | "S retract_of_space X \<longleftrightarrow> S \<subseteq> topspace X \<and> (\<exists>r. retraction_maps X (subtopology X S) r id)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1113 | by (auto simp: retract_of_space_def retraction_maps_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1114 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1115 | lemma retract_of_space_section_map: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1116 | "S retract_of_space X \<longleftrightarrow> S \<subseteq> topspace X \<and> section_map (subtopology X S) X id" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1117 | unfolding retract_of_space_def retraction_maps_def section_map_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1118 | by (auto simp: continuous_map_from_subtopology) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1119 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1120 | lemma retract_of_space_imp_subset: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1121 | "S retract_of_space X \<Longrightarrow> S \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1122 | by (simp add: retract_of_space_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1123 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1124 | lemma retract_of_space_topspace: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1125 | "topspace X retract_of_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1126 | using retract_of_space_def by force | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1127 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1128 | lemma retract_of_space_empty [simp]: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1129 |    "{} retract_of_space X \<longleftrightarrow> topspace X = {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1130 | by (auto simp: continuous_map_def retract_of_space_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1131 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1132 | lemma retract_of_space_singleton [simp]: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1133 |   "{a} retract_of_space X \<longleftrightarrow> a \<in> topspace X"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1134 | proof - | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1135 |   have "continuous_map X (subtopology X {a}) (\<lambda>x. a) \<and> (\<lambda>x. a) a = a" if "a \<in> topspace X"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1136 | using that by simp | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1137 | then show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1138 | by (force simp: retract_of_space_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1139 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1140 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1141 | lemma retract_of_space_clopen: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1142 |   assumes "openin X S" "closedin X S" "S = {} \<Longrightarrow> topspace X = {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1143 | shows "S retract_of_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1144 | proof (cases "S = {}")
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1145 | case False | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1146 | then obtain a where "a \<in> S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1147 | by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1148 | show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1149 | unfolding retract_of_space_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1150 | proof (intro exI conjI) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1151 | show "S \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1152 | by (simp add: assms closedin_subset) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1153 | have "continuous_map X X (\<lambda>x. if x \<in> S then x else a)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1154 | proof (rule continuous_map_cases) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1155 |       show "continuous_map (subtopology X (X closure_of {x. x \<in> S})) X (\<lambda>x. x)"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1156 | by (simp add: continuous_map_from_subtopology) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1157 |       show "continuous_map (subtopology X (X closure_of {x. x \<notin> S})) X (\<lambda>x. a)"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1158 | using \<open>S \<subseteq> topspace X\<close> \<open>a \<in> S\<close> by force | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1159 |       show "x = a" if "x \<in> X frontier_of {x. x \<in> S}" for x
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1160 | using assms that clopenin_eq_frontier_of by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1161 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1162 | then show "continuous_map X (subtopology X S) (\<lambda>x. if x \<in> S then x else a)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1163 | using \<open>S \<subseteq> topspace X\<close> \<open>a \<in> S\<close> by (auto simp: continuous_map_in_subtopology) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1164 | qed auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1165 | qed (use assms in auto) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1166 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1167 | lemma retract_of_space_disjoint_union: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1168 |   assumes "openin X S" "openin X T" and ST: "disjnt S T" "S \<union> T = topspace X" and "S = {} \<Longrightarrow> topspace X = {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1169 | shows "S retract_of_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1170 | proof (rule retract_of_space_clopen) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1171 |   have "S \<inter> T = {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1172 | by (meson ST disjnt_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1173 | then have "S = topspace X - T" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1174 | using ST by auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1175 | then show "closedin X S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1176 | using \<open>openin X T\<close> by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1177 | qed (auto simp: assms) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1178 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1179 | lemma retraction_maps_section_image1: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1180 | assumes "retraction_maps X Y r s" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1181 | shows "s ` (topspace Y) retract_of_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1182 | unfolding retract_of_space_section_map | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1183 | proof | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1184 | show "s ` topspace Y \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1185 | using assms continuous_map_image_subset_topspace retraction_maps_def by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1186 | show "section_map (subtopology X (s ` topspace Y)) X id" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1187 | unfolding section_map_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1188 | using assms retraction_maps_to_retract_maps by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1189 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1190 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1191 | lemma retraction_maps_section_image2: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1192 | "retraction_maps X Y r s | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1193 | \<Longrightarrow> subtopology X (s ` (topspace Y)) homeomorphic_space Y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1194 | using embedding_map_imp_homeomorphic_space homeomorphic_space_sym section_imp_embedding_map | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1195 | section_map_def by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1196 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1197 | subsection\<open>Paths and path-connectedness\<close> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1198 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1199 | definition pathin :: "'a topology \<Rightarrow> (real \<Rightarrow> 'a) \<Rightarrow> bool" where | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1200 |    "pathin X g \<equiv> continuous_map (subtopology euclideanreal {0..1}) X g"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1201 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1202 | lemma pathin_compose: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1203 | "\<lbrakk>pathin X g; continuous_map X Y f\<rbrakk> \<Longrightarrow> pathin Y (f \<circ> g)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1204 | by (simp add: continuous_map_compose pathin_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1205 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1206 | lemma pathin_subtopology: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1207 |      "pathin (subtopology X S) g \<longleftrightarrow> pathin X g \<and> (\<forall>x \<in> {0..1}. g x \<in> S)"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1208 | by (auto simp: pathin_def continuous_map_in_subtopology) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1209 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1210 | lemma pathin_const: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1211 | "pathin X (\<lambda>x. a) \<longleftrightarrow> a \<in> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1212 | by (simp add: pathin_def) | 
| 69939 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1213 | |
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1214 | lemma path_start_in_topspace: "pathin X g \<Longrightarrow> g 0 \<in> topspace X" | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1215 | by (force simp: pathin_def continuous_map) | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1216 | |
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1217 | lemma path_finish_in_topspace: "pathin X g \<Longrightarrow> g 1 \<in> topspace X" | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1218 | by (force simp: pathin_def continuous_map) | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1219 | |
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1220 | lemma path_image_subset_topspace: "pathin X g \<Longrightarrow> g ` ({0..1}) \<subseteq> topspace X"
 | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1221 | by (force simp: pathin_def continuous_map) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1222 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1223 | definition path_connected_space :: "'a topology \<Rightarrow> bool" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1224 | where "path_connected_space X \<equiv> \<forall>x \<in> topspace X. \<forall> y \<in> topspace X. \<exists>g. pathin X g \<and> g 0 = x \<and> g 1 = y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1225 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1226 | definition path_connectedin :: "'a topology \<Rightarrow> 'a set \<Rightarrow> bool" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1227 | where "path_connectedin X S \<equiv> S \<subseteq> topspace X \<and> path_connected_space(subtopology X S)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1228 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1229 | lemma path_connectedin_absolute [simp]: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1230 | "path_connectedin (subtopology X S) S \<longleftrightarrow> path_connectedin X S" | 
| 71172 | 1231 | by (simp add: path_connectedin_def subtopology_subtopology) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1232 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1233 | lemma path_connectedin_subset_topspace: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1234 | "path_connectedin X S \<Longrightarrow> S \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1235 | by (simp add: path_connectedin_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1236 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1237 | lemma path_connectedin_subtopology: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1238 | "path_connectedin (subtopology X S) T \<longleftrightarrow> path_connectedin X T \<and> T \<subseteq> S" | 
| 71172 | 1239 | by (auto simp: path_connectedin_def subtopology_subtopology inf.absorb2) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1240 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1241 | lemma path_connectedin: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1242 | "path_connectedin X S \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1243 | S \<subseteq> topspace X \<and> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1244 |         (\<forall>x \<in> S. \<forall>y \<in> S. \<exists>g. pathin X g \<and> g ` {0..1} \<subseteq> S \<and> g 0 = x \<and> g 1 = y)"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1245 | unfolding path_connectedin_def path_connected_space_def pathin_def continuous_map_in_subtopology | 
| 71172 | 1246 | by (intro conj_cong refl ball_cong) (simp_all add: inf.absorb_iff2) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1247 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1248 | lemma path_connectedin_topspace: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1249 | "path_connectedin X (topspace X) \<longleftrightarrow> path_connected_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1250 | by (simp add: path_connectedin_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1251 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1252 | lemma path_connected_imp_connected_space: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1253 | assumes "path_connected_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1254 | shows "connected_space X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1255 | proof - | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1256 | have *: "\<exists>S. connectedin X S \<and> g 0 \<in> S \<and> g 1 \<in> S" if "pathin X g" for g | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1257 | proof (intro exI conjI) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1258 |     have "continuous_map (subtopology euclideanreal {0..1}) X g"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1259 | using connectedin_absolute that by (simp add: pathin_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1260 |     then show "connectedin X (g ` {0..1})"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1261 | by (rule connectedin_continuous_map_image) auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1262 | qed auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1263 | show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1264 | using assms | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1265 | by (auto intro: * simp add: path_connected_space_def connected_space_subconnected Ball_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1266 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1267 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1268 | lemma path_connectedin_imp_connectedin: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1269 | "path_connectedin X S \<Longrightarrow> connectedin X S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1270 | by (simp add: connectedin_def path_connected_imp_connected_space path_connectedin_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1271 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1272 | lemma path_connected_space_topspace_empty: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1273 |      "topspace X = {} \<Longrightarrow> path_connected_space X"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1274 | by (simp add: path_connected_space_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1275 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1276 | lemma path_connectedin_empty [simp]: "path_connectedin X {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1277 | by (simp add: path_connectedin) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1278 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1279 | lemma path_connectedin_singleton [simp]: "path_connectedin X {a} \<longleftrightarrow> a \<in> topspace X"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1280 | proof | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1281 |   show "path_connectedin X {a} \<Longrightarrow> a \<in> topspace X"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1282 | by (simp add: path_connectedin) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1283 |   show "a \<in> topspace X \<Longrightarrow> path_connectedin X {a}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1284 | unfolding path_connectedin | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1285 | using pathin_const by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1286 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1287 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1288 | lemma path_connectedin_continuous_map_image: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1289 | assumes f: "continuous_map X Y f" and S: "path_connectedin X S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1290 | shows "path_connectedin Y (f ` S)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1291 | proof - | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1292 | have fX: "f ` (topspace X) \<subseteq> topspace Y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1293 | by (metis f continuous_map_image_subset_topspace) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1294 | show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1295 | unfolding path_connectedin | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1296 | proof (intro conjI ballI; clarify?) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1297 | fix x | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1298 | assume "x \<in> S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1299 | show "f x \<in> topspace Y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1300 | by (meson S fX \<open>x \<in> S\<close> image_subset_iff path_connectedin_subset_topspace set_mp) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1301 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1302 | fix x y | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1303 | assume "x \<in> S" and "y \<in> S" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1304 |     then obtain g where g: "pathin X g" "g ` {0..1} \<subseteq> S" "g 0 = x" "g 1 = y"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1305 | using S by (force simp: path_connectedin) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1306 |     show "\<exists>g. pathin Y g \<and> g ` {0..1} \<subseteq> f ` S \<and> g 0 = f x \<and> g 1 = f y"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1307 | proof (intro exI conjI) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1308 | show "pathin Y (f \<circ> g)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1309 | using \<open>pathin X g\<close> f pathin_compose by auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1310 | qed (use g in auto) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1311 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1312 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1313 | |
| 69939 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1314 | lemma path_connectedin_discrete_topology: | 
| 76894 | 1315 |   "path_connectedin (discrete_topology U) S \<longleftrightarrow> S \<subseteq> U \<and> (\<exists>a. S \<subseteq> {a})" (is "?lhs = ?rhs")
 | 
| 1316 | proof | |
| 1317 | show "?lhs \<Longrightarrow> ?rhs" | |
| 1318 | by (meson connectedin_discrete_topology path_connectedin_imp_connectedin) | |
| 1319 | show "?rhs \<Longrightarrow> ?lhs" | |
| 1320 | using subset_singletonD by fastforce | |
| 1321 | qed | |
| 69939 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1322 | |
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1323 | lemma path_connected_space_discrete_topology: | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1324 |    "path_connected_space (discrete_topology U) \<longleftrightarrow> (\<exists>a. U \<subseteq> {a})"
 | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1325 | by (metis path_connectedin_discrete_topology path_connectedin_topspace path_connected_space_topspace_empty | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1326 | subset_singletonD topspace_discrete_topology) | 
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1327 | |
| 
812ce526da33
new material on topology: products, etc. Some renamings, esp continuous_on_topo -> continuous_map
 paulson <lp15@cam.ac.uk> parents: 
69922diff
changeset | 1328 | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1329 | lemma homeomorphic_path_connected_space_imp: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1330 | "\<lbrakk>path_connected_space X; X homeomorphic_space Y\<rbrakk> \<Longrightarrow> path_connected_space Y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1331 | unfolding homeomorphic_space_def homeomorphic_maps_def | 
| 73932 
fd21b4a93043
added opaque_combs and renamed hide_lams to opaque_lifting
 desharna parents: 
72225diff
changeset | 1332 | by (metis (no_types, opaque_lifting) continuous_map_closedin continuous_map_image_subset_topspace imageI order_class.order.antisym path_connectedin_continuous_map_image path_connectedin_topspace subsetI) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1333 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1334 | lemma homeomorphic_path_connected_space: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1335 | "X homeomorphic_space Y \<Longrightarrow> path_connected_space X \<longleftrightarrow> path_connected_space Y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1336 | by (meson homeomorphic_path_connected_space_imp homeomorphic_space_sym) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1337 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1338 | lemma homeomorphic_map_path_connectedness: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1339 | assumes "homeomorphic_map X Y f" "U \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1340 | shows "path_connectedin Y (f ` U) \<longleftrightarrow> path_connectedin X U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1341 | unfolding path_connectedin_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1342 | proof (intro conj_cong homeomorphic_path_connected_space) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1343 | show "(f ` U \<subseteq> topspace Y) = (U \<subseteq> topspace X)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1344 | using assms homeomorphic_imp_surjective_map by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1345 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1346 | assume "U \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1347 | show "subtopology Y (f ` U) homeomorphic_space subtopology X U" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1348 | using assms unfolding homeomorphic_eq_everything_map | 
| 73932 
fd21b4a93043
added opaque_combs and renamed hide_lams to opaque_lifting
 desharna parents: 
72225diff
changeset | 1349 | by (metis (no_types, opaque_lifting) assms homeomorphic_map_subtopologies homeomorphic_space homeomorphic_space_sym image_mono inf.absorb_iff2) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1350 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1351 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1352 | lemma homeomorphic_map_path_connectedness_eq: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1353 | "homeomorphic_map X Y f \<Longrightarrow> path_connectedin X U \<longleftrightarrow> U \<subseteq> topspace X \<and> path_connectedin Y (f ` U)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1354 | by (meson homeomorphic_map_path_connectedness path_connectedin_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1355 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1356 | subsection\<open>Connected components\<close> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1357 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1358 | definition connected_component_of :: "'a topology \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> bool" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1359 | where "connected_component_of X x y \<equiv> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1360 | \<exists>T. connectedin X T \<and> x \<in> T \<and> y \<in> T" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1361 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1362 | abbreviation connected_component_of_set | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1363 | where "connected_component_of_set X x \<equiv> Collect (connected_component_of X x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1364 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1365 | definition connected_components_of :: "'a topology \<Rightarrow> ('a set) set"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1366 | where "connected_components_of X \<equiv> connected_component_of_set X ` topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1367 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1368 | lemma connected_component_in_topspace: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1369 | "connected_component_of X x y \<Longrightarrow> x \<in> topspace X \<and> y \<in> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1370 | by (meson connected_component_of_def connectedin_subset_topspace in_mono) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1371 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1372 | lemma connected_component_of_refl: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1373 | "connected_component_of X x x \<longleftrightarrow> x \<in> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1374 | by (meson connected_component_in_topspace connected_component_of_def connectedin_sing insertI1) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1375 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1376 | lemma connected_component_of_sym: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1377 | "connected_component_of X x y \<longleftrightarrow> connected_component_of X y x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1378 | by (meson connected_component_of_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1379 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1380 | lemma connected_component_of_trans: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1381 | "\<lbrakk>connected_component_of X x y; connected_component_of X y z\<rbrakk> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1382 | \<Longrightarrow> connected_component_of X x z" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1383 | unfolding connected_component_of_def | 
| 71842 
db120661dded
new HOL simproc: eliminate_false_implies
 Manuel Eberl <eberlm@in.tum.de> parents: 
71174diff
changeset | 1384 | using connectedin_Un by blast | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1385 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1386 | lemma connected_component_of_mono: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1387 | "\<lbrakk>connected_component_of (subtopology X S) x y; S \<subseteq> T\<rbrakk> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1388 | \<Longrightarrow> connected_component_of (subtopology X T) x y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1389 | by (metis connected_component_of_def connectedin_subtopology inf.absorb_iff2 subtopology_subtopology) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1390 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1391 | lemma connected_component_of_set: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1392 |    "connected_component_of_set X x = {y. \<exists>T. connectedin X T \<and> x \<in> T \<and> y \<in> T}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1393 | by (meson connected_component_of_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1394 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1395 | lemma connected_component_of_subset_topspace: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1396 | "connected_component_of_set X x \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1397 | using connected_component_in_topspace by force | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1398 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1399 | lemma connected_component_of_eq_empty: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1400 |    "connected_component_of_set X x = {} \<longleftrightarrow> (x \<notin> topspace X)"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1401 | using connected_component_in_topspace connected_component_of_refl by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1402 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1403 | lemma connected_space_iff_connected_component: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1404 | "connected_space X \<longleftrightarrow> (\<forall>x \<in> topspace X. \<forall>y \<in> topspace X. connected_component_of X x y)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1405 | by (simp add: connected_component_of_def connected_space_subconnected) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1406 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1407 | lemma connected_space_imp_connected_component_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1408 | "\<lbrakk>connected_space X; a \<in> topspace X; b \<in> topspace X\<rbrakk> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1409 | \<Longrightarrow> connected_component_of X a b" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1410 | by (simp add: connected_space_iff_connected_component) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1411 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1412 | lemma connected_space_connected_component_set: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1413 | "connected_space X \<longleftrightarrow> (\<forall>x \<in> topspace X. connected_component_of_set X x = topspace X)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1414 | using connected_component_of_subset_topspace connected_space_iff_connected_component by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1415 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1416 | lemma connected_component_of_maximal: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1417 | "\<lbrakk>connectedin X S; x \<in> S\<rbrakk> \<Longrightarrow> S \<subseteq> connected_component_of_set X x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1418 | by (meson Ball_Collect connected_component_of_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1419 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1420 | lemma connected_component_of_equiv: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1421 | "connected_component_of X x y \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1422 | x \<in> topspace X \<and> y \<in> topspace X \<and> connected_component_of X x = connected_component_of X y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1423 | apply (simp add: connected_component_in_topspace fun_eq_iff) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1424 | by (meson connected_component_of_refl connected_component_of_sym connected_component_of_trans) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1425 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1426 | lemma connected_component_of_disjoint: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1427 | "disjnt (connected_component_of_set X x) (connected_component_of_set X y) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1428 | \<longleftrightarrow> ~(connected_component_of X x y)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1429 | using connected_component_of_equiv unfolding disjnt_iff by force | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1430 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1431 | lemma connected_component_of_eq: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1432 | "connected_component_of X x = connected_component_of X y \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1433 | (x \<notin> topspace X) \<and> (y \<notin> topspace X) \<or> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1434 | x \<in> topspace X \<and> y \<in> topspace X \<and> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1435 | connected_component_of X x y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1436 | by (metis Collect_empty_eq_bot connected_component_of_eq_empty connected_component_of_equiv) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1437 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1438 | lemma connectedin_connected_component_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1439 | "connectedin X (connected_component_of_set X x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1440 | proof - | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1441 |   have "connected_component_of_set X x = \<Union> {T. connectedin X T \<and> x \<in> T}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1442 | by (auto simp: connected_component_of_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1443 | then show ?thesis | 
| 76894 | 1444 | by (metis (no_types, lifting) InterI connectedin_Union emptyE mem_Collect_eq) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1445 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1446 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1447 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1448 | lemma Union_connected_components_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1449 | "\<Union>(connected_components_of X) = topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1450 | unfolding connected_components_of_def | 
| 76894 | 1451 | using connected_component_in_topspace connected_component_of_refl by fastforce | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1452 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1453 | lemma connected_components_of_maximal: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1454 | "\<lbrakk>C \<in> connected_components_of X; connectedin X S; ~disjnt C S\<rbrakk> \<Longrightarrow> S \<subseteq> C" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1455 | unfolding connected_components_of_def disjnt_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1456 | apply clarify | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1457 | by (metis Int_emptyI connected_component_of_def connected_component_of_trans mem_Collect_eq) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1458 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1459 | lemma pairwise_disjoint_connected_components_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1460 | "pairwise disjnt (connected_components_of X)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1461 | unfolding connected_components_of_def pairwise_def | 
| 76894 | 1462 | by (smt (verit, best) connected_component_of_disjoint connected_component_of_eq imageE) | 
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1463 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1464 | lemma complement_connected_components_of_Union: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1465 | "C \<in> connected_components_of X | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1466 |       \<Longrightarrow> topspace X - C = \<Union> (connected_components_of X - {C})"
 | 
| 76894 | 1467 | by (metis Union_connected_components_of bot.extremum ccpo_Sup_singleton diff_Union_pairwise_disjoint | 
| 1468 | insert_subset pairwise_disjoint_connected_components_of) | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1469 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1470 | lemma nonempty_connected_components_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1471 |    "C \<in> connected_components_of X \<Longrightarrow> C \<noteq> {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1472 | unfolding connected_components_of_def | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1473 | by (metis (no_types, lifting) connected_component_of_eq_empty imageE) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1474 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1475 | lemma connected_components_of_subset: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1476 | "C \<in> connected_components_of X \<Longrightarrow> C \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1477 | using Union_connected_components_of by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1478 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1479 | lemma connectedin_connected_components_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1480 | assumes "C \<in> connected_components_of X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1481 | shows "connectedin X C" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1482 | proof - | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1483 | have "C \<in> connected_component_of_set X ` topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1484 | using assms connected_components_of_def by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1485 | then show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1486 | using connectedin_connected_component_of by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1487 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1488 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1489 | lemma connected_component_in_connected_components_of: | 
| 76894 | 1490 | "connected_component_of_set X a \<in> connected_components_of X \<longleftrightarrow> a \<in> topspace X" | 
| 1491 | by (metis (no_types, lifting) connected_component_of_eq_empty connected_components_of_def image_iff) | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1492 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1493 | lemma connected_space_iff_components_eq: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1494 | "connected_space X \<longleftrightarrow> (\<forall>C \<in> connected_components_of X. \<forall>C' \<in> connected_components_of X. C = C')" | 
| 76894 | 1495 | (is "?lhs = ?rhs") | 
| 1496 | proof | |
| 1497 | show "?lhs \<Longrightarrow> ?rhs" | |
| 1498 | by (simp add: connected_components_of_def connected_space_connected_component_set) | |
| 1499 | show "?rhs \<Longrightarrow> ?lhs" | |
| 1500 | by (metis Union_connected_components_of Union_iff connected_space_subconnected connectedin_connected_components_of) | |
| 1501 | qed | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1502 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1503 | lemma connected_components_of_eq_empty: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1504 |    "connected_components_of X = {} \<longleftrightarrow> topspace X = {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1505 | by (simp add: connected_components_of_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1506 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1507 | lemma connected_components_of_empty_space: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1508 |    "topspace X = {} \<Longrightarrow> connected_components_of X = {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1509 | by (simp add: connected_components_of_eq_empty) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1510 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1511 | lemma connected_components_of_subset_sing: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1512 |    "connected_components_of X \<subseteq> {S} \<longleftrightarrow> connected_space X \<and> (topspace X = {} \<or> topspace X = S)"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1513 | proof (cases "topspace X = {}")
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1514 | case True | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1515 | then show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1516 | by (simp add: connected_components_of_empty_space connected_space_topspace_empty) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1517 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1518 | case False | 
| 76894 | 1519 |   then have "\<lbrakk>connected_components_of X \<subseteq> {S}\<rbrakk> \<Longrightarrow> topspace X = S"
 | 
| 1520 | by (metis Sup_empty Union_connected_components_of ccpo_Sup_singleton subset_singleton_iff) | |
| 1521 | with False show ?thesis | |
| 1522 | unfolding connected_components_of_def | |
| 1523 | by (metis connected_space_connected_component_set empty_iff image_subset_iff insert_iff) | |
| 69922 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1524 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1525 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1526 | lemma connected_space_iff_components_subset_singleton: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1527 |    "connected_space X \<longleftrightarrow> (\<exists>a. connected_components_of X \<subseteq> {a})"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1528 | by (simp add: connected_components_of_subset_sing) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1529 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1530 | lemma connected_components_of_eq_singleton: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1531 |    "connected_components_of X = {S}
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1532 | \<longleftrightarrow> connected_space X \<and> topspace X \<noteq> {} \<and> S = topspace X"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1533 | by (metis ccpo_Sup_singleton connected_components_of_subset_sing insert_not_empty subset_singleton_iff) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1534 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1535 | lemma connected_components_of_connected_space: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1536 |    "connected_space X \<Longrightarrow> connected_components_of X = (if topspace X = {} then {} else {topspace X})"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1537 | by (simp add: connected_components_of_eq_empty connected_components_of_eq_singleton) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1538 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1539 | lemma exists_connected_component_of_superset: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1540 |   assumes "connectedin X S" and ne: "topspace X \<noteq> {}"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1541 | shows "\<exists>C. C \<in> connected_components_of X \<and> S \<subseteq> C" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1542 | proof (cases "S = {}")
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1543 | case True | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1544 | then show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1545 | using ne connected_components_of_def by blast | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1546 | next | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1547 | case False | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1548 | then show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1549 | by (meson all_not_in_conv assms(1) connected_component_in_connected_components_of connected_component_of_maximal connectedin_subset_topspace in_mono) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1550 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1551 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1552 | lemma closedin_connected_components_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1553 | assumes "C \<in> connected_components_of X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1554 | shows "closedin X C" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1555 | proof - | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1556 | obtain x where "x \<in> topspace X" and x: "C = connected_component_of_set X x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1557 | using assms by (auto simp: connected_components_of_def) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1558 | have "connected_component_of_set X x \<subseteq> topspace X" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1559 | by (simp add: connected_component_of_subset_topspace) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1560 | moreover have "X closure_of connected_component_of_set X x \<subseteq> connected_component_of_set X x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1561 | proof (rule connected_component_of_maximal) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1562 | show "connectedin X (X closure_of connected_component_of_set X x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1563 | by (simp add: connectedin_closure_of connectedin_connected_component_of) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1564 | show "x \<in> X closure_of connected_component_of_set X x" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1565 | by (simp add: \<open>x \<in> topspace X\<close> closure_of connected_component_of_refl) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1566 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1567 | ultimately | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1568 | show ?thesis | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1569 | using closure_of_subset_eq x by auto | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1570 | qed | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1571 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1572 | lemma closedin_connected_component_of: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1573 | "closedin X (connected_component_of_set X x)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1574 | by (metis closedin_connected_components_of closedin_empty connected_component_in_connected_components_of connected_component_of_eq_empty) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1575 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1576 | lemma connected_component_of_eq_overlap: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1577 | "connected_component_of_set X x = connected_component_of_set X y \<longleftrightarrow> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1578 | (x \<notin> topspace X) \<and> (y \<notin> topspace X) \<or> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1579 |       ~(connected_component_of_set X x \<inter> connected_component_of_set X y = {})"
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1580 | using connected_component_of_equiv by fastforce | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1581 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1582 | lemma connected_component_of_nonoverlap: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1583 |    "connected_component_of_set X x \<inter> connected_component_of_set X y = {} \<longleftrightarrow>
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1584 | (x \<notin> topspace X) \<or> (y \<notin> topspace X) \<or> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1585 | ~(connected_component_of_set X x = connected_component_of_set X y)" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1586 | by (metis connected_component_of_eq_empty connected_component_of_eq_overlap inf.idem) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1587 | |
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1588 | lemma connected_component_of_overlap: | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1589 |    "~(connected_component_of_set X x \<inter> connected_component_of_set X y = {}) \<longleftrightarrow>
 | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1590 | x \<in> topspace X \<and> y \<in> topspace X \<and> | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1591 | connected_component_of_set X x = connected_component_of_set X y" | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1592 | by (meson connected_component_of_nonoverlap) | 
| 
4a9167f377b0
new material about topology, etc.; also fixes for yesterday's
 paulson <lp15@cam.ac.uk> parents: 
69753diff
changeset | 1593 | |
| 69616 
d18dc9c5c456
split off theory combining Elementary_Topology and Abstract_Topology
 immler parents: diff
changeset | 1594 | end |