src/HOL/Topological_Spaces.thy
changeset 67727 ce3e87a51488
parent 67707 68ca05a7f159
child 67950 99eaa5cedbb7
equal deleted inserted replaced
67726:0cd2fd0c2dcf 67727:ce3e87a51488
  1286 lemma filterlim_subseq: "strict_mono f \<Longrightarrow> filterlim f sequentially sequentially"
  1286 lemma filterlim_subseq: "strict_mono f \<Longrightarrow> filterlim f sequentially sequentially"
  1287   unfolding filterlim_iff by (metis eventually_subseq)
  1287   unfolding filterlim_iff by (metis eventually_subseq)
  1288 
  1288 
  1289 lemma strict_mono_o: "strict_mono r \<Longrightarrow> strict_mono s \<Longrightarrow> strict_mono (r \<circ> s)"
  1289 lemma strict_mono_o: "strict_mono r \<Longrightarrow> strict_mono s \<Longrightarrow> strict_mono (r \<circ> s)"
  1290   unfolding strict_mono_def by simp
  1290   unfolding strict_mono_def by simp
       
  1291 
       
  1292 lemma strict_mono_compose: "strict_mono r \<Longrightarrow> strict_mono s \<Longrightarrow> strict_mono (\<lambda>x. r (s x))"
       
  1293   using strict_mono_o[of r s] by (simp add: o_def)
  1291 
  1294 
  1292 lemma incseq_imp_monoseq:  "incseq X \<Longrightarrow> monoseq X"
  1295 lemma incseq_imp_monoseq:  "incseq X \<Longrightarrow> monoseq X"
  1293   by (simp add: incseq_def monoseq_def)
  1296   by (simp add: incseq_def monoseq_def)
  1294 
  1297 
  1295 lemma decseq_imp_monoseq:  "decseq X \<Longrightarrow> monoseq X"
  1298 lemma decseq_imp_monoseq:  "decseq X \<Longrightarrow> monoseq X"
  1881   using continuous_on_open_Union [of "{s,t}"] by auto
  1884   using continuous_on_open_Union [of "{s,t}"] by auto
  1882 
  1885 
  1883 lemma continuous_on_closed_Un:
  1886 lemma continuous_on_closed_Un:
  1884   "closed s \<Longrightarrow> closed t \<Longrightarrow> continuous_on s f \<Longrightarrow> continuous_on t f \<Longrightarrow> continuous_on (s \<union> t) f"
  1887   "closed s \<Longrightarrow> closed t \<Longrightarrow> continuous_on s f \<Longrightarrow> continuous_on t f \<Longrightarrow> continuous_on (s \<union> t) f"
  1885   by (auto simp add: continuous_on_closed_vimage closed_Un Int_Un_distrib)
  1888   by (auto simp add: continuous_on_closed_vimage closed_Un Int_Un_distrib)
       
  1889 
       
  1890 lemma continuous_on_closed_Union:
       
  1891   assumes "finite I"
       
  1892     "\<And>i. i \<in> I \<Longrightarrow> closed (U i)"
       
  1893     "\<And>i. i \<in> I \<Longrightarrow> continuous_on (U i) f"
       
  1894   shows "continuous_on (\<Union> i \<in> I. U i) f"
       
  1895   using assms
       
  1896   by (induction I) (auto intro!: continuous_on_closed_Un)
  1886 
  1897 
  1887 lemma continuous_on_If:
  1898 lemma continuous_on_If:
  1888   assumes closed: "closed s" "closed t"
  1899   assumes closed: "closed s" "closed t"
  1889     and cont: "continuous_on s f" "continuous_on t g"
  1900     and cont: "continuous_on s f" "continuous_on t g"
  1890     and P: "\<And>x. x \<in> s \<Longrightarrow> \<not> P x \<Longrightarrow> f x = g x" "\<And>x. x \<in> t \<Longrightarrow> P x \<Longrightarrow> f x = g x"
  1901     and P: "\<And>x. x \<in> s \<Longrightarrow> \<not> P x \<Longrightarrow> f x = g x" "\<And>x. x \<in> t \<Longrightarrow> P x \<Longrightarrow> f x = g x"