src/HOL/Multivariate_Analysis/Ordered_Euclidean_Space.thy
changeset 62620 d21dab28b3f9
parent 62376 85f38d5f8807
child 63469 b6900858dcb9
equal deleted inserted replaced
62619:7f17ebd3293e 62620:d21dab28b3f9
   221 lemma compact_interval:
   221 lemma compact_interval:
   222   fixes a b::"'a::ordered_euclidean_space"
   222   fixes a b::"'a::ordered_euclidean_space"
   223   shows "compact {a .. b}"
   223   shows "compact {a .. b}"
   224   by (metis compact_cbox interval_cbox)
   224   by (metis compact_cbox interval_cbox)
   225 
   225 
       
   226 lemma homeomorphic_closed_intervals:
       
   227   fixes a :: "'a::euclidean_space" and b and c :: "'a::euclidean_space" and d
       
   228   assumes "box a b \<noteq> {}" and "box c d \<noteq> {}"
       
   229     shows "(cbox a b) homeomorphic (cbox c d)"
       
   230 apply (rule homeomorphic_convex_compact)
       
   231 using assms apply auto
       
   232 done
       
   233 
       
   234 lemma homeomorphic_closed_intervals_real:
       
   235   fixes a::real and b and c::real and d
       
   236   assumes "a<b" and "c<d"
       
   237     shows "{a..b} homeomorphic {c..d}"
       
   238 by (metis assms compact_interval continuous_on_id convex_real_interval(5) emptyE homeomorphic_convex_compact interior_atLeastAtMost_real mvt)
       
   239 
   226 no_notation
   240 no_notation
   227   eucl_less (infix "<e" 50)
   241   eucl_less (infix "<e" 50)
   228 
   242 
   229 lemma One_nonneg: "0 \<le> (\<Sum>Basis::'a::ordered_euclidean_space)"
   243 lemma One_nonneg: "0 \<le> (\<Sum>Basis::'a::ordered_euclidean_space)"
   230   by (auto intro: setsum_nonneg)
   244   by (auto intro: setsum_nonneg)