# HG changeset patch # User paulson # Date 1622292146 -3600 # Node ID a1086aebcd78b577745c244d337fe2986b275983 # Parent aab7975fa070bf59093221ba793754b2dd5d8fe6# Parent e10d530f157a0d7cf1a60e8691dad0cd2cce46c5 merged diff -r aab7975fa070 -r a1086aebcd78 src/HOL/Analysis/Elementary_Normed_Spaces.thy --- a/src/HOL/Analysis/Elementary_Normed_Spaces.thy Fri May 28 20:21:25 2021 +0000 +++ b/src/HOL/Analysis/Elementary_Normed_Spaces.thy Sat May 29 13:42:26 2021 +0100 @@ -763,6 +763,18 @@ using bounded_minus_comp [of fst "S \ T" snd] assms by (auto simp: split_def split: if_split_asm) +lemma bounded_sums: + fixes S :: "'a::real_normed_vector set" + assumes "bounded S" and "bounded T" + shows "bounded (\x\ S. \y \ T. {x + y})" + using assms by (simp add: bounded_iff) (meson norm_triangle_mono) + +lemma bounded_differences: + fixes S :: "'a::real_normed_vector set" + assumes "bounded S" and "bounded T" + shows "bounded (\x\ S. \y \ T. {x - y})" + using assms by (simp add: bounded_iff) (meson add_mono norm_triangle_le_diff) + lemma not_bounded_UNIV[simp]: "\ bounded (UNIV :: 'a::{real_normed_vector, perfect_space} set)" proof (auto simp: bounded_pos not_le) @@ -1292,6 +1304,28 @@ using compact_sums[OF assms(1) compact_negations[OF assms(2)]] by auto qed +lemma compact_sums': + fixes S :: "'a::real_normed_vector set" + assumes "compact S" and "compact T" + shows "compact (\x\ S. \y \ T. {x + y})" +proof - + have "(\x\S. \y\T. {x + y}) = {x + y |x y. x \ S \ y \ T}" + by blast + then show ?thesis + using compact_sums [OF assms] by simp +qed + +lemma compact_differences': + fixes S :: "'a::real_normed_vector set" + assumes "compact S" and "compact T" + shows "compact (\x\ S. \y \ T. {x - y})" +proof - + have "(\x\S. \y\T. {x - y}) = {x - y |x y. x \ S \ y \ T}" + by blast + then show ?thesis + using compact_differences [OF assms] by simp +qed + lemma compact_translation: "compact ((+) a ` s)" if "compact s" for s :: "'a::real_normed_vector set" proof - diff -r aab7975fa070 -r a1086aebcd78 src/HOL/Complex_Analysis/Cauchy_Integral_Formula.thy --- a/src/HOL/Complex_Analysis/Cauchy_Integral_Formula.thy Fri May 28 20:21:25 2021 +0000 +++ b/src/HOL/Complex_Analysis/Cauchy_Integral_Formula.thy Sat May 29 13:42:26 2021 +0100 @@ -2482,12 +2482,13 @@ theorem Liouville_theorem: assumes holf: "f holomorphic_on UNIV" and bf: "bounded (range f)" - obtains c where "\z. f z = c" + shows "f constant_on UNIV" proof - obtain B where "\z. cmod (f z) \ B" by (meson bf bounded_pos rangeI) then show ?thesis - using Liouville_polynomial [OF holf, of 0 B 0, simplified] that by blast + using Liouville_polynomial [OF holf, of 0 B 0, simplified] + by (meson constant_on_def) qed text\A holomorphic function f has only isolated zeros unless f is 0.\