src/HOL/Analysis/Topology_Euclidean_Space.thy
author wenzelm
Wed, 12 Mar 2025 11:39:00 +0100
changeset 82265 4b875a4c83b0
parent 81128 5b201b24d99b
child 82518 da14e77a48b2
permissions -rw-r--r--
update for release;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
63938
f6ce08859d4c More mainly topological results
paulson <lp15@cam.ac.uk>
parents: 63928
diff changeset
     1
(*  Author:     L C Paulson, University of Cambridge
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     2
    Author:     Amine Chaieb, University of Cambridge
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     3
    Author:     Robert Himmelmann, TU Muenchen
44075
5952bd355779 generalize more lemmas about compactness
huffman
parents: 44074
diff changeset
     4
    Author:     Brian Huffman, Portland State University
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     5
*)
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     6
69676
56acd449da41 chapters for analysis manual
immler
parents: 69619
diff changeset
     7
chapter \<open>Vector Analysis\<close>
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     8
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     9
theory Topology_Euclidean_Space
69516
09bb8f470959 most of Topology_Euclidean_Space (now Elementary_Topology) requires fewer dependencies
immler
parents: 69508
diff changeset
    10
  imports
69544
5aa5a8d6e5b5 split off theorems involving classes below metric_space and real_normed_vector
immler
parents: 69516
diff changeset
    11
    Elementary_Normed_Spaces
69516
09bb8f470959 most of Topology_Euclidean_Space (now Elementary_Topology) requires fewer dependencies
immler
parents: 69508
diff changeset
    12
    Linear_Algebra
09bb8f470959 most of Topology_Euclidean_Space (now Elementary_Topology) requires fewer dependencies
immler
parents: 69508
diff changeset
    13
    Norm_Arith
51343
b61b32f62c78 use generate_topology for second countable topologies, does not require intersection stable basis
hoelzl
parents: 51342
diff changeset
    14
begin
b61b32f62c78 use generate_topology for second countable topologies, does not require intersection stable basis
hoelzl
parents: 51342
diff changeset
    15
69676
56acd449da41 chapters for analysis manual
immler
parents: 69619
diff changeset
    16
section \<open>Elementary Topology in Euclidean Space\<close>
56acd449da41 chapters for analysis manual
immler
parents: 69619
diff changeset
    17
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
    18
lemma euclidean_dist_l2:
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
    19
  fixes x y :: "'a :: euclidean_space"
67155
9e5b05d54f9d canonical name
nipkow
parents: 66939
diff changeset
    20
  shows "dist x y = L2_set (\<lambda>i. dist (x \<bullet> i) (y \<bullet> i)) Basis"
9e5b05d54f9d canonical name
nipkow
parents: 66939
diff changeset
    21
  unfolding dist_norm norm_eq_sqrt_inner L2_set_def
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
    22
  by (subst euclidean_inner) (simp add: power2_eq_square inner_diff_left)
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
    23
67685
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    24
lemma norm_nth_le: "norm (x \<bullet> i) \<le> norm x" if "i \<in> Basis"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    25
proof -
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    26
  have "(x \<bullet> i)\<^sup>2 = (\<Sum>i\<in>{i}. (x \<bullet> i)\<^sup>2)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    27
    by simp
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    28
  also have "\<dots> \<le> (\<Sum>i\<in>Basis. (x \<bullet> i)\<^sup>2)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    29
    by (intro sum_mono2) (auto simp: that)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    30
  finally show ?thesis
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    31
    unfolding norm_conv_dist euclidean_dist_l2[of x] L2_set_def
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    32
    by (auto intro!: real_le_rsqrt)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    33
qed
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
    34
71033
nipkow
parents: 71030
diff changeset
    35
subsection\<^marker>\<open>tag unimportant\<close> \<open>Continuity of the representation WRT an orthogonal basis\<close>
70065
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    36
70086
72c52a897de2 First tranche of the Homology development: Simplices
paulson <lp15@cam.ac.uk>
parents: 70065
diff changeset
    37
lemma orthogonal_Basis: "pairwise orthogonal Basis"
72c52a897de2 First tranche of the Homology development: Simplices
paulson <lp15@cam.ac.uk>
parents: 70065
diff changeset
    38
  by (simp add: inner_not_same_Basis orthogonal_def pairwise_def)
72c52a897de2 First tranche of the Homology development: Simplices
paulson <lp15@cam.ac.uk>
parents: 70065
diff changeset
    39
70065
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    40
lemma representation_bound:
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    41
  fixes B :: "'N::real_inner set"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    42
  assumes "finite B" "independent B" "b \<in> B" and orth: "pairwise orthogonal B"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    43
  obtains m where "m > 0" "\<And>x. x \<in> span B \<Longrightarrow> \<bar>representation B x b\<bar> \<le> m * norm x"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    44
proof 
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    45
  fix x
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    46
  assume x: "x \<in> span B"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    47
  have "b \<noteq> 0"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    48
    using \<open>independent B\<close> \<open>b \<in> B\<close> dependent_zero by blast
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    49
  have [simp]: "b \<bullet> b' = (if b' = b then (norm b)\<^sup>2 else 0)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    50
    if "b \<in> B" "b' \<in> B" for b b'
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    51
    using orth by (simp add: orthogonal_def pairwise_def norm_eq_sqrt_inner that)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    52
  have "norm x = norm (\<Sum>b\<in>B. representation B x b *\<^sub>R b)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    53
    using real_vector.sum_representation_eq [OF \<open>independent B\<close> x \<open>finite B\<close> order_refl]
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    54
    by simp
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    55
  also have "\<dots> = sqrt ((\<Sum>b\<in>B. representation B x b *\<^sub>R b) \<bullet> (\<Sum>b\<in>B. representation B x b *\<^sub>R b))"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    56
    by (simp add: norm_eq_sqrt_inner)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    57
  also have "\<dots> = sqrt (\<Sum>b\<in>B. (representation B x b *\<^sub>R b) \<bullet> (representation B x b *\<^sub>R b))"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    58
    using \<open>finite B\<close>
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    59
    by (simp add: inner_sum_left inner_sum_right if_distrib [of "\<lambda>x. _ * x"] cong: if_cong sum.cong_simp)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    60
  also have "\<dots> = sqrt (\<Sum>b\<in>B. (norm (representation B x b *\<^sub>R b))\<^sup>2)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    61
    by (simp add: mult.commute mult.left_commute power2_eq_square)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    62
  also have "\<dots> = sqrt (\<Sum>b\<in>B. (representation B x b)\<^sup>2 * (norm b)\<^sup>2)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    63
    by (simp add: norm_mult power_mult_distrib)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    64
  finally have "norm x = sqrt (\<Sum>b\<in>B. (representation B x b)\<^sup>2 * (norm b)\<^sup>2)" .
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    65
  moreover
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    66
  have "sqrt ((representation B x b)\<^sup>2 * (norm b)\<^sup>2) \<le> sqrt (\<Sum>b\<in>B. (representation B x b)\<^sup>2 * (norm b)\<^sup>2)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    67
    using \<open>b \<in> B\<close> \<open>finite B\<close> by (auto intro: member_le_sum)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    68
  then have "\<bar>representation B x b\<bar> \<le> (1 / norm b) * sqrt (\<Sum>b\<in>B. (representation B x b)\<^sup>2 * (norm b)\<^sup>2)"
70817
dd675800469d dedicated fact collections for algebraic simplification rules potentially splitting goals
haftmann
parents: 70802
diff changeset
    69
    using \<open>b \<noteq> 0\<close> by (simp add: field_split_simps real_sqrt_mult del: real_sqrt_le_iff)
70065
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    70
  ultimately show "\<bar>representation B x b\<bar> \<le> (1 / norm b) * norm x"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    71
    by simp
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    72
next
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    73
  show "0 < 1 / norm b"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    74
    using \<open>independent B\<close> \<open>b \<in> B\<close> dependent_zero by auto
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    75
qed 
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    76
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    77
lemma continuous_on_representation:
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    78
  fixes B :: "'N::euclidean_space set"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    79
  assumes "finite B" "independent B" "b \<in> B" "pairwise orthogonal B" 
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    80
  shows "continuous_on (span B) (\<lambda>x. representation B x b)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    81
proof
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    82
  show "\<exists>d>0. \<forall>x'\<in>span B. dist x' x < d \<longrightarrow> dist (representation B x' b) (representation B x b) \<le> e"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    83
    if "e > 0" "x \<in> span B" for x e
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    84
  proof -
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    85
    obtain m where "m > 0" and m: "\<And>x. x \<in> span B \<Longrightarrow> \<bar>representation B x b\<bar> \<le> m * norm x"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    86
      using assms representation_bound by blast
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    87
    show ?thesis
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    88
      unfolding dist_norm
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    89
    proof (intro exI conjI ballI impI)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    90
      show "e/m > 0"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    91
        by (simp add: \<open>e > 0\<close> \<open>m > 0\<close>)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    92
      show "norm (representation B x' b - representation B x b) \<le> e"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    93
        if x': "x' \<in> span B" and less: "norm (x'-x) < e/m" for x' 
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    94
      proof -
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    95
        have "\<bar>representation B (x'-x) b\<bar> \<le> m * norm (x'-x)"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    96
          using m [of "x'-x"] \<open>x \<in> span B\<close> span_diff x' by blast
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    97
        also have "\<dots> < e"
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    98
          by (metis \<open>m > 0\<close> less mult.commute pos_less_divide_eq)
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
    99
        finally have "\<bar>representation B (x'-x) b\<bar> \<le> e" by simp
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
   100
        then show ?thesis
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
   101
          by (simp add: \<open>x \<in> span B\<close> \<open>independent B\<close> representation_diff x')
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
   102
      qed
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
   103
    qed
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
   104
  qed
cc89a395b5a3 Free_Abelian_Groups finally working; fixed some duplicates; cleaned up some proofs
paulson <lp15@cam.ac.uk>
parents: 70019
diff changeset
   105
qed
67685
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   106
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
   107
subsection\<^marker>\<open>tag unimportant\<close>\<open>Balls in Euclidean Space\<close>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   108
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   109
lemma cball_subset_cball_iff:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   110
  fixes a :: "'a :: euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   111
  shows "cball a r \<subseteq> cball a' r' \<longleftrightarrow> dist a a' + r \<le> r' \<or> r < 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   112
    (is "?lhs \<longleftrightarrow> ?rhs")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   113
proof
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   114
  assume ?lhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   115
  then show ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   116
  proof (cases "r < 0")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   117
    case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   118
    then show ?rhs by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   119
  next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   120
    case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   121
    then have [simp]: "r \<ge> 0" by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   122
    have "norm (a - a') + r \<le> r'"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   123
    proof (cases "a = a'")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   124
      case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   125
      then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   126
        using subsetD [where c = "a + r *\<^sub>R (SOME i. i \<in> Basis)", OF \<open>?lhs\<close>] subsetD [where c = a, OF \<open>?lhs\<close>]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   127
        by (force simp: SOME_Basis dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   128
    next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   129
      case False
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   130
      have "norm (a' - (a + (r / norm (a - a')) *\<^sub>R (a - a'))) = norm ((-1 - (r / norm (a - a'))) *\<^sub>R (a - a'))"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   131
        by (simp add: algebra_simps)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   132
      also from \<open>a \<noteq> a'\<close> have "... = \<bar>- norm (a - a') - r\<bar>"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   133
        by (simp add: divide_simps)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   134
      finally have [simp]: "norm (a' - (a + (r / norm (a - a')) *\<^sub>R (a - a'))) = \<bar>norm (a - a') + r\<bar>"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   135
        by linarith
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   136
      from \<open>a \<noteq> a'\<close> show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   137
        using subsetD [where c = "a' + (1 + r / norm(a - a')) *\<^sub>R (a - a')", OF \<open>?lhs\<close>]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   138
        by (simp add: dist_norm scaleR_add_left)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   139
    qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   140
    then show ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   141
      by (simp add: dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   142
  qed
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   143
qed metric
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   144
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   145
lemma cball_subset_ball_iff: "cball a r \<subseteq> ball a' r' \<longleftrightarrow> dist a a' + r < r' \<or> r < 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   146
  (is "?lhs \<longleftrightarrow> ?rhs")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   147
  for a :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   148
proof
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   149
  assume ?lhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   150
  then show ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   151
  proof (cases "r < 0")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   152
    case True then
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   153
    show ?rhs by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   154
  next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   155
    case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   156
    then have [simp]: "r \<ge> 0" by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   157
    have "norm (a - a') + r < r'"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   158
    proof (cases "a = a'")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   159
      case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   160
      then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   161
        using subsetD [where c = "a + r *\<^sub>R (SOME i. i \<in> Basis)", OF \<open>?lhs\<close>] subsetD [where c = a, OF \<open>?lhs\<close>]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   162
        by (force simp: SOME_Basis dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   163
    next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   164
      case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   165
      have False if "norm (a - a') + r \<ge> r'"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   166
      proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   167
        from that have "\<bar>r' - norm (a - a')\<bar> \<le> r"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   168
          by (smt (verit, best) \<open>0 \<le> r\<close> \<open>?lhs\<close> ball_subset_cball cball_subset_cball_iff dist_norm order_trans)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   169
        then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   170
          using subsetD [where c = "a + (r' / norm(a - a') - 1) *\<^sub>R (a - a')", OF \<open>?lhs\<close>] \<open>a \<noteq> a'\<close>
70802
160eaf566bcb formally augmented corresponding rules for field_simps
haftmann
parents: 70136
diff changeset
   171
          apply (simp add: dist_norm)
160eaf566bcb formally augmented corresponding rules for field_simps
haftmann
parents: 70136
diff changeset
   172
          apply (simp add: scaleR_left_diff_distrib)
160eaf566bcb formally augmented corresponding rules for field_simps
haftmann
parents: 70136
diff changeset
   173
          apply (simp add: field_simps)
160eaf566bcb formally augmented corresponding rules for field_simps
haftmann
parents: 70136
diff changeset
   174
          done
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   175
      qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   176
      then show ?thesis by force
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   177
    qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   178
    then show ?rhs by (simp add: dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   179
  qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   180
next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   181
  assume ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   182
  then show ?lhs
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   183
    by metric
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   184
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   185
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   186
lemma ball_subset_cball_iff: "ball a r \<subseteq> cball a' r' \<longleftrightarrow> dist a a' + r \<le> r' \<or> r \<le> 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   187
  (is "?lhs = ?rhs")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   188
  for a :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   189
proof (cases "r \<le> 0")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   190
  case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   191
  then show ?thesis
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   192
    by metric
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   193
next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   194
  case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   195
  show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   196
  proof
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   197
    assume ?lhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   198
    then have "(cball a r \<subseteq> cball a' r')"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   199
      by (metis False closed_cball closure_ball closure_closed closure_mono not_less)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   200
    with False show ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   201
      by (fastforce iff: cball_subset_cball_iff)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   202
  next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   203
    assume ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   204
    with False show ?lhs
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   205
      by metric
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   206
  qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   207
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   208
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   209
lemma ball_subset_ball_iff:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   210
  fixes a :: "'a :: euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   211
  shows "ball a r \<subseteq> ball a' r' \<longleftrightarrow> dist a a' + r \<le> r' \<or> r \<le> 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   212
        (is "?lhs = ?rhs")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   213
proof (cases "r \<le> 0")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   214
  case True then show ?thesis
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   215
    by metric
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   216
next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   217
  case False show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   218
  proof
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   219
    assume ?lhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   220
    then have "0 < r'"
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   221
      using False by metric
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   222
    then have "cball a r \<subseteq> cball a' r'"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   223
      by (metis False \<open>?lhs\<close> closure_ball closure_mono not_less)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   224
    then show ?rhs
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   225
      using False cball_subset_cball_iff by fastforce
70952
f140135ff375 example applications of the 'metric' decision procedure, by Maximilian Schäffeler
immler
parents: 70817
diff changeset
   226
  qed metric
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   227
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   228
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   229
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   230
lemma ball_eq_ball_iff:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   231
  fixes x :: "'a :: euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   232
  shows "ball x d = ball y e \<longleftrightarrow> d \<le> 0 \<and> e \<le> 0 \<or> x=y \<and> d=e"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   233
  by (smt (verit, del_insts) ball_empty ball_subset_cball_iff dist_norm norm_pths(2))
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   234
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   235
lemma cball_eq_cball_iff:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   236
  fixes x :: "'a :: euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   237
  shows "cball x d = cball y e \<longleftrightarrow> d < 0 \<and> e < 0 \<or> x=y \<and> d=e"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   238
  by (smt (verit, ccfv_SIG) cball_empty cball_subset_cball_iff dist_norm norm_pths(2) zero_le_dist)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   239
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   240
lemma ball_eq_cball_iff:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   241
  fixes x :: "'a :: euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   242
  shows "ball x d = cball y e \<longleftrightarrow> d \<le> 0 \<and> e < 0" (is "?lhs = ?rhs")
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   243
  by (smt (verit) ball_eq_empty ball_subset_cball_iff cball_eq_empty cball_subset_ball_iff order.refl)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   244
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   245
lemma cball_eq_ball_iff:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   246
  fixes x :: "'a :: euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   247
  shows "cball x d = ball y e \<longleftrightarrow> d < 0 \<and> e \<le> 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   248
  using ball_eq_cball_iff by blast
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   249
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   250
lemma finite_ball_avoid:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   251
  fixes S :: "'a :: euclidean_space set"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   252
  assumes "open S" "finite X" "p \<in> S"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   253
  shows "\<exists>e>0. \<forall>w\<in>ball p e. w\<in>S \<and> (w\<noteq>p \<longrightarrow> w\<notin>X)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   254
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   255
  obtain e1 where "0 < e1" and e1_b:"ball p e1 \<subseteq> S"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   256
    using open_contains_ball_eq[OF \<open>open S\<close>] assms by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   257
  obtain e2 where "0 < e2" and "\<forall>x\<in>X. x \<noteq> p \<longrightarrow> e2 \<le> dist p x"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   258
    using finite_set_avoid[OF \<open>finite X\<close>,of p] by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   259
  hence "\<forall>w\<in>ball p (min e1 e2). w\<in>S \<and> (w\<noteq>p \<longrightarrow> w\<notin>X)" using e1_b by auto
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   260
  thus "\<exists>e>0. \<forall>w\<in>ball p e. w \<in> S \<and> (w \<noteq> p \<longrightarrow> w \<notin> X)" 
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   261
    using \<open>e2>0\<close> \<open>e1>0\<close> by (rule_tac x="min e1 e2" in exI) auto
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   262
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   263
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   264
lemma finite_cball_avoid:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   265
  fixes S :: "'a :: euclidean_space set"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   266
  assumes "open S" "finite X" "p \<in> S"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   267
  shows "\<exists>e>0. \<forall>w\<in>cball p e. w\<in>S \<and> (w\<noteq>p \<longrightarrow> w\<notin>X)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   268
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   269
  obtain e1 where "e1>0" and e1: "\<forall>w\<in>ball p e1. w\<in>S \<and> (w\<noteq>p \<longrightarrow> w\<notin>X)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   270
    using finite_ball_avoid[OF assms] by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   271
  define e2 where "e2 \<equiv> e1/2"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   272
  have "e2>0" and "e2 < e1" unfolding e2_def using \<open>e1>0\<close> by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   273
  then have "cball p e2 \<subseteq> ball p e1" by (subst cball_subset_ball_iff,auto)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   274
  then show "\<exists>e>0. \<forall>w\<in>cball p e. w \<in> S \<and> (w \<noteq> p \<longrightarrow> w \<notin> X)" using \<open>e2>0\<close> e1 by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   275
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   276
69619
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   277
lemma dim_cball:
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   278
  assumes "e > 0"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   279
  shows "dim (cball (0 :: 'n::euclidean_space) e) = DIM('n)"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   280
proof -
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   281
  {
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   282
    fix x :: "'n::euclidean_space"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   283
    define y where "y = (e / norm x) *\<^sub>R x"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   284
    then have "y \<in> cball 0 e"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   285
      using assms by auto
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   286
    moreover have *: "x = (norm x / e) *\<^sub>R y"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   287
      using y_def assms by simp
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   288
    moreover from * have "x = (norm x/e) *\<^sub>R y"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   289
      by auto
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   290
    ultimately have "x \<in> span (cball 0 e)"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   291
      using span_scale[of y "cball 0 e" "norm x/e"]
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   292
        span_superset[of "cball 0 e"]
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   293
      by (simp add: span_base)
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   294
  }
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   295
  then have "span (cball 0 e) = (UNIV :: 'n::euclidean_space set)"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   296
    by auto
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   297
  then show ?thesis
71172
nipkow
parents: 71033
diff changeset
   298
    using dim_span[of "cball (0 :: 'n::euclidean_space) e"] by (auto)
69619
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   299
qed
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   300
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   301
60420
884f54e01427 isabelle update_cartouches;
wenzelm
parents: 60176
diff changeset
   302
subsection \<open>Boxes\<close>
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   303
71033
nipkow
parents: 71030
diff changeset
   304
abbreviation\<^marker>\<open>tag important\<close> One :: "'a::euclidean_space" where
nipkow
parents: 71030
diff changeset
   305
"One \<equiv> \<Sum>Basis"
57447
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   306
63114
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   307
lemma One_non_0: assumes "One = (0::'a::euclidean_space)" shows False
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   308
proof -
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   309
  have "dependent (Basis :: 'a set)"
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   310
    apply (simp add: dependent_finite)
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   311
    apply (rule_tac x="\<lambda>i. 1" in exI)
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   312
    using SOME_Basis apply (auto simp: assms)
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   313
    done
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   314
  with independent_Basis show False by force
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   315
qed
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   316
71033
nipkow
parents: 71030
diff changeset
   317
corollary\<^marker>\<open>tag unimportant\<close> One_neq_0[iff]: "One \<noteq> 0"
63114
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   318
  by (metis One_non_0)
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   319
71033
nipkow
parents: 71030
diff changeset
   320
corollary\<^marker>\<open>tag unimportant\<close> Zero_neq_One[iff]: "0 \<noteq> One"
63114
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   321
  by (metis One_non_0)
27afe7af7379 Lots of new material for multivariate analysis
paulson <lp15@cam.ac.uk>
parents: 63105
diff changeset
   322
80914
d97fdabd9e2b standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents: 80034
diff changeset
   323
definition\<^marker>\<open>tag important\<close> (in euclidean_space) eucl_less (infix \<open><e\<close> 50) where 
71033
nipkow
parents: 71030
diff changeset
   324
"eucl_less a b \<longleftrightarrow> (\<forall>i\<in>Basis. a \<bullet> i < b \<bullet> i)"
54775
2d3df8633dad prefer box over greaterThanLessThan on euclidean_space
immler
parents: 54489
diff changeset
   325
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
   326
definition\<^marker>\<open>tag important\<close> box_eucl_less: "box a b = {x. a <e x \<and> x <e b}"
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
   327
definition\<^marker>\<open>tag important\<close> "cbox a b = {x. \<forall>i\<in>Basis. a \<bullet> i \<le> x \<bullet> i \<and> x \<bullet> i \<le> b \<bullet> i}"
54775
2d3df8633dad prefer box over greaterThanLessThan on euclidean_space
immler
parents: 54489
diff changeset
   328
2d3df8633dad prefer box over greaterThanLessThan on euclidean_space
immler
parents: 54489
diff changeset
   329
lemma box_def: "box a b = {x. \<forall>i\<in>Basis. a \<bullet> i < x \<bullet> i \<and> x \<bullet> i < b \<bullet> i}"
2d3df8633dad prefer box over greaterThanLessThan on euclidean_space
immler
parents: 54489
diff changeset
   330
  and in_box_eucl_less: "x \<in> box a b \<longleftrightarrow> a <e x \<and> x <e b"
56188
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   331
  and mem_box: "x \<in> box a b \<longleftrightarrow> (\<forall>i\<in>Basis. a \<bullet> i < x \<bullet> i \<and> x \<bullet> i < b \<bullet> i)"
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   332
    "x \<in> cbox a b \<longleftrightarrow> (\<forall>i\<in>Basis. a \<bullet> i \<le> x \<bullet> i \<and> x \<bullet> i \<le> b \<bullet> i)"
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   333
  by (auto simp: box_eucl_less eucl_less_def cbox_def)
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   334
60615
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   335
lemma cbox_Pair_eq: "cbox (a, c) (b, d) = cbox a b \<times> cbox c d"
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   336
  by (force simp: cbox_def Basis_prod_def)
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   337
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   338
lemma cbox_Pair_iff [iff]: "(x, y) \<in> cbox (a, c) (b, d) \<longleftrightarrow> x \<in> cbox a b \<and> y \<in> cbox c d"
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   339
  by (force simp: cbox_Pair_eq)
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   340
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 65585
diff changeset
   341
lemma cbox_Complex_eq: "cbox (Complex a c) (Complex b d) = (\<lambda>(x,y). Complex x y) ` (cbox a b \<times> cbox c d)"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   342
  by (force simp: cbox_def Basis_complex_def)
65587
16a8991ab398 New material (and some tidying) purely in the Analysis directory
paulson <lp15@cam.ac.uk>
parents: 65585
diff changeset
   343
60615
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   344
lemma cbox_Pair_eq_0: "cbox (a, c) (b, d) = {} \<longleftrightarrow> cbox a b = {} \<or> cbox c d = {}"
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   345
  by (force simp: cbox_Pair_eq)
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   346
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   347
lemma swap_cbox_Pair [simp]: "prod.swap ` cbox (c, a) (d, b) = cbox (a,c) (b,d)"
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   348
  by auto
e5fa1d5d3952 Useful lemmas. The theorem concerning swapping the variables in a double integral.
paulson <lp15@cam.ac.uk>
parents: 60585
diff changeset
   349
56188
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   350
lemma mem_box_real[simp]:
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   351
  "(x::real) \<in> box a b \<longleftrightarrow> a < x \<and> x < b"
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   352
  "(x::real) \<in> cbox a b \<longleftrightarrow> a \<le> x \<and> x \<le> b"
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   353
  by (auto simp: mem_box)
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   354
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   355
lemma box_real[simp]:
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   356
  fixes a b:: real
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   357
  shows "box a b = {a <..< b}" "cbox a b = {a .. b}"
0268784f60da use cbox to relax class constraints
immler
parents: 56166
diff changeset
   358
  by auto
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   359
57447
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   360
lemma box_Int_box:
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   361
  fixes a :: "'a::euclidean_space"
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   362
  shows "box a b \<inter> box c d =
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   363
    box (\<Sum>i\<in>Basis. max (a\<bullet>i) (c\<bullet>i) *\<^sub>R i) (\<Sum>i\<in>Basis. min (b\<bullet>i) (d\<bullet>i) *\<^sub>R i)"
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   364
  unfolding set_eq_iff and Int_iff and mem_box by auto
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   365
50087
635d73673b5e regularity of measures, therefore:
immler
parents: 49962
diff changeset
   366
lemma rational_boxes:
61076
bdc1e2f0a86a eliminated \<Colon>;
wenzelm
parents: 60974
diff changeset
   367
  fixes x :: "'a::euclidean_space"
53291
f7fa953bd15b tuned proofs;
wenzelm
parents: 53282
diff changeset
   368
  assumes "e > 0"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
   369
  shows "\<exists>a b. (\<forall>i\<in>Basis. a \<bullet> i \<in> \<rat> \<and> b \<bullet> i \<in> \<rat>) \<and> x \<in> box a b \<and> box a b \<subseteq> ball x e"
50087
635d73673b5e regularity of measures, therefore:
immler
parents: 49962
diff changeset
   370
proof -
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 63007
diff changeset
   371
  define e' where "e' = e / (2 * sqrt (real (DIM ('a))))"
53291
f7fa953bd15b tuned proofs;
wenzelm
parents: 53282
diff changeset
   372
  then have e: "e' > 0"
71172
nipkow
parents: 71033
diff changeset
   373
    using assms by (auto)
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   374
  have "\<exists>y. y \<in> \<rat> \<and> y < x \<bullet> i \<and> x \<bullet> i - y < e'" for i
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   375
    using Rats_dense_in_real[of "x \<bullet> i - e'" "x \<bullet> i"] e by force
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   376
  then obtain a where
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   377
    a: "\<And>u. a u \<in> \<rat> \<and> a u < x \<bullet> u \<and> x \<bullet> u - a u < e'" by metis
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   378
  have "\<exists>y. y \<in> \<rat> \<and> x \<bullet> i < y \<and> y - x \<bullet> i < e'" for i
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   379
    using Rats_dense_in_real[of "x \<bullet> i" "x \<bullet> i + e'"] e by force
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   380
  then obtain b where
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   381
    b: "\<And>u. b u \<in> \<rat> \<and> x \<bullet> u < b u \<and> b u - x \<bullet> u < e'" by metis
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   382
  let ?a = "\<Sum>i\<in>Basis. a i *\<^sub>R i" and ?b = "\<Sum>i\<in>Basis. b i *\<^sub>R i"
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   383
  show ?thesis
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   384
  proof (rule exI[of _ ?a], rule exI[of _ ?b], safe)
53255
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   385
    fix y :: 'a
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   386
    assume *: "y \<in> box ?a ?b"
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52625
diff changeset
   387
    have "dist x y = sqrt (\<Sum>i\<in>Basis. (dist (x \<bullet> i) (y \<bullet> i))\<^sup>2)"
67155
9e5b05d54f9d canonical name
nipkow
parents: 66939
diff changeset
   388
      unfolding L2_set_def[symmetric] by (rule euclidean_dist_l2)
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   389
    also have "\<dots> < sqrt (\<Sum>(i::'a)\<in>Basis. e^2 / real (DIM('a)))"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 64240
diff changeset
   390
    proof (rule real_sqrt_less_mono, rule sum_strict_mono)
53255
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   391
      fix i :: "'a"
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   392
      assume i: "i \<in> Basis"
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   393
      have "a i < y\<bullet>i \<and> y\<bullet>i < b i"
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   394
        using * i by (auto simp: box_def)
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   395
      moreover have "a i < x\<bullet>i" "x\<bullet>i - a i < e'" "x\<bullet>i < b i" "b i - x\<bullet>i < e'"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   396
        using a b by auto
53255
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   397
      ultimately have "\<bar>x\<bullet>i - y\<bullet>i\<bar> < 2 * e'"
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   398
        by auto
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   399
      then have "dist (x \<bullet> i) (y \<bullet> i) < e/sqrt (real (DIM('a)))"
50087
635d73673b5e regularity of measures, therefore:
immler
parents: 49962
diff changeset
   400
        unfolding e'_def by (auto simp: dist_real_def)
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52625
diff changeset
   401
      then have "(dist (x \<bullet> i) (y \<bullet> i))\<^sup>2 < (e/sqrt (real (DIM('a))))\<^sup>2"
50087
635d73673b5e regularity of measures, therefore:
immler
parents: 49962
diff changeset
   402
        by (rule power_strict_mono) auto
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52625
diff changeset
   403
      then show "(dist (x \<bullet> i) (y \<bullet> i))\<^sup>2 < e\<^sup>2 / real DIM('a)"
50087
635d73673b5e regularity of measures, therefore:
immler
parents: 49962
diff changeset
   404
        by (simp add: power_divide)
635d73673b5e regularity of measures, therefore:
immler
parents: 49962
diff changeset
   405
    qed auto
53255
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   406
    also have "\<dots> = e"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   407
      using \<open>0 < e\<close> by simp
53255
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   408
    finally show "y \<in> ball x e"
addd7b9b2bff tuned proofs;
wenzelm
parents: 53015
diff changeset
   409
      by (auto simp: ball_def)
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   410
  qed (use a b in \<open>auto simp: box_def\<close>)
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   411
qed
51103
5dd7b89a16de generalized
immler
parents: 51102
diff changeset
   412
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   413
lemma open_UNION_box:
61076
bdc1e2f0a86a eliminated \<Colon>;
wenzelm
parents: 60974
diff changeset
   414
  fixes M :: "'a::euclidean_space set"
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
   415
  assumes "open M"
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   416
  defines "a' \<equiv> \<lambda>f :: 'a \<Rightarrow> real \<times> real. (\<Sum>(i::'a)\<in>Basis. fst (f i) *\<^sub>R i)"
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   417
  defines "b' \<equiv> \<lambda>f :: 'a \<Rightarrow> real \<times> real. (\<Sum>(i::'a)\<in>Basis. snd (f i) *\<^sub>R i)"
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52625
diff changeset
   418
  defines "I \<equiv> {f\<in>Basis \<rightarrow>\<^sub>E \<rat> \<times> \<rat>. box (a' f) (b' f) \<subseteq> M}"
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 50324
diff changeset
   419
  shows "M = (\<Union>f\<in>I. box (a' f) (b' f))"
52624
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   420
proof -
60462
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   421
  have "x \<in> (\<Union>f\<in>I. box (a' f) (b' f))" if "x \<in> M" for x
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   422
  proof -
52624
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   423
    obtain e where e: "e > 0" "ball x e \<subseteq> M"
60420
884f54e01427 isabelle update_cartouches;
wenzelm
parents: 60176
diff changeset
   424
      using openE[OF \<open>open M\<close> \<open>x \<in> M\<close>] by auto
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
   425
    moreover obtain a b where ab:
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
   426
      "x \<in> box a b"
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
   427
      "\<forall>i \<in> Basis. a \<bullet> i \<in> \<rat>"
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
   428
      "\<forall>i\<in>Basis. b \<bullet> i \<in> \<rat>"
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
   429
      "box a b \<subseteq> ball x e"
52624
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   430
      using rational_boxes[OF e(1)] by metis
60462
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   431
    ultimately show ?thesis
52624
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   432
       by (intro UN_I[of "\<lambda>i\<in>Basis. (a \<bullet> i, b \<bullet> i)"])
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   433
          (auto simp: euclidean_representation I_def a'_def b'_def)
60462
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   434
  qed
52624
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   435
  then show ?thesis by (auto simp: I_def)
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   436
qed
8a7b59a81088 tuned proofs;
wenzelm
parents: 52141
diff changeset
   437
66154
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   438
corollary open_countable_Union_open_box:
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   439
  fixes S :: "'a :: euclidean_space set"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   440
  assumes "open S"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   441
  obtains \<D> where "countable \<D>" "\<D> \<subseteq> Pow S" "\<And>X. X \<in> \<D> \<Longrightarrow> \<exists>a b. X = box a b" "\<Union>\<D> = S"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   442
proof -
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   443
  let ?a = "\<lambda>f. (\<Sum>(i::'a)\<in>Basis. fst (f i) *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   444
  let ?b = "\<lambda>f. (\<Sum>(i::'a)\<in>Basis. snd (f i) *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   445
  let ?I = "{f\<in>Basis \<rightarrow>\<^sub>E \<rat> \<times> \<rat>. box (?a f) (?b f) \<subseteq> S}"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   446
  let ?\<D> = "(\<lambda>f. box (?a f) (?b f)) ` ?I"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   447
  show ?thesis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   448
  proof
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   449
    have "countable ?I"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   450
      by (simp add: countable_PiE countable_rat)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   451
    then show "countable ?\<D>"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   452
      by blast
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   453
    show "\<Union>?\<D> = S"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   454
      using open_UNION_box [OF assms] by metis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   455
  qed auto
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   456
qed
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   457
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   458
lemma rational_cboxes:
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   459
  fixes x :: "'a::euclidean_space"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   460
  assumes "e > 0"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   461
  shows "\<exists>a b. (\<forall>i\<in>Basis. a \<bullet> i \<in> \<rat> \<and> b \<bullet> i \<in> \<rat>) \<and> x \<in> cbox a b \<and> cbox a b \<subseteq> ball x e"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   462
proof -
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   463
  define e' where "e' = e / (2 * sqrt (real (DIM ('a))))"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   464
  then have e: "e' > 0"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   465
    using assms by auto
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   466
  have "\<exists>y. y \<in> \<rat> \<and> y < x \<bullet> i \<and> x \<bullet> i - y < e'" for i
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   467
    using Rats_dense_in_real[of "x \<bullet> i - e'" "x \<bullet> i"] e by force
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   468
  then obtain a where
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   469
    a: "\<forall>u. a u \<in> \<rat> \<and> a u < x \<bullet> u \<and> x \<bullet> u - a u < e'" by metis
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   470
  have "\<exists>y. y \<in> \<rat> \<and> x \<bullet> i < y \<and> y - x \<bullet> i < e'" for i
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   471
    using Rats_dense_in_real[of "x \<bullet> i" "x \<bullet> i + e'"] e by force
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   472
  then obtain b where
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   473
    b: "\<forall>u. b u \<in> \<rat> \<and> x \<bullet> u < b u \<and> b u - x \<bullet> u < e'" by metis
66154
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   474
  let ?a = "\<Sum>i\<in>Basis. a i *\<^sub>R i" and ?b = "\<Sum>i\<in>Basis. b i *\<^sub>R i"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   475
  show ?thesis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   476
  proof (rule exI[of _ ?a], rule exI[of _ ?b], safe)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   477
    fix y :: 'a
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   478
    assume *: "y \<in> cbox ?a ?b"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   479
    have "dist x y = sqrt (\<Sum>i\<in>Basis. (dist (x \<bullet> i) (y \<bullet> i))\<^sup>2)"
67155
9e5b05d54f9d canonical name
nipkow
parents: 66939
diff changeset
   480
      unfolding L2_set_def[symmetric] by (rule euclidean_dist_l2)
66154
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   481
    also have "\<dots> < sqrt (\<Sum>(i::'a)\<in>Basis. e^2 / real (DIM('a)))"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   482
    proof (rule real_sqrt_less_mono, rule sum_strict_mono)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   483
      fix i :: "'a"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   484
      assume i: "i \<in> Basis"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   485
      have "a i \<le> y\<bullet>i \<and> y\<bullet>i \<le> b i"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   486
        using * i by (auto simp: cbox_def)
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   487
      moreover have "a i < x\<bullet>i" "x\<bullet>i - a i < e'" "x\<bullet>i < b i" "b i - x\<bullet>i < e'"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   488
        using a b by auto
66154
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   489
      ultimately have "\<bar>x\<bullet>i - y\<bullet>i\<bar> < 2 * e'"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   490
        by auto
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   491
      then have "dist (x \<bullet> i) (y \<bullet> i) < e/sqrt (real (DIM('a)))"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   492
        unfolding e'_def by (auto simp: dist_real_def)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   493
      then have "(dist (x \<bullet> i) (y \<bullet> i))\<^sup>2 < (e/sqrt (real (DIM('a))))\<^sup>2"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   494
        by (rule power_strict_mono) auto
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   495
      then show "(dist (x \<bullet> i) (y \<bullet> i))\<^sup>2 < e\<^sup>2 / real DIM('a)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   496
        by (simp add: power_divide)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   497
    qed auto
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   498
    also have "\<dots> = e"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   499
      using \<open>0 < e\<close> by simp
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   500
    finally show "y \<in> ball x e"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   501
      by (auto simp: ball_def)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   502
  next
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   503
    show "x \<in> cbox (\<Sum>i\<in>Basis. a i *\<^sub>R i) (\<Sum>i\<in>Basis. b i *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   504
      using a b less_imp_le by (auto simp: cbox_def)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   505
  qed (use a b cbox_def in auto)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   506
qed
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   507
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   508
lemma open_UNION_cbox:
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   509
  fixes M :: "'a::euclidean_space set"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   510
  assumes "open M"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   511
  defines "a' \<equiv> \<lambda>f. (\<Sum>(i::'a)\<in>Basis. fst (f i) *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   512
  defines "b' \<equiv> \<lambda>f. (\<Sum>(i::'a)\<in>Basis. snd (f i) *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   513
  defines "I \<equiv> {f\<in>Basis \<rightarrow>\<^sub>E \<rat> \<times> \<rat>. cbox (a' f) (b' f) \<subseteq> M}"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   514
  shows "M = (\<Union>f\<in>I. cbox (a' f) (b' f))"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   515
proof -
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   516
  have "x \<in> (\<Union>f\<in>I. cbox (a' f) (b' f))" if "x \<in> M" for x
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   517
  proof -
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   518
    obtain e where e: "e > 0" "ball x e \<subseteq> M"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   519
      using openE[OF \<open>open M\<close> \<open>x \<in> M\<close>] by auto
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   520
    moreover obtain a b where ab: "x \<in> cbox a b" "\<forall>i \<in> Basis. a \<bullet> i \<in> \<rat>"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   521
                                  "\<forall>i \<in> Basis. b \<bullet> i \<in> \<rat>" "cbox a b \<subseteq> ball x e"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   522
      using rational_cboxes[OF e(1)] by metis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   523
    ultimately show ?thesis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   524
       by (intro UN_I[of "\<lambda>i\<in>Basis. (a \<bullet> i, b \<bullet> i)"])
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   525
          (auto simp: euclidean_representation I_def a'_def b'_def)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   526
  qed
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   527
  then show ?thesis by (auto simp: I_def)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   528
qed
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   529
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   530
corollary open_countable_Union_open_cbox:
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   531
  fixes S :: "'a :: euclidean_space set"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   532
  assumes "open S"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   533
  obtains \<D> where "countable \<D>" "\<D> \<subseteq> Pow S" "\<And>X. X \<in> \<D> \<Longrightarrow> \<exists>a b. X = cbox a b" "\<Union>\<D> = S"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   534
proof -
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   535
  let ?a = "\<lambda>f. (\<Sum>(i::'a)\<in>Basis. fst (f i) *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   536
  let ?b = "\<lambda>f. (\<Sum>(i::'a)\<in>Basis. snd (f i) *\<^sub>R i)"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   537
  let ?I = "{f\<in>Basis \<rightarrow>\<^sub>E \<rat> \<times> \<rat>. cbox (?a f) (?b f) \<subseteq> S}"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   538
  let ?\<D> = "(\<lambda>f. cbox (?a f) (?b f)) ` ?I"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   539
  show ?thesis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   540
  proof
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   541
    have "countable ?I"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   542
      by (simp add: countable_PiE countable_rat)
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   543
    then show "countable ?\<D>"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   544
      by blast
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   545
    show "\<Union>?\<D> = S"
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   546
      using open_UNION_cbox [OF assms] by metis
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   547
  qed auto
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   548
qed
bc5e6461f759 Tidying up integration theory and some new theorems
paulson <lp15@cam.ac.uk>
parents: 66112
diff changeset
   549
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   550
lemma box_eq_empty:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   551
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   552
  shows "(box a b = {} \<longleftrightarrow> (\<exists>i\<in>Basis. b\<bullet>i \<le> a\<bullet>i))" (is ?th1)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   553
    and "(cbox a b = {} \<longleftrightarrow> (\<exists>i\<in>Basis. b\<bullet>i < a\<bullet>i))" (is ?th2)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   554
proof -
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   555
  have False if "i \<in> Basis" and "b\<bullet>i \<le> a\<bullet>i" and "x \<in> box a b" for i x
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   556
    by (smt (verit, ccfv_SIG) mem_box(1) that)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   557
  moreover
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   558
  { assume as: "\<forall>i\<in>Basis. \<not> (b\<bullet>i \<le> a\<bullet>i)"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   559
    let ?x = "(1/2) *\<^sub>R (a + b)"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   560
    { fix i :: 'a
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   561
      assume i: "i \<in> Basis"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   562
      have "a\<bullet>i < b\<bullet>i"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   563
        using as i by fastforce
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   564
      then have "a\<bullet>i < ((1/2) *\<^sub>R (a+b)) \<bullet> i" "((1/2) *\<^sub>R (a+b)) \<bullet> i < b\<bullet>i"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   565
        by (auto simp: inner_add_left)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   566
    }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   567
    then have "box a b \<noteq> {}"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   568
      by (metis (no_types, opaque_lifting) emptyE mem_box(1))
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   569
  }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   570
  ultimately show ?th1 by blast
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   571
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   572
  have False if "i\<in>Basis" and "b\<bullet>i < a\<bullet>i" and "x \<in> cbox a b" for i x
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   573
    using mem_box(2) that by force
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   574
  moreover
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   575
  have "cbox a b \<noteq> {}" if "\<forall>i\<in>Basis. \<not> (b\<bullet>i < a\<bullet>i)"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   576
    by (metis emptyE linorder_linear mem_box(2) order.strict_iff_not that)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   577
  ultimately show ?th2 by blast
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   578
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   579
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   580
lemma box_ne_empty:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   581
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   582
  shows "cbox a b \<noteq> {} \<longleftrightarrow> (\<forall>i\<in>Basis. a\<bullet>i \<le> b\<bullet>i)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   583
  and "box a b \<noteq> {} \<longleftrightarrow> (\<forall>i\<in>Basis. a\<bullet>i < b\<bullet>i)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   584
  unfolding box_eq_empty[of a b] by fastforce+
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   585
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   586
lemma
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   587
  fixes a :: "'a::euclidean_space"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   588
  shows cbox_idem [simp]: "cbox a a = {a}"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   589
    and box_idem [simp]: "box a a = {}"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   590
  unfolding set_eq_iff mem_box eq_iff [symmetric] using euclidean_eq_iff by fastforce+
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   591
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   592
lemma subset_box_imp:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   593
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   594
  shows "(\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i) \<Longrightarrow> cbox c d \<subseteq> cbox a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   595
    and "(\<forall>i\<in>Basis. a\<bullet>i < c\<bullet>i \<and> d\<bullet>i < b\<bullet>i) \<Longrightarrow> cbox c d \<subseteq> box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   596
    and "(\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i) \<Longrightarrow> box c d \<subseteq> cbox a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   597
     and "(\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i) \<Longrightarrow> box c d \<subseteq> box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   598
  unfolding subset_eq[unfolded Ball_def] unfolding mem_box
58757
7f4924f23158 tuned whitespace;
wenzelm
parents: 58184
diff changeset
   599
  by (best intro: order_trans less_le_trans le_less_trans less_imp_le)+
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   600
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   601
lemma box_subset_cbox:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   602
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   603
  shows "box a b \<subseteq> cbox a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   604
  unfolding subset_eq [unfolded Ball_def] mem_box
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   605
  by (fast intro: less_imp_le)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   606
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   607
lemma subset_box:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   608
  fixes a :: "'a::euclidean_space"
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   609
  shows "cbox c d \<subseteq> cbox a b \<longleftrightarrow> (\<forall>i\<in>Basis. c\<bullet>i \<le> d\<bullet>i) \<longrightarrow> (\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i)" (is ?th1)
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   610
    and "cbox c d \<subseteq> box a b \<longleftrightarrow> (\<forall>i\<in>Basis. c\<bullet>i \<le> d\<bullet>i) \<longrightarrow> (\<forall>i\<in>Basis. a\<bullet>i < c\<bullet>i \<and> d\<bullet>i < b\<bullet>i)" (is ?th2)
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   611
    and "box c d \<subseteq> cbox a b \<longleftrightarrow> (\<forall>i\<in>Basis. c\<bullet>i < d\<bullet>i) \<longrightarrow> (\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i)" (is ?th3)
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   612
    and "box c d \<subseteq> box a b \<longleftrightarrow> (\<forall>i\<in>Basis. c\<bullet>i < d\<bullet>i) \<longrightarrow> (\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i)" (is ?th4)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   613
proof -
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   614
  let ?lesscd = "\<forall>i\<in>Basis. c\<bullet>i < d\<bullet>i"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   615
  let ?lerhs = "\<forall>i\<in>Basis. a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   616
  show ?th1 ?th2
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   617
    by (fastforce simp: mem_box)+
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   618
  have acdb: "a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   619
    if i: "i \<in> Basis" and box: "box c d \<subseteq> cbox a b" and cd: "\<And>i. i \<in> Basis \<Longrightarrow> c\<bullet>i < d\<bullet>i" for i
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   620
  proof -
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   621
    have "box c d \<noteq> {}"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   622
      using that
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   623
      unfolding box_eq_empty by force
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   624
    { let ?x = "(\<Sum>j\<in>Basis. (if j=i then ((min (a\<bullet>j) (d\<bullet>j))+c\<bullet>j)/2 else (c\<bullet>j+d\<bullet>j)/2) *\<^sub>R j)::'a"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   625
      assume *: "a\<bullet>i > c\<bullet>i"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   626
      then have "c \<bullet> j < ?x \<bullet> j \<and> ?x \<bullet> j < d \<bullet> j" if "j \<in> Basis" for j
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   627
        using cd that by (fastforce simp add: i *)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   628
      then have "?x \<in> box c d"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   629
        unfolding mem_box by auto
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   630
      moreover have "?x \<notin> cbox a b"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   631
        using i cd * by (force simp: mem_box)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   632
      ultimately have False using box by auto
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   633
    }
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   634
    then have "a\<bullet>i \<le> c\<bullet>i" by force
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   635
    moreover
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   636
    { let ?x = "(\<Sum>j\<in>Basis. (if j=i then ((max (b\<bullet>j) (c\<bullet>j))+d\<bullet>j)/2 else (c\<bullet>j+d\<bullet>j)/2) *\<^sub>R j)::'a"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   637
      assume *: "b\<bullet>i < d\<bullet>i"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   638
      then have "d \<bullet> j > ?x \<bullet> j \<and> ?x \<bullet> j > c \<bullet> j" if "j \<in> Basis" for j
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   639
        using cd that by (fastforce simp add: i *)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   640
      then have "?x \<in> box c d"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   641
        unfolding mem_box by auto
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   642
      moreover have "?x \<notin> cbox a b"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   643
        using i cd * by (force simp: mem_box)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   644
      ultimately have False using box by auto
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   645
    }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   646
    then have "b\<bullet>i \<ge> d\<bullet>i" by (rule ccontr) auto
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   647
    ultimately show ?thesis by auto
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   648
  qed
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   649
  show ?th3
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   650
    using acdb by (fastforce simp add: mem_box)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   651
  have acdb': "a\<bullet>i \<le> c\<bullet>i \<and> d\<bullet>i \<le> b\<bullet>i"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   652
    if "i \<in> Basis" "box c d \<subseteq> box a b" "\<And>i. i \<in> Basis \<Longrightarrow> c\<bullet>i < d\<bullet>i" for i
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   653
      using box_subset_cbox[of a b] that acdb by auto
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   654
  show ?th4
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   655
    using acdb' by (fastforce simp add: mem_box)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   656
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   657
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   658
lemma eq_cbox: "cbox a b = cbox c d \<longleftrightarrow> cbox a b = {} \<and> cbox c d = {} \<or> a = c \<and> b = d"
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   659
      (is "?lhs = ?rhs")
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   660
proof
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   661
  assume ?lhs
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   662
  then have "cbox a b \<subseteq> cbox c d" "cbox c d \<subseteq> cbox a b"
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   663
    by auto
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   664
  then show ?rhs
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
   665
    by (force simp: subset_box box_eq_empty intro: antisym euclidean_eqI)
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   666
qed auto
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   667
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   668
lemma eq_cbox_box [simp]: "cbox a b = box c d \<longleftrightarrow> cbox a b = {} \<and> box c d = {}"
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   669
  (is "?lhs \<longleftrightarrow> ?rhs")
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   670
proof
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   671
  assume L: ?lhs
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   672
  then have "cbox a b \<subseteq> box c d" "box c d \<subseteq> cbox a b"
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   673
    by auto
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   674
  with L subset_box show ?rhs
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   675
    by (smt (verit) SOME_Basis box_ne_empty(1))
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   676
qed force
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   677
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   678
lemma eq_box_cbox [simp]: "box a b = cbox c d \<longleftrightarrow> box a b = {} \<and> cbox c d = {}"
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   679
  by (metis eq_cbox_box)
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   680
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   681
lemma eq_box: "box a b = box c d \<longleftrightarrow> box a b = {} \<and> box c d = {} \<or> a = c \<and> b = d"
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   682
  (is "?lhs \<longleftrightarrow> ?rhs")
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   683
proof
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   684
  assume L: ?lhs
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   685
  then have "box a b \<subseteq> box c d" "box c d \<subseteq> box a b"
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   686
    by auto
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   687
  then show ?rhs
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   688
    unfolding subset_box by (smt (verit) box_ne_empty(2) euclidean_eq_iff)+
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
   689
qed force
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   690
66466
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   691
lemma subset_box_complex:
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
   692
   "cbox a b \<subseteq> cbox c d \<longleftrightarrow>
66466
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   693
      (Re a \<le> Re b \<and> Im a \<le> Im b) \<longrightarrow> Re a \<ge> Re c \<and> Im a \<ge> Im c \<and> Re b \<le> Re d \<and> Im b \<le> Im d"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
   694
   "cbox a b \<subseteq> box c d \<longleftrightarrow>
66466
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   695
      (Re a \<le> Re b \<and> Im a \<le> Im b) \<longrightarrow> Re a > Re c \<and> Im a > Im c \<and> Re b < Re d \<and> Im b < Im d"
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   696
   "box a b \<subseteq> cbox c d \<longleftrightarrow>
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   697
      (Re a < Re b \<and> Im a < Im b) \<longrightarrow> Re a \<ge> Re c \<and> Im a \<ge> Im c \<and> Re b \<le> Re d \<and> Im b \<le> Im d"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
   698
   "box a b \<subseteq> box c d \<longleftrightarrow>
66466
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   699
      (Re a < Re b \<and> Im a < Im b) \<longrightarrow> Re a \<ge> Re c \<and> Im a \<ge> Im c \<and> Re b \<le> Re d \<and> Im b \<le> Im d"
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   700
  by (subst subset_box; force simp: Basis_complex_def)+
aec5d9c88d69 More lemmas for HOL-Analysis
Manuel Eberl <eberlm@in.tum.de>
parents: 66453
diff changeset
   701
71029
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   702
lemma in_cbox_complex_iff:
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   703
  "x \<in> cbox a b \<longleftrightarrow> Re x \<in> {Re a..Re b} \<and> Im x \<in> {Im a..Im b}"
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   704
  by (cases x; cases a; cases b) (auto simp: cbox_Complex_eq)
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   705
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   706
lemma cbox_complex_of_real: "cbox (complex_of_real x) (complex_of_real y) = complex_of_real ` {x..y}"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   707
proof -
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   708
  have "(x \<le> Re z \<and> Re z \<le> y \<and> Im z = 0) = (z \<in> complex_of_real ` {x..y})" for z
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   709
    by (cases z) (simp add: complex_eq_cancel_iff2 image_iff)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   710
  then show ?thesis
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   711
    by (auto simp: in_cbox_complex_iff)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   712
qed
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   713
71029
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   714
lemma box_Complex_eq:
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   715
  "box (Complex a c) (Complex b d) = (\<lambda>(x,y). Complex x y) ` (box a b \<times> box c d)"
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   716
  by (auto simp: box_def Basis_complex_def image_iff complex_eq_iff)
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   717
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   718
lemma in_box_complex_iff:
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   719
  "x \<in> box a b \<longleftrightarrow> Re x \<in> {Re a<..<Re b} \<and> Im x \<in> {Im a<..<Im b}"
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   720
  by (cases x; cases a; cases b) (auto simp: box_Complex_eq)
934e0044e94b Moved or deleted some out of place material, also eliminating obsolete naming conventions
paulson <lp15@cam.ac.uk>
parents: 70952
diff changeset
   721
75462
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   722
lemma box_complex_of_real [simp]: "box (complex_of_real x) (complex_of_real y) = {}"
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   723
  by (auto simp: in_box_complex_iff)
7448423e5dba Renamed the misleading has_field_derivative_iff_has_vector_derivative. Inserted a number of minor lemmas
paulson <lp15@cam.ac.uk>
parents: 73932
diff changeset
   724
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
   725
lemma Int_interval:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   726
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   727
  shows "cbox a b \<inter> cbox c d =
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   728
    cbox (\<Sum>i\<in>Basis. max (a\<bullet>i) (c\<bullet>i) *\<^sub>R i) (\<Sum>i\<in>Basis. min (b\<bullet>i) (d\<bullet>i) *\<^sub>R i)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   729
  unfolding set_eq_iff and Int_iff and mem_box
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   730
  by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   731
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   732
lemma disjoint_interval:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   733
  fixes a::"'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   734
  shows "cbox a b \<inter> cbox c d = {} \<longleftrightarrow> (\<exists>i\<in>Basis. (b\<bullet>i < a\<bullet>i \<or> d\<bullet>i < c\<bullet>i \<or> b\<bullet>i < c\<bullet>i \<or> d\<bullet>i < a\<bullet>i))" (is ?th1)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   735
    and "cbox a b \<inter> box c d = {} \<longleftrightarrow> (\<exists>i\<in>Basis. (b\<bullet>i < a\<bullet>i \<or> d\<bullet>i \<le> c\<bullet>i \<or> b\<bullet>i \<le> c\<bullet>i \<or> d\<bullet>i \<le> a\<bullet>i))" (is ?th2)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   736
    and "box a b \<inter> cbox c d = {} \<longleftrightarrow> (\<exists>i\<in>Basis. (b\<bullet>i \<le> a\<bullet>i \<or> d\<bullet>i < c\<bullet>i \<or> b\<bullet>i \<le> c\<bullet>i \<or> d\<bullet>i \<le> a\<bullet>i))" (is ?th3)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   737
    and "box a b \<inter> box c d = {} \<longleftrightarrow> (\<exists>i\<in>Basis. (b\<bullet>i \<le> a\<bullet>i \<or> d\<bullet>i \<le> c\<bullet>i \<or> b\<bullet>i \<le> c\<bullet>i \<or> d\<bullet>i \<le> a\<bullet>i))" (is ?th4)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   738
proof -
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   739
  let ?z = "(\<Sum>i\<in>Basis. (((max (a\<bullet>i) (c\<bullet>i)) + (min (b\<bullet>i) (d\<bullet>i))) / 2) *\<^sub>R i)::'a"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   740
  have **: "\<And>P Q. (\<And>i :: 'a. i \<in> Basis \<Longrightarrow> Q ?z i \<Longrightarrow> P i) \<Longrightarrow>
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   741
      (\<And>i x :: 'a. i \<in> Basis \<Longrightarrow> P i \<Longrightarrow> Q x i) \<Longrightarrow> (\<forall>x. \<exists>i\<in>Basis. Q x i) \<longleftrightarrow> (\<exists>i\<in>Basis. P i)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   742
    by blast
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   743
  note * = set_eq_iff Int_iff empty_iff mem_box ball_conj_distrib[symmetric] eq_False ball_simps(10)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   744
  show ?th1 unfolding * by (intro **) auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   745
  show ?th2 unfolding * by (intro **) auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   746
  show ?th3 unfolding * by (intro **) auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   747
  show ?th4 unfolding * by (intro **) auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   748
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   749
57447
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   750
lemma UN_box_eq_UNIV: "(\<Union>i::nat. box (- (real i *\<^sub>R One)) (real i *\<^sub>R One)) = UNIV"
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   751
proof -
61942
f02b26f7d39d prefer symbols for "floor", "ceiling";
wenzelm
parents: 61915
diff changeset
   752
  have "\<bar>x \<bullet> b\<bar> < real_of_int (\<lceil>Max ((\<lambda>b. \<bar>x \<bullet> b\<bar>)`Basis)\<rceil> + 1)"
60462
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   753
    if [simp]: "b \<in> Basis" for x b :: 'a
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   754
  proof -
61942
f02b26f7d39d prefer symbols for "floor", "ceiling";
wenzelm
parents: 61915
diff changeset
   755
    have "\<bar>x \<bullet> b\<bar> \<le> real_of_int \<lceil>\<bar>x \<bullet> b\<bar>\<rceil>"
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   756
      by (rule le_of_int_ceiling)
61942
f02b26f7d39d prefer symbols for "floor", "ceiling";
wenzelm
parents: 61915
diff changeset
   757
    also have "\<dots> \<le> real_of_int \<lceil>Max ((\<lambda>b. \<bar>x \<bullet> b\<bar>)`Basis)\<rceil>"
59587
8ea7b22525cb Removed the obsolete functions "natfloor" and "natceiling"
nipkow
parents: 58877
diff changeset
   758
      by (auto intro!: ceiling_mono)
61942
f02b26f7d39d prefer symbols for "floor", "ceiling";
wenzelm
parents: 61915
diff changeset
   759
    also have "\<dots> < real_of_int (\<lceil>Max ((\<lambda>b. \<bar>x \<bullet> b\<bar>)`Basis)\<rceil> + 1)"
57447
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   760
      by simp
60462
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   761
    finally show ?thesis .
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   762
  qed
7c5e22e6b89f tuned proofs;
wenzelm
parents: 60420
diff changeset
   763
  then have "\<exists>n::nat. \<forall>b\<in>Basis. \<bar>x \<bullet> b\<bar> < real n" for x :: 'a
59587
8ea7b22525cb Removed the obsolete functions "natfloor" and "natceiling"
nipkow
parents: 58877
diff changeset
   764
    by (metis order.strict_trans reals_Archimedean2)
57447
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   765
  moreover have "\<And>x b::'a. \<And>n::nat.  \<bar>x \<bullet> b\<bar> < real n \<longleftrightarrow> - real n < x \<bullet> b \<and> x \<bullet> b < real n"
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   766
    by auto
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   767
  ultimately show ?thesis
64267
b9a1486e79be setsum -> sum
nipkow
parents: 64240
diff changeset
   768
    by (auto simp: box_def inner_sum_left inner_Basis sum.If_cases)
57447
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   769
qed
87429bdecad5 import more stuff from the CLT proof; base the lborel measure on interval_measure; remove lebesgue measure
hoelzl
parents: 57418
diff changeset
   770
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   771
lemma image_affinity_cbox: fixes m::real
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   772
  fixes a b c :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   773
  shows "(\<lambda>x. m *\<^sub>R x + c) ` cbox a b =
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   774
    (if cbox a b = {} then {}
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   775
     else (if 0 \<le> m then cbox (m *\<^sub>R a + c) (m *\<^sub>R b + c)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   776
     else cbox (m *\<^sub>R b + c) (m *\<^sub>R a + c)))"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   777
proof (cases "m = 0")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   778
  case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   779
  {
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   780
    fix x
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   781
    assume "\<forall>i\<in>Basis. x \<bullet> i \<le> c \<bullet> i" "\<forall>i\<in>Basis. c \<bullet> i \<le> x \<bullet> i"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   782
    then have "x = c"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   783
      by (simp add: dual_order.antisym euclidean_eqI)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   784
  }
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   785
  moreover have "c \<in> cbox (m *\<^sub>R a + c) (m *\<^sub>R b + c)"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   786
    unfolding True by auto
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   787
  ultimately show ?thesis using True by (auto simp: cbox_def)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   788
next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   789
  case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   790
  {
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   791
    fix y
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   792
    assume "\<forall>i\<in>Basis. a \<bullet> i \<le> y \<bullet> i" "\<forall>i\<in>Basis. y \<bullet> i \<le> b \<bullet> i" "m > 0"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   793
    then have "\<forall>i\<in>Basis. (m *\<^sub>R a + c) \<bullet> i \<le> (m *\<^sub>R y + c) \<bullet> i" 
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   794
          and "\<forall>i\<in>Basis. (m *\<^sub>R y + c) \<bullet> i \<le> (m *\<^sub>R b + c) \<bullet> i"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   795
      by (auto simp: inner_distrib)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   796
  }
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   797
  moreover
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   798
  {
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   799
    fix y
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   800
    assume "\<forall>i\<in>Basis. a \<bullet> i \<le> y \<bullet> i" "\<forall>i\<in>Basis. y \<bullet> i \<le> b \<bullet> i" "m < 0"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   801
    then have "\<forall>i\<in>Basis. (m *\<^sub>R b + c) \<bullet> i \<le> (m *\<^sub>R y + c) \<bullet> i"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   802
         and  "\<forall>i\<in>Basis. (m *\<^sub>R y + c) \<bullet> i \<le> (m *\<^sub>R a + c) \<bullet> i"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   803
      by (auto simp: mult_left_mono_neg inner_distrib)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   804
  }
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   805
  moreover
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   806
  {
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   807
    fix y
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   808
    assume "m > 0" and "\<forall>i\<in>Basis. (m *\<^sub>R a + c) \<bullet> i \<le> y \<bullet> i"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   809
      and  "\<forall>i\<in>Basis. y \<bullet> i \<le> (m *\<^sub>R b + c) \<bullet> i"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   810
    then have "y \<in> (\<lambda>x. m *\<^sub>R x + c) ` cbox a b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   811
      unfolding image_iff Bex_def mem_box
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   812
      apply (intro exI[where x="(1 / m) *\<^sub>R (y - c)"])
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   813
      apply (auto simp: pos_le_divide_eq pos_divide_le_eq mult.commute inner_distrib inner_diff_left)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   814
      done
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   815
  }
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   816
  moreover
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   817
  {
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   818
    fix y
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   819
    assume "\<forall>i\<in>Basis. (m *\<^sub>R b + c) \<bullet> i \<le> y \<bullet> i" "\<forall>i\<in>Basis. y \<bullet> i \<le> (m *\<^sub>R a + c) \<bullet> i" "m < 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   820
    then have "y \<in> (\<lambda>x. m *\<^sub>R x + c) ` cbox a b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   821
      unfolding image_iff Bex_def mem_box
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   822
      apply (intro exI[where x="(1 / m) *\<^sub>R (y - c)"])
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   823
      apply (auto simp: neg_le_divide_eq neg_divide_le_eq mult.commute inner_distrib inner_diff_left)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   824
      done
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   825
  }
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   826
  ultimately show ?thesis using False by (auto simp: cbox_def)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   827
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   828
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   829
lemma image_smult_cbox:"(\<lambda>x. m *\<^sub>R (x::_::euclidean_space)) ` cbox a b =
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   830
  (if cbox a b = {} then {} else if 0 \<le> m then cbox (m *\<^sub>R a) (m *\<^sub>R b) else cbox (m *\<^sub>R b) (m *\<^sub>R a))"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   831
  using image_affinity_cbox[of m 0 a b] by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
   832
69619
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   833
lemma swap_continuous:
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   834
  assumes "continuous_on (cbox (a,c) (b,d)) (\<lambda>(x,y). f x y)"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   835
    shows "continuous_on (cbox (c,a) (d,b)) (\<lambda>(x, y). f y x)"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   836
proof -
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   837
  have "(\<lambda>(x, y). f y x) = (\<lambda>(x, y). f x y) \<circ> prod.swap"
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   838
    by auto
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   839
  then show ?thesis
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   840
    by (metis assms continuous_on_compose continuous_on_swap swap_cbox_Pair)
69619
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   841
qed
3f7d8e05e0f2 split off Convex.thy: material that does not require Topology_Euclidean_Space
immler
parents: 69618
diff changeset
   842
77490
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   843
lemma open_contains_cbox:
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   844
  fixes x :: "'a :: euclidean_space"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   845
  assumes "open A" "x \<in> A"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   846
  obtains a b where "cbox a b \<subseteq> A" "x \<in> box a b" "\<forall>i\<in>Basis. a \<bullet> i < b \<bullet> i"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   847
proof -
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   848
  from assms obtain R where R: "R > 0" "ball x R \<subseteq> A"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   849
    by (auto simp: open_contains_ball)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   850
  define r :: real where "r = R / (2 * sqrt DIM('a))"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   851
  from \<open>R > 0\<close> have [simp]: "r > 0" by (auto simp: r_def)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   852
  define d :: 'a where "d = r *\<^sub>R Topology_Euclidean_Space.One"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   853
  have "cbox (x - d) (x + d) \<subseteq> A"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   854
  proof safe
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   855
    fix y assume y: "y \<in> cbox (x - d) (x + d)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   856
    have "dist x y = sqrt (\<Sum>i\<in>Basis. (dist (x \<bullet> i) (y \<bullet> i))\<^sup>2)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   857
      by (subst euclidean_dist_l2) (auto simp: L2_set_def)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   858
    also from y have "sqrt (\<Sum>i\<in>Basis. (dist (x \<bullet> i) (y \<bullet> i))\<^sup>2) \<le> sqrt (\<Sum>i\<in>(Basis::'a set). r\<^sup>2)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   859
      by (intro real_sqrt_le_mono sum_mono power_mono)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   860
         (auto simp: dist_norm d_def cbox_def algebra_simps)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   861
    also have "\<dots> = sqrt (DIM('a) * r\<^sup>2)" by simp
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   862
    also have "DIM('a) * r\<^sup>2 = (R / 2) ^ 2"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   863
      by (simp add: r_def power_divide)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   864
    also have "sqrt \<dots> = R / 2"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   865
      using \<open>R > 0\<close> by simp
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   866
    also from \<open>R > 0\<close> have "\<dots> < R" by simp
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   867
    finally have "y \<in> ball x R" by simp
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   868
    with R show "y \<in> A" by blast
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   869
  qed
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   870
  thus ?thesis
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   871
    using that[of "x - d" "x + d"] by (auto simp: algebra_simps d_def box_def)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   872
qed
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   873
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   874
lemma open_contains_box:
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   875
  fixes x :: "'a :: euclidean_space"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   876
  assumes "open A" "x \<in> A"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   877
  obtains a b where "box a b \<subseteq> A" "x \<in> box a b" "\<forall>i\<in>Basis. a \<bullet> i < b \<bullet> i"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   878
  by (meson assms box_subset_cbox dual_order.trans open_contains_cbox)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   879
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   880
lemma inner_image_box:
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   881
  assumes "(i :: 'a :: euclidean_space) \<in> Basis"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   882
  assumes "\<forall>i\<in>Basis. a \<bullet> i < b \<bullet> i"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   883
  shows   "(\<lambda>x. x \<bullet> i) ` box a b = {a \<bullet> i<..<b \<bullet> i}"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   884
proof safe
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   885
  fix x assume x: "x \<in> {a \<bullet> i<..<b \<bullet> i}"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   886
  let ?y = "(\<Sum>j\<in>Basis. (if i = j then x else (a + b) \<bullet> j / 2) *\<^sub>R j)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   887
  from x assms have "?y \<bullet> i \<in> (\<lambda>x. x \<bullet> i) ` box a b"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   888
    by (intro imageI) (auto simp: box_def algebra_simps)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   889
  also have "?y \<bullet> i = (\<Sum>j\<in>Basis. (if i = j then x else (a + b) \<bullet> j / 2) * (j \<bullet> i))"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   890
    by (simp add: inner_sum_left)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   891
  also have "\<dots> = (\<Sum>j\<in>Basis. if i = j then x else 0)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   892
    by (intro sum.cong) (auto simp: inner_not_same_Basis assms)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   893
  also have "\<dots> = x" using assms by simp
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   894
  finally show "x \<in> (\<lambda>x. x \<bullet> i) ` box a b"  .
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   895
qed (insert assms, auto simp: box_def)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   896
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   897
lemma inner_image_cbox:
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   898
  assumes "(i :: 'a :: euclidean_space) \<in> Basis"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   899
  assumes "\<forall>i\<in>Basis. a \<bullet> i \<le> b \<bullet> i"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   900
  shows   "(\<lambda>x. x \<bullet> i) ` cbox a b = {a \<bullet> i..b \<bullet> i}"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   901
proof safe
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   902
  fix x assume x: "x \<in> {a \<bullet> i..b \<bullet> i}"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   903
  let ?y = "(\<Sum>j\<in>Basis. (if i = j then x else a \<bullet> j) *\<^sub>R j)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   904
  from x assms have "?y \<bullet> i \<in> (\<lambda>x. x \<bullet> i) ` cbox a b"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   905
    by (intro imageI) (auto simp: cbox_def)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   906
  also have "?y \<bullet> i = (\<Sum>j\<in>Basis. (if i = j then x else a \<bullet> j) * (j \<bullet> i))"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   907
    by (simp add: inner_sum_left)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   908
  also have "\<dots> = (\<Sum>j\<in>Basis. if i = j then x else 0)"
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   909
    by (intro sum.cong) (auto simp: inner_not_same_Basis assms)
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   910
  also have "\<dots> = x" using assms by simp
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   911
  finally show "x \<in> (\<lambda>x. x \<bullet> i) ` cbox a b"  .
2c86ea8961b5 Some new lemmas. Some tidying up
paulson <lp15@cam.ac.uk>
parents: 76836
diff changeset
   912
qed (insert assms, auto simp: cbox_def)
69516
09bb8f470959 most of Topology_Euclidean_Space (now Elementary_Topology) requires fewer dependencies
immler
parents: 69508
diff changeset
   913
69508
2a4c8a2a3f8e tuned headers; ~ -> \<not>
nipkow
parents: 69325
diff changeset
   914
subsection \<open>General Intervals\<close>
67962
0acdcd8f4ba1 a first shot at tagging for HOL-Analysis manual
immler
parents: 67727
diff changeset
   915
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
   916
definition\<^marker>\<open>tag important\<close> "is_interval (s::('a::euclidean_space) set) \<longleftrightarrow>
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   917
  (\<forall>a\<in>s. \<forall>b\<in>s. \<forall>x. (\<forall>i\<in>Basis. ((a\<bullet>i \<le> x\<bullet>i \<and> x\<bullet>i \<le> b\<bullet>i) \<or> (b\<bullet>i \<le> x\<bullet>i \<and> x\<bullet>i \<le> a\<bullet>i))) \<longrightarrow> x \<in> s)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   918
67685
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   919
lemma is_interval_1:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   920
  "is_interval (s::real set) \<longleftrightarrow> (\<forall>a\<in>s. \<forall>b\<in>s. \<forall> x. a \<le> x \<and> x \<le> b \<longrightarrow> x \<in> s)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   921
  unfolding is_interval_def by auto
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   922
70019
095dce9892e8 A few results in Algebra, and bits for Analysis
paulson <lp15@cam.ac.uk>
parents: 69922
diff changeset
   923
lemma is_interval_Int: "is_interval X \<Longrightarrow> is_interval Y \<Longrightarrow> is_interval (X \<inter> Y)"
67685
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   924
  unfolding is_interval_def
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   925
  by blast
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
   926
66089
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
   927
lemma is_interval_cbox [simp]: "is_interval (cbox a (b::'a::euclidean_space))" (is ?th1)
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
   928
  and is_interval_box [simp]: "is_interval (box a b)" (is ?th2)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   929
  unfolding is_interval_def mem_box Ball_def atLeastAtMost_iff
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   930
  by (meson order_trans le_less_trans less_le_trans less_trans)+
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   931
61609
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   932
lemma is_interval_empty [iff]: "is_interval {}"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   933
  unfolding is_interval_def  by simp
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   934
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   935
lemma is_interval_univ [iff]: "is_interval UNIV"
77b453bd616f Coercion "real" now has type nat => real only and is no longer overloaded. Type class "real_of" is gone. Many duplicate theorems removed.
paulson <lp15@cam.ac.uk>
parents: 61552
diff changeset
   936
  unfolding is_interval_def  by simp
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   937
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   938
lemma mem_is_intervalI:
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   939
  assumes "is_interval S"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   940
    and "a \<in> S" "b \<in> S"
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   941
    and "\<And>i. i \<in> Basis \<Longrightarrow> a \<bullet> i \<le> x \<bullet> i \<and> x \<bullet> i \<le> b \<bullet> i \<or> b \<bullet> i \<le> x \<bullet> i \<and> x \<bullet> i \<le> a \<bullet> i"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   942
  shows "x \<in> S"
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   943
  using assms is_interval_def by force
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   944
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   945
lemma interval_subst:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   946
  fixes S::"'a::euclidean_space set"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   947
  assumes "is_interval S"
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   948
    and "x \<in> S" "y j \<in> S"
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   949
    and "j \<in> Basis"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   950
  shows "(\<Sum>i\<in>Basis. (if i = j then y i \<bullet> i else x \<bullet> i) *\<^sub>R i) \<in> S"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   951
  by (rule mem_is_intervalI[OF assms(1,2)]) (auto simp: assms)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   952
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   953
lemma mem_box_componentwiseI:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   954
  fixes S::"'a::euclidean_space set"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   955
  assumes "is_interval S"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   956
  assumes "\<And>i. i \<in> Basis \<Longrightarrow> x \<bullet> i \<in> ((\<lambda>x. x \<bullet> i) ` S)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   957
  shows "x \<in> S"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   958
proof -
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   959
  from assms have "\<forall>i \<in> Basis. \<exists>s \<in> S. x \<bullet> i = s \<bullet> i"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   960
    by auto
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   961
  with finite_Basis obtain s and bs::"'a list"
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   962
    where s: "\<And>i. i \<in> Basis \<Longrightarrow> x \<bullet> i = s i \<bullet> i" "\<And>i. i \<in> Basis \<Longrightarrow> s i \<in> S"
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   963
      and bs: "set bs = Basis" "distinct bs"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   964
    by (metis finite_distinct_list)
64539
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   965
  from nonempty_Basis s obtain j where j: "j \<in> Basis" "s j \<in> S"
a868c83aa66e misc tuning and modernization;
wenzelm
parents: 64394
diff changeset
   966
    by blast
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 63007
diff changeset
   967
  define y where
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 63007
diff changeset
   968
    "y = rec_list (s j) (\<lambda>j _ Y. (\<Sum>i\<in>Basis. (if i = j then s i \<bullet> i else Y \<bullet> i) *\<^sub>R i))"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   969
  have "x = (\<Sum>i\<in>Basis. (if i \<in> set bs then s i \<bullet> i else s j \<bullet> i) *\<^sub>R i)"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
   970
    using bs by (auto simp: s(1)[symmetric] euclidean_representation)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   971
  also have [symmetric]: "y bs = \<dots>"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   972
    using bs(2) bs(1)[THEN equalityD1]
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   973
    by (induct bs) (auto simp: y_def euclidean_representation intro!: euclidean_eqI[where 'a='a])
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   974
  also have "y bs \<in> S"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   975
    using bs(1)[THEN equalityD1]
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   976
  proof (induction bs)
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   977
    case Nil
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   978
    then show ?case
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   979
      by (simp add: j y_def)
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   980
  next
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   981
    case (Cons a bs)
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   982
    then show ?case
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   983
      using interval_subst[OF assms(1)] s by (simp add: y_def)
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
   984
  qed
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   985
  finally show ?thesis .
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   986
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
   987
63007
aa894a49f77d new theorems about convex hulls, etc.; also, renamed some theorems
paulson <lp15@cam.ac.uk>
parents: 62948
diff changeset
   988
lemma cbox01_nonempty [simp]: "cbox 0 One \<noteq> {}"
64267
b9a1486e79be setsum -> sum
nipkow
parents: 64240
diff changeset
   989
  by (simp add: box_ne_empty inner_Basis inner_sum_left sum_nonneg)
63007
aa894a49f77d new theorems about convex hulls, etc.; also, renamed some theorems
paulson <lp15@cam.ac.uk>
parents: 62948
diff changeset
   990
aa894a49f77d new theorems about convex hulls, etc.; also, renamed some theorems
paulson <lp15@cam.ac.uk>
parents: 62948
diff changeset
   991
lemma box01_nonempty [simp]: "box 0 One \<noteq> {}"
66089
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
   992
  by (simp add: box_ne_empty inner_Basis inner_sum_left)
63075
60a42a4166af lemmas about dimension, hyperplanes, span, etc.
paulson <lp15@cam.ac.uk>
parents: 63040
diff changeset
   993
64773
223b2ebdda79 Many new theorems, and more tidying
paulson <lp15@cam.ac.uk>
parents: 64758
diff changeset
   994
lemma empty_as_interval: "{} = cbox One (0::'a::euclidean_space)"
223b2ebdda79 Many new theorems, and more tidying
paulson <lp15@cam.ac.uk>
parents: 64758
diff changeset
   995
  using nonempty_Basis box01_nonempty box_eq_empty(1) box_ne_empty(1) by blast
223b2ebdda79 Many new theorems, and more tidying
paulson <lp15@cam.ac.uk>
parents: 64758
diff changeset
   996
66089
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
   997
lemma interval_subset_is_interval:
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
   998
  assumes "is_interval S"
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
   999
  shows "cbox a b \<subseteq> S \<longleftrightarrow> cbox a b = {} \<or> a \<in> S \<and> b \<in> S" (is "?lhs = ?rhs")
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1000
proof
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1001
  assume ?lhs
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1002
  then show ?rhs  using box_ne_empty(1) mem_box(2) by fastforce
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1003
next
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1004
  assume ?rhs
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1005
  have "cbox a b \<subseteq> S" if "a \<in> S" "b \<in> S"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1006
    using assms that 
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1007
    by (force simp: mem_box intro: mem_is_intervalI)
66089
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1008
  with \<open>?rhs\<close> show ?lhs
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1009
    by blast
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1010
qed
def95e0bc529 Some new material. SIMPRULE STATUS for sum/prod.delta rules!
paulson <lp15@cam.ac.uk>
parents: 65587
diff changeset
  1011
67685
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1012
lemma is_real_interval_union:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1013
  "is_interval (X \<union> Y)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1014
  if X: "is_interval X" and Y: "is_interval Y" and I: "(X \<noteq> {} \<Longrightarrow> Y \<noteq> {} \<Longrightarrow> X \<inter> Y \<noteq> {})"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1015
  for X Y::"real set"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1016
proof -
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1017
  consider "X \<noteq> {}" "Y \<noteq> {}" | "X = {}" | "Y = {}" by blast
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1018
  then show ?thesis
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1019
  proof cases
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1020
    case 1
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1021
    then obtain r where "r \<in> X \<or> X \<inter> Y = {}" "r \<in> Y \<or> X \<inter> Y = {}"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1022
      by blast
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1023
    then show ?thesis
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1024
      using I 1 X Y unfolding is_interval_1
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1025
      by (metis (full_types) Un_iff le_cases)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1026
  qed (use that in auto)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1027
qed
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1028
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1029
lemma is_interval_translationI:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1030
  assumes "is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1031
  shows "is_interval ((+) x ` X)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1032
  unfolding is_interval_def
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1033
proof safe
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1034
  fix b d e
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1035
  assume "b \<in> X" "d \<in> X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1036
    "\<forall>i\<in>Basis. (x + b) \<bullet> i \<le> e \<bullet> i \<and> e \<bullet> i \<le> (x + d) \<bullet> i \<or>
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1037
       (x + d) \<bullet> i \<le> e \<bullet> i \<and> e \<bullet> i \<le> (x + b) \<bullet> i"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1038
  hence "e - x \<in> X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1039
    by (intro mem_is_intervalI[OF assms \<open>b \<in> X\<close> \<open>d \<in> X\<close>, of "e - x"])
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1040
      (auto simp: algebra_simps)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1041
  thus "e \<in> (+) x ` X" by force
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1042
qed
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1043
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1044
lemma is_interval_uminusI:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1045
  assumes "is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1046
  shows "is_interval (uminus ` X)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1047
  unfolding is_interval_def
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1048
proof safe
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1049
  fix b d e
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1050
  assume "b \<in> X" "d \<in> X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1051
    "\<forall>i\<in>Basis. (- b) \<bullet> i \<le> e \<bullet> i \<and> e \<bullet> i \<le> (- d) \<bullet> i \<or>
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1052
       (- d) \<bullet> i \<le> e \<bullet> i \<and> e \<bullet> i \<le> (- b) \<bullet> i"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1053
  hence "- e \<in> X"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1054
    by (smt (verit, ccfv_threshold) assms inner_minus_left mem_is_intervalI)
67685
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1055
  thus "e \<in> uminus ` X" by force
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1056
qed
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1057
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1058
lemma is_interval_uminus[simp]: "is_interval (uminus ` x) = is_interval x"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1059
  using is_interval_uminusI[of x] is_interval_uminusI[of "uminus ` x"]
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1060
  by (auto simp: image_image)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1061
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1062
lemma is_interval_neg_translationI:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1063
  assumes "is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1064
  shows "is_interval ((-) x ` X)"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1065
proof -
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1066
  have "(-) x ` X = (+) x ` uminus ` X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1067
    by (force simp: algebra_simps)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1068
  also have "is_interval \<dots>"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1069
    by (metis is_interval_uminusI is_interval_translationI assms)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1070
  finally show ?thesis .
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1071
qed
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1072
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1073
lemma is_interval_translation[simp]:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1074
  "is_interval ((+) x ` X) = is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1075
  using is_interval_neg_translationI[of "(+) x ` X" x]
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1076
  by (auto intro!: is_interval_translationI simp: image_image)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1077
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1078
lemma is_interval_minus_translation[simp]:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1079
  shows "is_interval ((-) x ` X) = is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1080
proof -
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1081
  have "(-) x ` X = (+) x ` uminus ` X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1082
    by (force simp: algebra_simps)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1083
  also have "is_interval \<dots> = is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1084
    by simp
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1085
  finally show ?thesis .
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1086
qed
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1087
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1088
lemma is_interval_minus_translation'[simp]:
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1089
  shows "is_interval ((\<lambda>x. x - c) ` X) = is_interval X"
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1090
  using is_interval_translation[of "-c" X]
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1091
  by (metis image_cong uminus_add_conv_diff)
bdff8bf0a75b moved theorems from AFP/Affine_Arithmetic and AFP/Ordinary_Differential_Equations
immler
parents: 67613
diff changeset
  1092
71028
c2465b429e6e Line_Segment is independent of Convex_Euclidean_Space
immler
parents: 71025
diff changeset
  1093
lemma is_interval_cball_1[intro, simp]: "is_interval (cball a b)" for a b::real
c2465b429e6e Line_Segment is independent of Convex_Euclidean_Space
immler
parents: 71025
diff changeset
  1094
  by (simp add: cball_eq_atLeastAtMost is_interval_def)
c2465b429e6e Line_Segment is independent of Convex_Euclidean_Space
immler
parents: 71025
diff changeset
  1095
c2465b429e6e Line_Segment is independent of Convex_Euclidean_Space
immler
parents: 71025
diff changeset
  1096
lemma is_interval_ball_real: "is_interval (ball a b)" for a b::real
c2465b429e6e Line_Segment is independent of Convex_Euclidean_Space
immler
parents: 71025
diff changeset
  1097
  by (simp add: ball_eq_greaterThanLessThan is_interval_def)
c2465b429e6e Line_Segment is independent of Convex_Euclidean_Space
immler
parents: 71025
diff changeset
  1098
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1099
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1100
subsection\<^marker>\<open>tag unimportant\<close> \<open>Bounded Projections\<close>
62127
d8e7738bd2e9 generalized proofs
immler
parents: 62101
diff changeset
  1101
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1102
lemma bounded_inner_imp_bdd_above:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1103
  assumes "bounded s"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1104
    shows "bdd_above ((\<lambda>x. x \<bullet> a) ` s)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1105
by (simp add: assms bounded_imp_bdd_above bounded_linear_image bounded_linear_inner_left)
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1106
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1107
lemma bounded_inner_imp_bdd_below:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1108
  assumes "bounded s"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1109
    shows "bdd_below ((\<lambda>x. x \<bullet> a) ` s)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1110
by (simp add: assms bounded_imp_bdd_below bounded_linear_image bounded_linear_inner_left)
44632
076a45f65e12 simplify/generalize some proofs
huffman
parents: 44628
diff changeset
  1111
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1112
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1113
subsection\<^marker>\<open>tag unimportant\<close> \<open>Structural rules for pointwise continuity\<close>
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1114
51361
21e5b6efb317 changed continuous_intros into a named theorems collection
hoelzl
parents: 51351
diff changeset
  1115
lemma continuous_infnorm[continuous_intros]:
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1116
  "continuous F f \<Longrightarrow> continuous F (\<lambda>x. infnorm (f x))"
44647
e4de7750cdeb modernize lemmas about 'continuous' and 'continuous_on';
huffman
parents: 44632
diff changeset
  1117
  unfolding continuous_def by (rule tendsto_infnorm)
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1118
51361
21e5b6efb317 changed continuous_intros into a named theorems collection
hoelzl
parents: 51351
diff changeset
  1119
lemma continuous_inner[continuous_intros]:
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1120
  assumes "continuous F f"
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1121
    and "continuous F g"
44647
e4de7750cdeb modernize lemmas about 'continuous' and 'continuous_on';
huffman
parents: 44632
diff changeset
  1122
  shows "continuous F (\<lambda>x. inner (f x) (g x))"
e4de7750cdeb modernize lemmas about 'continuous' and 'continuous_on';
huffman
parents: 44632
diff changeset
  1123
  using assms unfolding continuous_def by (rule tendsto_inner)
e4de7750cdeb modernize lemmas about 'continuous' and 'continuous_on';
huffman
parents: 44632
diff changeset
  1124
69516
09bb8f470959 most of Topology_Euclidean_Space (now Elementary_Topology) requires fewer dependencies
immler
parents: 69508
diff changeset
  1125
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1126
subsection\<^marker>\<open>tag unimportant\<close> \<open>Structural rules for setwise continuity\<close>
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1127
56371
fb9ae0727548 extend continuous_intros; remove continuous_on_intros and isCont_intros
hoelzl
parents: 56290
diff changeset
  1128
lemma continuous_on_infnorm[continuous_intros]:
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1129
  "continuous_on s f \<Longrightarrow> continuous_on s (\<lambda>x. infnorm (f x))"
44647
e4de7750cdeb modernize lemmas about 'continuous' and 'continuous_on';
huffman
parents: 44632
diff changeset
  1130
  unfolding continuous_on by (fast intro: tendsto_infnorm)
e4de7750cdeb modernize lemmas about 'continuous' and 'continuous_on';
huffman
parents: 44632
diff changeset
  1131
56371
fb9ae0727548 extend continuous_intros; remove continuous_on_intros and isCont_intros
hoelzl
parents: 56290
diff changeset
  1132
lemma continuous_on_inner[continuous_intros]:
44531
1d477a2b1572 replace some continuous_on lemmas with more general versions
huffman
parents: 44530
diff changeset
  1133
  fixes g :: "'a::topological_space \<Rightarrow> 'b::real_inner"
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1134
  assumes "continuous_on s f"
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1135
    and "continuous_on s g"
44531
1d477a2b1572 replace some continuous_on lemmas with more general versions
huffman
parents: 44530
diff changeset
  1136
  shows "continuous_on s (\<lambda>x. inner (f x) (g x))"
1d477a2b1572 replace some continuous_on lemmas with more general versions
huffman
parents: 44530
diff changeset
  1137
  using bounded_bilinear_inner assms
1d477a2b1572 replace some continuous_on lemmas with more general versions
huffman
parents: 44530
diff changeset
  1138
  by (rule bounded_bilinear.continuous_on)
1d477a2b1572 replace some continuous_on lemmas with more general versions
huffman
parents: 44530
diff changeset
  1139
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1140
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1141
subsection\<^marker>\<open>tag unimportant\<close> \<open>Openness of halfspaces.\<close>
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1142
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1143
lemma open_halfspace_lt: "open {x. inner a x < b}"
71172
nipkow
parents: 71033
diff changeset
  1144
  by (simp add: open_Collect_less continuous_on_inner)
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1145
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1146
lemma open_halfspace_gt: "open {x. inner a x > b}"
71172
nipkow
parents: 71033
diff changeset
  1147
  by (simp add: open_Collect_less continuous_on_inner)
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1148
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1149
lemma open_halfspace_component_lt: "open {x::'a::euclidean_space. x\<bullet>i < a}"
71172
nipkow
parents: 71033
diff changeset
  1150
  by (simp add: open_Collect_less continuous_on_inner)
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1151
53282
9d6e263fa921 tuned proofs;
wenzelm
parents: 53255
diff changeset
  1152
lemma open_halfspace_component_gt: "open {x::'a::euclidean_space. x\<bullet>i > a}"
71172
nipkow
parents: 71033
diff changeset
  1153
  by (simp add: open_Collect_less continuous_on_inner)
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1154
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1155
lemma eucl_less_eq_halfspaces:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1156
  fixes a :: "'a::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1157
  shows "{x. x <e a} = (\<Inter>i\<in>Basis. {x. x \<bullet> i < a \<bullet> i})"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1158
        "{x. a <e x} = (\<Inter>i\<in>Basis. {x. a \<bullet> i < x \<bullet> i})"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1159
  by (auto simp: eucl_less_def)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1160
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1161
lemma open_Collect_eucl_less[simp, intro]:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1162
  fixes a :: "'a::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1163
  shows "open {x. x <e a}" "open {x. a <e x}"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1164
  by (auto simp: eucl_less_eq_halfspaces open_halfspace_component_lt open_halfspace_component_gt)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1165
71025
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1166
subsection\<^marker>\<open>tag unimportant\<close> \<open>Closure and Interior of halfspaces and hyperplanes\<close>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1167
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1168
lemma continuous_at_inner: "continuous (at x) (inner a)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1169
  unfolding continuous_at by (intro tendsto_intros)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1170
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1171
lemma closed_halfspace_le: "closed {x. inner a x \<le> b}"
71172
nipkow
parents: 71033
diff changeset
  1172
  by (simp add: closed_Collect_le continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1173
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1174
lemma closed_halfspace_ge: "closed {x. inner a x \<ge> b}"
71172
nipkow
parents: 71033
diff changeset
  1175
  by (simp add: closed_Collect_le continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1176
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1177
lemma closed_hyperplane: "closed {x. inner a x = b}"
71172
nipkow
parents: 71033
diff changeset
  1178
  by (simp add: closed_Collect_eq continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1179
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1180
lemma closed_halfspace_component_le: "closed {x::'a::euclidean_space. x\<bullet>i \<le> a}"
71172
nipkow
parents: 71033
diff changeset
  1181
  by (simp add: closed_Collect_le continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1182
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1183
lemma closed_halfspace_component_ge: "closed {x::'a::euclidean_space. x\<bullet>i \<ge> a}"
71172
nipkow
parents: 71033
diff changeset
  1184
  by (simp add: closed_Collect_le continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1185
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1186
lemma closed_interval_left:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1187
  fixes b :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1188
  shows "closed {x::'a. \<forall>i\<in>Basis. x\<bullet>i \<le> b\<bullet>i}"
71172
nipkow
parents: 71033
diff changeset
  1189
  by (simp add: Collect_ball_eq closed_INT closed_Collect_le continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1190
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1191
lemma closed_interval_right:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1192
  fixes a :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1193
  shows "closed {x::'a. \<forall>i\<in>Basis. a\<bullet>i \<le> x\<bullet>i}"
71172
nipkow
parents: 71033
diff changeset
  1194
  by (simp add: Collect_ball_eq closed_INT closed_Collect_le continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1195
71025
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1196
lemma interior_halfspace_le [simp]:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1197
  assumes "a \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1198
    shows "interior {x. a \<bullet> x \<le> b} = {x. a \<bullet> x < b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1199
proof -
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1200
  have *: "a \<bullet> x < b" if x: "x \<in> S" and S: "S \<subseteq> {x. a \<bullet> x \<le> b}" and "open S" for S x
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1201
  proof -
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1202
    obtain e where "e>0" and e: "cball x e \<subseteq> S"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1203
      using \<open>open S\<close> open_contains_cball x by blast
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1204
    then have "x + (e / norm a) *\<^sub>R a \<in> cball x e"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1205
      by (simp add: dist_norm)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1206
    then have "x + (e / norm a) *\<^sub>R a \<in> S"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1207
      using e by blast
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1208
    then have "x + (e / norm a) *\<^sub>R a \<in> {x. a \<bullet> x \<le> b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1209
      using S by blast
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1210
    moreover have "e * (a \<bullet> a) / norm a > 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1211
      by (simp add: \<open>0 < e\<close> assms)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1212
    ultimately show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1213
      by (simp add: algebra_simps)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1214
  qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1215
  show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1216
    by (rule interior_unique) (auto simp: open_halfspace_lt *)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1217
qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1218
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1219
lemma interior_halfspace_ge [simp]:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1220
   "a \<noteq> 0 \<Longrightarrow> interior {x. a \<bullet> x \<ge> b} = {x. a \<bullet> x > b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1221
using interior_halfspace_le [of "-a" "-b"] by simp
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1222
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1223
lemma closure_halfspace_lt [simp]:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1224
  assumes "a \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1225
    shows "closure {x. a \<bullet> x < b} = {x. a \<bullet> x \<le> b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1226
proof -
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1227
  have [simp]: "-{x. a \<bullet> x < b} = {x. a \<bullet> x \<ge> b}"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1228
    by force
71025
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1229
  then show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1230
    using interior_halfspace_ge [of a b] assms
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1231
    by (force simp: closure_interior)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1232
qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1233
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1234
lemma closure_halfspace_gt [simp]:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1235
   "a \<noteq> 0 \<Longrightarrow> closure {x. a \<bullet> x > b} = {x. a \<bullet> x \<ge> b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1236
using closure_halfspace_lt [of "-a" "-b"] by simp
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1237
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1238
lemma interior_hyperplane [simp]:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1239
  assumes "a \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1240
    shows "interior {x. a \<bullet> x = b} = {}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1241
proof -
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1242
  have [simp]: "{x. a \<bullet> x = b} = {x. a \<bullet> x \<le> b} \<inter> {x. a \<bullet> x \<ge> b}"
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1243
    by force
71025
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1244
  then show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1245
    by (auto simp: assms)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1246
qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1247
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1248
lemma frontier_halfspace_le:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1249
  assumes "a \<noteq> 0 \<or> b \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1250
    shows "frontier {x. a \<bullet> x \<le> b} = {x. a \<bullet> x = b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1251
proof (cases "a = 0")
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1252
  case True with assms show ?thesis by simp
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1253
next
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1254
  case False then show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1255
    by (force simp: frontier_def closed_halfspace_le)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1256
qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1257
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1258
lemma frontier_halfspace_ge:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1259
  assumes "a \<noteq> 0 \<or> b \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1260
    shows "frontier {x. a \<bullet> x \<ge> b} = {x. a \<bullet> x = b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1261
proof (cases "a = 0")
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1262
  case True with assms show ?thesis by simp
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1263
next
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1264
  case False then show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1265
    by (force simp: frontier_def closed_halfspace_ge)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1266
qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1267
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1268
lemma frontier_halfspace_lt:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1269
  assumes "a \<noteq> 0 \<or> b \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1270
    shows "frontier {x. a \<bullet> x < b} = {x. a \<bullet> x = b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1271
proof (cases "a = 0")
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1272
  case True with assms show ?thesis by simp
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1273
next
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1274
  case False then show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1275
    by (force simp: frontier_def interior_open open_halfspace_lt)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1276
qed
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1277
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1278
lemma frontier_halfspace_gt:
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1279
  assumes "a \<noteq> 0 \<or> b \<noteq> 0"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1280
    shows "frontier {x. a \<bullet> x > b} = {x. a \<bullet> x = b}"
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1281
proof (cases "a = 0")
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1282
  case True with assms show ?thesis by simp
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1283
next
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1284
  case False then show ?thesis
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1285
    by (force simp: frontier_def interior_open open_halfspace_gt)
be8cec1abcbb reduce dependencies of Ordered_Euclidean_Space; move more general material from Cartesian_Euclidean_Space
immler
parents: 70952
diff changeset
  1286
qed
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1287
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1288
subsection\<^marker>\<open>tag unimportant\<close>\<open>Some more convenient intermediate-value theorem formulations\<close>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1289
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1290
lemma connected_ivt_hyperplane:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1291
  assumes "connected S" and xy: "x \<in> S" "y \<in> S" and b: "inner a x \<le> b" "b \<le> inner a y"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1292
  shows "\<exists>z \<in> S. inner a z = b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1293
proof (rule ccontr)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1294
  assume as:"\<not> (\<exists>z\<in>S. inner a z = b)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1295
  let ?A = "{x. inner a x < b}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1296
  let ?B = "{x. inner a x > b}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1297
  have "open ?A" "open ?B"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1298
    using open_halfspace_lt and open_halfspace_gt by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1299
  moreover have "?A \<inter> ?B = {}" by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1300
  moreover have "S \<subseteq> ?A \<union> ?B" using as by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1301
  ultimately show False
76834
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1302
    using \<open>connected S\<close> unfolding connected_def
4645ca4457db Continued proof simplifications
paulson <lp15@cam.ac.uk>
parents: 75462
diff changeset
  1303
    by (smt (verit, del_insts) as b disjoint_iff empty_iff mem_Collect_eq xy)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1304
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1305
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1306
lemma connected_ivt_component:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1307
  fixes x::"'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1308
  shows "connected S \<Longrightarrow> x \<in> S \<Longrightarrow> y \<in> S \<Longrightarrow> x\<bullet>k \<le> a \<Longrightarrow> a \<le> y\<bullet>k \<Longrightarrow> (\<exists>z\<in>S.  z\<bullet>k = a)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1309
  using connected_ivt_hyperplane[of S x y "k::'a" a]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1310
  by (auto simp: inner_commute)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1311
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1312
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1313
subsection \<open>Limit Component Bounds\<close>
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  1314
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1315
lemma Lim_component_le:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1316
  fixes f :: "'a \<Rightarrow> 'b::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1317
  assumes "(f \<longlongrightarrow> l) net"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1318
    and "\<not> (trivial_limit net)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1319
    and "eventually (\<lambda>x. f(x)\<bullet>i \<le> b) net"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1320
  shows "l\<bullet>i \<le> b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1321
  by (rule tendsto_le[OF assms(2) tendsto_const tendsto_inner[OF assms(1) tendsto_const] assms(3)])
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1322
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1323
lemma Lim_component_ge:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1324
  fixes f :: "'a \<Rightarrow> 'b::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1325
  assumes "(f \<longlongrightarrow> l) net"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1326
    and "\<not> (trivial_limit net)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1327
    and "eventually (\<lambda>x. b \<le> (f x)\<bullet>i) net"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1328
  shows "b \<le> l\<bullet>i"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1329
  by (rule tendsto_le[OF assms(2) tendsto_inner[OF assms(1) tendsto_const] tendsto_const assms(3)])
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1330
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1331
lemma Lim_component_eq:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1332
  fixes f :: "'a \<Rightarrow> 'b::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1333
  assumes net: "(f \<longlongrightarrow> l) net" "\<not> trivial_limit net"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1334
    and ev:"eventually (\<lambda>x. f(x)\<bullet>i = b) net"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1335
  shows "l\<bullet>i = b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1336
  using ev[unfolded order_eq_iff eventually_conj_iff]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1337
  using Lim_component_ge[OF net, of b i]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1338
  using Lim_component_le[OF net, of i b]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1339
  by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1340
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1341
lemma open_box[intro]: "open (box a b)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1342
proof -
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 67155
diff changeset
  1343
  have "open (\<Inter>i\<in>Basis. ((\<bullet>) i) -` {a \<bullet> i <..< b \<bullet> i})"
62533
bc25f3916a99 new material to Blochj's theorem, as well as supporting lemmas
paulson <lp15@cam.ac.uk>
parents: 62466
diff changeset
  1344
    by (auto intro!: continuous_open_vimage continuous_inner continuous_ident continuous_const)
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 67155
diff changeset
  1345
  also have "(\<Inter>i\<in>Basis. ((\<bullet>) i) -` {a \<bullet> i <..< b \<bullet> i}) = box a b"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
  1346
    by (auto simp: box_def inner_commute)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1347
  finally show ?thesis .
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1348
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1349
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1350
lemma closed_cbox[intro]:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1351
  fixes a b :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1352
  shows "closed (cbox a b)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1353
proof -
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1354
  have "closed (\<Inter>i\<in>Basis. (\<lambda>x. x\<bullet>i) -` {a\<bullet>i .. b\<bullet>i})"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1355
    by (intro closed_INT ballI continuous_closed_vimage allI
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1356
      linear_continuous_at closed_real_atLeastAtMost finite_Basis bounded_linear_inner_left)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1357
  also have "(\<Inter>i\<in>Basis. (\<lambda>x. x\<bullet>i) -` {a\<bullet>i .. b\<bullet>i}) = cbox a b"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
  1358
    by (auto simp: cbox_def)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1359
  finally show "closed (cbox a b)" .
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1360
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1361
62618
f7f2467ab854 Refactoring (moving theorems into better locations), plus a bit of new material
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
  1362
lemma interior_cbox [simp]:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1363
  fixes a b :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1364
  shows "interior (cbox a b) = box a b" (is "?L = ?R")
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1365
proof(rule subset_antisym)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1366
  show "?R \<subseteq> ?L"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1367
    using box_subset_cbox open_box
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1368
    by (rule interior_maximal)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1369
  {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1370
    fix x
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1371
    assume "x \<in> interior (cbox a b)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1372
    then obtain s where s: "open s" "x \<in> s" "s \<subseteq> cbox a b" ..
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1373
    then obtain e where "e>0" and e:"\<forall>x'. dist x' x < e \<longrightarrow> x' \<in> cbox a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1374
      unfolding open_dist and subset_eq by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1375
    {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1376
      fix i :: 'a
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1377
      assume i: "i \<in> Basis"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1378
      have "dist (x - (e / 2) *\<^sub>R i) x < e"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1379
        and "dist (x + (e / 2) *\<^sub>R i) x < e"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1380
         using norm_Basis[OF i] \<open>e>0\<close> by (auto simp: dist_norm)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1381
      then have "a \<bullet> i \<le> (x - (e / 2) *\<^sub>R i) \<bullet> i" and "(x + (e / 2) *\<^sub>R i) \<bullet> i \<le> b \<bullet> i"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1382
        using e[THEN spec[where x="x - (e/2) *\<^sub>R i"]]
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1383
          and e[THEN spec[where x="x + (e/2) *\<^sub>R i"]]
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1384
        unfolding mem_box using i by blast+
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1385
      then have "a \<bullet> i < x \<bullet> i" and "x \<bullet> i < b \<bullet> i"
60420
884f54e01427 isabelle update_cartouches;
wenzelm
parents: 60176
diff changeset
  1386
        using \<open>e>0\<close> i
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1387
        by (auto simp: inner_diff_left inner_Basis inner_add_left)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1388
    }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1389
    then have "x \<in> box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1390
      unfolding mem_box by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1391
  }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1392
  then show "?L \<subseteq> ?R" ..
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1393
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1394
63928
d81fb5b46a5c new material about topological concepts, etc
paulson <lp15@cam.ac.uk>
parents: 63881
diff changeset
  1395
lemma bounded_cbox [simp]:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1396
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1397
  shows "bounded (cbox a b)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1398
proof -
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1399
  let ?b = "\<Sum>i\<in>Basis. \<bar>a\<bullet>i\<bar> + \<bar>b\<bullet>i\<bar>"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1400
  {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1401
    fix x :: "'a"
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1402
    assume "\<And>i. i\<in>Basis \<Longrightarrow> a \<bullet> i \<le> x \<bullet> i \<and> x \<bullet> i \<le> b \<bullet> i"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1403
    then have "(\<Sum>i\<in>Basis. \<bar>x \<bullet> i\<bar>) \<le> ?b"
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1404
      by (force simp: intro!: sum_mono)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1405
    then have "norm x \<le> ?b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1406
      using norm_le_l1[of x] by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1407
  }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1408
  then show ?thesis
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1409
    unfolding cbox_def bounded_iff by force
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1410
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1411
62618
f7f2467ab854 Refactoring (moving theorems into better locations), plus a bit of new material
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
  1412
lemma bounded_box [simp]:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1413
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1414
  shows "bounded (box a b)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1415
  by (metis bounded_cbox bounded_interior interior_cbox)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1416
62618
f7f2467ab854 Refactoring (moving theorems into better locations), plus a bit of new material
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
  1417
lemma not_interval_UNIV [simp]:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1418
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1419
  shows "cbox a b \<noteq> UNIV" "box a b \<noteq> UNIV"
62618
f7f2467ab854 Refactoring (moving theorems into better locations), plus a bit of new material
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
  1420
  using bounded_box[of a b] bounded_cbox[of a b] by force+
f7f2467ab854 Refactoring (moving theorems into better locations), plus a bit of new material
paulson <lp15@cam.ac.uk>
parents: 62533
diff changeset
  1421
63945
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
  1422
lemma not_interval_UNIV2 [simp]:
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
  1423
  fixes a :: "'a::euclidean_space"
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
  1424
  shows "UNIV \<noteq> cbox a b" "UNIV \<noteq> box a b"
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
  1425
  using bounded_box[of a b] bounded_cbox[of a b] by force+
444eafb6e864 a few new theorems and a renaming
paulson <lp15@cam.ac.uk>
parents: 63938
diff changeset
  1426
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1427
lemma box_midpoint:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1428
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1429
  assumes "box a b \<noteq> {}"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1430
  shows "((1/2) *\<^sub>R (a + b)) \<in> box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1431
proof -
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1432
  have "a \<bullet> i < ((1 / 2) *\<^sub>R (a + b)) \<bullet> i \<and> ((1 / 2) *\<^sub>R (a + b)) \<bullet> i < b \<bullet> i" if "i \<in> Basis" for i
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1433
    using assms that by (auto simp: inner_add_left box_ne_empty)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1434
  then show ?thesis unfolding mem_box by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1435
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1436
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1437
lemma open_cbox_convex:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1438
  fixes x :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1439
  assumes x: "x \<in> box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1440
    and y: "y \<in> cbox a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1441
    and e: "0 < e" "e \<le> 1"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1442
  shows "(e *\<^sub>R x + (1 - e) *\<^sub>R y) \<in> box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1443
proof -
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1444
  {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1445
    fix i :: 'a
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1446
    assume i: "i \<in> Basis"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1447
    have "a \<bullet> i = e * (a \<bullet> i) + (1 - e) * (a \<bullet> i)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1448
      unfolding left_diff_distrib by simp
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1449
    also have "\<dots> < e * (x \<bullet> i) + (1 - e) * (y \<bullet> i)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1450
      by (smt (verit, best) e i mem_box mult_le_cancel_left_pos mult_left_mono x y)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1451
    finally have "a \<bullet> i < (e *\<^sub>R x + (1 - e) *\<^sub>R y) \<bullet> i"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1452
      unfolding inner_simps by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1453
    moreover
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1454
    {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1455
      have "b \<bullet> i = e * (b\<bullet>i) + (1 - e) * (b\<bullet>i)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1456
        unfolding left_diff_distrib by simp
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1457
      also have "\<dots> > e * (x \<bullet> i) + (1 - e) * (y \<bullet> i)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1458
        by (smt (verit, best) e i mem_box mult_le_cancel_left_pos mult_left_mono x y)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1459
      finally have "(e *\<^sub>R x + (1 - e) *\<^sub>R y) \<bullet> i < b \<bullet> i"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1460
        unfolding inner_simps by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1461
    }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1462
    ultimately have "a \<bullet> i < (e *\<^sub>R x + (1 - e) *\<^sub>R y) \<bullet> i \<and> (e *\<^sub>R x + (1 - e) *\<^sub>R y) \<bullet> i < b \<bullet> i"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1463
      by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1464
  }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1465
  then show ?thesis
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1466
    unfolding mem_box by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1467
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1468
63881
b746b19197bd lots of new results about topology, affine dimension etc
paulson <lp15@cam.ac.uk>
parents: 63627
diff changeset
  1469
lemma closure_cbox [simp]: "closure (cbox a b) = cbox a b"
b746b19197bd lots of new results about topology, affine dimension etc
paulson <lp15@cam.ac.uk>
parents: 63627
diff changeset
  1470
  by (simp add: closed_cbox)
b746b19197bd lots of new results about topology, affine dimension etc
paulson <lp15@cam.ac.uk>
parents: 63627
diff changeset
  1471
b746b19197bd lots of new results about topology, affine dimension etc
paulson <lp15@cam.ac.uk>
parents: 63627
diff changeset
  1472
lemma closure_box [simp]:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1473
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1474
   assumes "box a b \<noteq> {}"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1475
  shows "closure (box a b) = cbox a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1476
proof -
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1477
  have ab: "a <e b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1478
    using assms by (simp add: eucl_less_def box_ne_empty)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1479
  let ?c = "(1 / 2) *\<^sub>R (a + b)"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1480
  {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1481
    fix x
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1482
    assume as: "x \<in> cbox a b"
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 63007
diff changeset
  1483
    define f where [abs_def]: "f n = x + (inverse (real n + 1)) *\<^sub>R (?c - x)" for n
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1484
    {
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1485
      fix n
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1486
      assume fn: "f n <e b \<longrightarrow> a <e f n \<longrightarrow> f n = x" and xc: "x \<noteq> ?c"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1487
      have *: "0 < inverse (real n + 1)" "inverse (real n + 1) \<le> 1"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1488
        unfolding inverse_le_1_iff by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1489
      have "(inverse (real n + 1)) *\<^sub>R ((1 / 2) *\<^sub>R (a + b)) + (1 - inverse (real n + 1)) *\<^sub>R x =
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1490
        x + (inverse (real n + 1)) *\<^sub>R (((1 / 2) *\<^sub>R (a + b)) - x)"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
  1491
        by (auto simp: algebra_simps)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1492
      then have "f n <e b" and "a <e f n"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1493
        using open_cbox_convex[OF box_midpoint[OF assms] as *]
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1494
        unfolding f_def by (auto simp: box_def eucl_less_def)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1495
      then have False
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1496
        using fn unfolding f_def using xc by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1497
    }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1498
    moreover
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1499
    {
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1500
      have "\<exists>N::nat. \<forall>n\<ge>N. inverse (real n + 1) < \<epsilon>" if "\<epsilon> > 0" for \<epsilon>
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1501
          using reals_Archimedean [of \<epsilon>] that
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1502
          by (metis inverse_inverse_eq inverse_less_imp_less nat_le_real_less order_less_trans 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1503
                  reals_Archimedean2)
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1504
      then have "(\<lambda>n. inverse (real n + 1)) \<longlonglongrightarrow> 0"
66643
f7e38b8583a0 Correction of typos and a bit of streamlining
paulson <lp15@cam.ac.uk>
parents: 66641
diff changeset
  1505
        unfolding lim_sequentially by(auto simp: dist_norm)
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1506
      then have "f \<longlonglongrightarrow> x"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1507
        unfolding f_def
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1508
        using tendsto_add[OF tendsto_const, of "\<lambda>n. (inverse (real n + 1)) *\<^sub>R ((1 / 2) *\<^sub>R (a + b) - x)" 0 sequentially x]
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1509
        using tendsto_scaleR [OF _ tendsto_const, of "\<lambda>n. inverse (real n + 1)" 0 sequentially "((1 / 2) *\<^sub>R (a + b) - x)"]
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1510
        by auto
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1511
    }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1512
    ultimately have "x \<in> closure (box a b)"
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1513
      using as box_midpoint[OF assms]
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1514
      unfolding closure_def islimpt_sequential
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1515
      by (cases "x=?c") (auto simp: in_box_eucl_less)
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1516
  }
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1517
  then show ?thesis
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1518
    using closure_minimal[OF box_subset_cbox, of a b] by blast
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1519
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1520
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1521
lemma bounded_subset_box_symmetric:
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1522
  fixes S :: "('a::euclidean_space) set"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1523
  assumes "bounded S"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1524
  obtains a where "S \<subseteq> box (-a) a"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1525
proof -
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1526
  obtain b where "b>0" and b: "\<forall>x\<in>S. norm x \<le> b"
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1527
    using assms[unfolded bounded_pos] by auto
63040
eb4ddd18d635 eliminated old 'def';
wenzelm
parents: 63007
diff changeset
  1528
  define a :: 'a where "a = (\<Sum>i\<in>Basis. (b + 1) *\<^sub>R i)"
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1529
  have "(-a)\<bullet>i < x\<bullet>i" and "x\<bullet>i < a\<bullet>i" if "x \<in> S" and i: "i \<in> Basis" for x i
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1530
    using b Basis_le_norm[OF i, of x] that by (auto simp: a_def)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1531
  then have "S \<subseteq> box (-a) a"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1532
    by (auto simp: simp add: box_def)
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1533
  then show ?thesis ..
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1534
qed
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1535
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1536
lemma bounded_subset_cbox_symmetric:
68120
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1537
  fixes S :: "('a::euclidean_space) set"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1538
  assumes "bounded S"
2f161c6910f7 tidying more messy proofs
paulson <lp15@cam.ac.uk>
parents: 68072
diff changeset
  1539
  obtains a where "S \<subseteq> cbox (-a) a"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1540
  by (meson assms bounded_subset_box_symmetric box_subset_cbox order.trans)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1541
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1542
lemma frontier_cbox:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1543
  fixes a b :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1544
  shows "frontier (cbox a b) = cbox a b - box a b"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1545
  unfolding frontier_def unfolding interior_cbox and closure_closed[OF closed_cbox] ..
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1546
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1547
lemma frontier_box:
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1548
  fixes a b :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1549
  shows "frontier (box a b) = (if box a b = {} then {} else cbox a b - box a b)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1550
  by (simp add: frontier_def interior_open open_box)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1551
66884
c2128ab11f61 Switching to inverse image and constant_on, plus some new material
paulson <lp15@cam.ac.uk>
parents: 66827
diff changeset
  1552
lemma Int_interval_mixed_eq_empty:
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1553
  fixes a :: "'a::euclidean_space"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1554
   assumes "box c d \<noteq> {}"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1555
  shows "box a b \<inter> cbox c d = {} \<longleftrightarrow> box a b \<inter> box c d = {}"
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1556
  unfolding closure_box[OF assms, symmetric]
62843
313d3b697c9a Mostly renaming (from HOL Light to Isabelle conventions), with a couple of new results
paulson <lp15@cam.ac.uk>
parents: 62623
diff changeset
  1557
  unfolding open_Int_closure_eq_empty[OF open_box] ..
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  1558
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1559
subsection \<open>Class Instances\<close>
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1560
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1561
lemma compact_lemma:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1562
  fixes f :: "nat \<Rightarrow> 'a::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1563
  assumes "bounded (range f)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1564
  shows "\<forall>d\<subseteq>Basis. \<exists>l::'a. \<exists> r.
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1565
    strict_mono r \<and> (\<forall>e>0. eventually (\<lambda>n. \<forall>i\<in>d. dist (f (r n) \<bullet> i) (l \<bullet> i) < e) sequentially)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1566
  by (rule compact_lemma_general[where unproj="\<lambda>e. \<Sum>i\<in>Basis. e i *\<^sub>R i"])
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1567
     (auto intro!: assms bounded_linear_inner_left bounded_linear_image
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1568
       simp: euclidean_representation)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1569
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1570
instance\<^marker>\<open>tag important\<close> euclidean_space \<subseteq> heine_borel
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1571
proof
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1572
  fix f :: "nat \<Rightarrow> 'a"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1573
  assume f: "bounded (range f)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1574
  then obtain l::'a and r where r: "strict_mono r"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1575
    and l: "\<forall>e>0. eventually (\<lambda>n. \<forall>i\<in>Basis. dist (f (r n) \<bullet> i) (l \<bullet> i) < e) sequentially"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1576
    using compact_lemma [OF f] by blast
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1577
  {
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1578
    fix e::real
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1579
    assume "e > 0"
71172
nipkow
parents: 71033
diff changeset
  1580
    hence "e / real_of_nat DIM('a) > 0" by (simp)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1581
    with l have "eventually (\<lambda>n. \<forall>i\<in>Basis. dist (f (r n) \<bullet> i) (l \<bullet> i) < e / (real_of_nat DIM('a))) sequentially"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1582
      by simp
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1583
    moreover
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1584
    { fix n
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1585
      assume n: "\<forall>i\<in>Basis. dist (f (r n) \<bullet> i) (l \<bullet> i) < e / (real_of_nat DIM('a))"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1586
      have "dist (f (r n)) l \<le> (\<Sum>i\<in>Basis. dist (f (r n) \<bullet> i) (l \<bullet> i))"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1587
        using L2_set_le_sum [OF zero_le_dist] by (subst euclidean_dist_l2)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1588
      also have "\<dots> < (\<Sum>i\<in>(Basis::'a set). e / (real_of_nat DIM('a)))"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1589
        by (meson eucl.finite_Basis n nonempty_Basis sum_strict_mono)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1590
      finally have "dist (f (r n)) l < e"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1591
        by auto
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1592
    }
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1593
    ultimately have "\<forall>\<^sub>F n in sequentially. dist (f (r n)) l < e"
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1594
      by (rule eventually_mono)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1595
  }
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1596
  then have *: "(f \<circ> r) \<longlonglongrightarrow> l"
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1597
    unfolding o_def tendsto_iff by simp
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1598
  with r show "\<exists>l r. strict_mono r \<and> (f \<circ> r) \<longlonglongrightarrow> l"
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1599
    by auto
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1600
qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1601
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1602
instance\<^marker>\<open>tag important\<close> euclidean_space \<subseteq> banach ..
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1603
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1604
instance euclidean_space \<subseteq> second_countable_topology
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1605
proof
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1606
  define a where "a f = (\<Sum>i\<in>Basis. fst (f i) *\<^sub>R i)" for f :: "'a \<Rightarrow> real \<times> real"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1607
  then have a: "\<And>f. (\<Sum>i\<in>Basis. fst (f i) *\<^sub>R i) = a f"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1608
    by simp
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1609
  define b where "b f = (\<Sum>i\<in>Basis. snd (f i) *\<^sub>R i)" for f :: "'a \<Rightarrow> real \<times> real"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1610
  then have b: "\<And>f. (\<Sum>i\<in>Basis. snd (f i) *\<^sub>R i) = b f"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1611
    by simp
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1612
  define B where "B = (\<lambda>f. box (a f) (b f)) ` (Basis \<rightarrow>\<^sub>E (\<rat> \<times> \<rat>))"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1613
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1614
  have "Ball B open" by (simp add: B_def open_box)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1615
  moreover have "(\<forall>A. open A \<longrightarrow> (\<exists>B'\<subseteq>B. \<Union>B' = A))"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1616
  proof safe
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1617
    fix A::"'a set"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1618
    assume "open A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1619
    show "\<exists>B'\<subseteq>B. \<Union>B' = A"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1620
      using open_UNION_box[OF \<open>open A\<close>]
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1621
      by (smt (verit, ccfv_threshold) B_def a b image_iff mem_Collect_eq subsetI)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1622
  qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1623
  ultimately
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1624
  have "topological_basis B"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1625
    unfolding topological_basis_def by blast
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1626
  moreover
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1627
  have "countable B"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1628
    unfolding B_def
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1629
    by (intro countable_image countable_PiE finite_Basis countable_SIGMA countable_rat)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1630
  ultimately show "\<exists>B::'a set set. countable B \<and> open = generate_topology B"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1631
    by (blast intro: topological_basis_imp_subbasis)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1632
qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1633
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1634
instance euclidean_space \<subseteq> polish_space ..
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1635
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1636
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1637
subsection \<open>Compact Boxes\<close>
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1638
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1639
lemma compact_cbox [simp]:
61076
bdc1e2f0a86a eliminated \<Colon>;
wenzelm
parents: 60974
diff changeset
  1640
  fixes a :: "'a::euclidean_space"
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1641
  shows "compact (cbox a b)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1642
  using bounded_closed_imp_seq_compact[of "cbox a b"] using bounded_cbox[of a b]
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1643
  by (auto simp: compact_eq_seq_compact_metric)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1644
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1645
proposition is_interval_compact:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1646
   "is_interval S \<and> compact S \<longleftrightarrow> (\<exists>a b. S = cbox a b)"   (is "?lhs = ?rhs")
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1647
proof (cases "S = {}")
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1648
  case True
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1649
  with empty_as_interval show ?thesis by auto
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1650
next
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1651
  case False
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1652
  show ?thesis
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1653
  proof
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1654
    assume L: ?lhs
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1655
    then have "is_interval S" "compact S" by auto
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1656
    define a where "a \<equiv> \<Sum>i\<in>Basis. (INF x\<in>S. x \<bullet> i) *\<^sub>R i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1657
    define b where "b \<equiv> \<Sum>i\<in>Basis. (SUP x\<in>S. x \<bullet> i) *\<^sub>R i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1658
    have 1: "\<And>x i. \<lbrakk>x \<in> S; i \<in> Basis\<rbrakk> \<Longrightarrow> (INF x\<in>S. x \<bullet> i) \<le> x \<bullet> i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1659
      by (simp add: cInf_lower bounded_inner_imp_bdd_below compact_imp_bounded L)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1660
    have 2: "\<And>x i. \<lbrakk>x \<in> S; i \<in> Basis\<rbrakk> \<Longrightarrow> x \<bullet> i \<le> (SUP x\<in>S. x \<bullet> i)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1661
      by (simp add: cSup_upper bounded_inner_imp_bdd_above compact_imp_bounded L)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1662
    have 3: "x \<in> S" if inf: "\<And>i. i \<in> Basis \<Longrightarrow> (INF x\<in>S. x \<bullet> i) \<le> x \<bullet> i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1663
                   and sup: "\<And>i. i \<in> Basis \<Longrightarrow> x \<bullet> i \<le> (SUP x\<in>S. x \<bullet> i)" for x
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1664
    proof (rule mem_box_componentwiseI [OF \<open>is_interval S\<close>])
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1665
      fix i::'a
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1666
      assume i: "i \<in> Basis"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1667
      have cont: "continuous_on S (\<lambda>x. x \<bullet> i)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1668
        by (intro continuous_intros)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1669
      obtain a where "a \<in> S" and a: "\<And>y. y\<in>S \<Longrightarrow> a \<bullet> i \<le> y \<bullet> i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1670
        using continuous_attains_inf [OF \<open>compact S\<close> False cont] by blast
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1671
      obtain b where "b \<in> S" and b: "\<And>y. y\<in>S \<Longrightarrow> y \<bullet> i \<le> b \<bullet> i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1672
        using continuous_attains_sup [OF \<open>compact S\<close> False cont] by blast
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1673
      have "a \<bullet> i \<le> (INF x\<in>S. x \<bullet> i)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1674
        by (simp add: False a cINF_greatest)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1675
      also have "\<dots> \<le> x \<bullet> i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1676
        by (simp add: i inf)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1677
      finally have ai: "a \<bullet> i \<le> x \<bullet> i" .
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1678
      have "x \<bullet> i \<le> (SUP x\<in>S. x \<bullet> i)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1679
        by (simp add: i sup)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1680
      also have "(SUP x\<in>S. x \<bullet> i) \<le> b \<bullet> i"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1681
        by (simp add: False b cSUP_least)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1682
      finally have bi: "x \<bullet> i \<le> b \<bullet> i" .
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1683
      show "x \<bullet> i \<in> (\<lambda>x. x \<bullet> i) ` S"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1684
        apply (rule_tac x="\<Sum>j\<in>Basis. (((\<bullet>)a)(i := x \<bullet> j))j *\<^sub>R j" in image_eqI)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1685
        apply (simp add: i)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1686
        apply (rule mem_is_intervalI [OF \<open>is_interval S\<close> \<open>a \<in> S\<close> \<open>b \<in> S\<close>])
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1687
        using i ai bi 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1688
        apply force
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1689
        done
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1690
    qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1691
    have "S = cbox a b"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1692
      by (auto simp: a_def b_def mem_box intro: 1 2 3)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1693
    then show ?rhs
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1694
      by blast
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1695
  next
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1696
    assume R: ?rhs
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1697
    then show ?lhs
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1698
      using compact_cbox is_interval_cbox by blast
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1699
  qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1700
qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1701
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  1702
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1703
subsection\<^marker>\<open>tag unimportant\<close>\<open>Componentwise limits and continuity\<close>
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1704
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1705
text\<open>But is the premise really necessary? Need to generalise @{thm euclidean_dist_l2}\<close>
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1706
lemma Euclidean_dist_upper: "i \<in> Basis \<Longrightarrow> dist (x \<bullet> i) (y \<bullet> i) \<le> dist x y"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1707
  by (metis (no_types) member_le_L2_set euclidean_dist_l2 finite_Basis)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1708
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1709
text\<open>But is the premise \<^term>\<open>i \<in> Basis\<close> really necessary?\<close>
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1710
lemma open_preimage_inner:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1711
  assumes "open S" "i \<in> Basis"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1712
    shows "open {x. x \<bullet> i \<in> S}"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1713
proof (rule openI, simp)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1714
  fix x
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1715
  assume x: "x \<bullet> i \<in> S"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1716
  with assms obtain e where "0 < e" and e: "ball (x \<bullet> i) e \<subseteq> S"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1717
    by (auto simp: open_contains_ball_eq)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1718
  have "\<exists>e>0. ball (y \<bullet> i) e \<subseteq> S" if dxy: "dist x y < e / 2" for y
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1719
  proof (intro exI conjI)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1720
    have "dist (x \<bullet> i) (y \<bullet> i) < e / 2"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1721
      by (meson \<open>i \<in> Basis\<close> dual_order.trans Euclidean_dist_upper not_le that)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1722
    then have "dist (x \<bullet> i) z < e" if "dist (y \<bullet> i) z < e / 2" for z
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1723
      by (metis dist_commute dist_triangle_half_l that)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1724
    then have "ball (y \<bullet> i) (e / 2) \<subseteq> ball (x \<bullet> i) e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1725
      using mem_ball by blast
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1726
      with e show "ball (y \<bullet> i) (e / 2) \<subseteq> S"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1727
        by (metis order_trans)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1728
  qed (simp add: \<open>0 < e\<close>)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1729
  then show "\<exists>e>0. ball x e \<subseteq> {s. s \<bullet> i \<in> S}"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1730
    by (metis (no_types, lifting) \<open>0 < e\<close> \<open>open S\<close> half_gt_zero_iff mem_Collect_eq mem_ball open_contains_ball_eq subsetI)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1731
qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1732
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1733
proposition tendsto_componentwise_iff:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1734
  fixes f :: "_ \<Rightarrow> 'b::euclidean_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1735
  shows "(f \<longlongrightarrow> l) F \<longleftrightarrow> (\<forall>i \<in> Basis. ((\<lambda>x. (f x \<bullet> i)) \<longlongrightarrow> (l \<bullet> i)) F)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1736
         (is "?lhs = ?rhs")
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1737
proof
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1738
  assume ?lhs
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1739
  then show ?rhs
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1740
    unfolding tendsto_def
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1741
    by (smt (verit) eventually_elim2 mem_Collect_eq open_preimage_inner)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1742
next
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1743
  assume R: ?rhs
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1744
  then have "\<And>e. e > 0 \<Longrightarrow> \<forall>i\<in>Basis. \<forall>\<^sub>F x in F. dist (f x \<bullet> i) (l \<bullet> i) < e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1745
    unfolding tendsto_iff by blast
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1746
  then have R': "\<And>e. e > 0 \<Longrightarrow> \<forall>\<^sub>F x in F. \<forall>i\<in>Basis. dist (f x \<bullet> i) (l \<bullet> i) < e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1747
      by (simp add: eventually_ball_finite_distrib [symmetric])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1748
  show ?lhs
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1749
  unfolding tendsto_iff
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1750
  proof clarify
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1751
    fix e::real
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1752
    assume "0 < e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1753
    have *: "L2_set (\<lambda>i. dist (f x \<bullet> i) (l \<bullet> i)) Basis < e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1754
             if "\<forall>i\<in>Basis. dist (f x \<bullet> i) (l \<bullet> i) < e / real DIM('b)" for x
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1755
    proof -
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1756
      have "L2_set (\<lambda>i. dist (f x \<bullet> i) (l \<bullet> i)) Basis \<le> sum (\<lambda>i. dist (f x \<bullet> i) (l \<bullet> i)) Basis"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1757
        by (simp add: L2_set_le_sum)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1758
      also have "... < DIM('b) * (e / real DIM('b))"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1759
        by (meson DIM_positive sum_bounded_above_strict that)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1760
      also have "... = e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1761
        by (simp add: field_simps)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1762
      finally show "L2_set (\<lambda>i. dist (f x \<bullet> i) (l \<bullet> i)) Basis < e" .
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1763
    qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1764
    have "\<forall>\<^sub>F x in F. \<forall>i\<in>Basis. dist (f x \<bullet> i) (l \<bullet> i) < e / DIM('b)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1765
      by (simp add: R' \<open>0 < e\<close>)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1766
    then show "\<forall>\<^sub>F x in F. dist (f x) l < e"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1767
      by eventually_elim (metis (full_types) "*" euclidean_dist_l2)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1768
  qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1769
qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1770
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1771
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1772
corollary continuous_componentwise:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1773
   "continuous F f \<longleftrightarrow> (\<forall>i \<in> Basis. continuous F (\<lambda>x. (f x \<bullet> i)))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1774
by (simp add: continuous_def tendsto_componentwise_iff [symmetric])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1775
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1776
corollary continuous_on_componentwise:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1777
  fixes S :: "'a :: t2_space set"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1778
  shows "continuous_on S f \<longleftrightarrow> (\<forall>i \<in> Basis. continuous_on S (\<lambda>x. (f x \<bullet> i)))"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1779
  by (metis continuous_componentwise continuous_on_eq_continuous_within)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1780
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1781
lemma linear_componentwise_iff:
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1782
     "linear f' \<longleftrightarrow> (\<forall>i\<in>Basis. linear (\<lambda>x. f' x \<bullet> i))" (is "?lhs \<longleftrightarrow> ?rhs")
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1783
proof
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1784
  show "?lhs \<Longrightarrow> ?rhs"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1785
    by (simp add: Real_Vector_Spaces.linear_iff inner_left_distrib)
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1786
  show "?rhs \<Longrightarrow> ?lhs"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1787
    by (simp add: linear_iff) (metis euclidean_eqI inner_left_distrib inner_scaleR_left)
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1788
qed
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1789
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1790
lemma bounded_linear_componentwise_iff:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1791
     "(bounded_linear f') \<longleftrightarrow> (\<forall>i\<in>Basis. bounded_linear (\<lambda>x. f' x \<bullet> i))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1792
     (is "?lhs = ?rhs")
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1793
proof
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1794
  assume ?rhs
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1795
  then have "(\<forall>i\<in>Basis. \<exists>K. \<forall>x. \<bar>f' x \<bullet> i\<bar> \<le> norm x * K)" "linear f'"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1796
    by (auto simp: bounded_linear_def bounded_linear_axioms_def linear_componentwise_iff [symmetric] ball_conj_distrib)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1797
  then obtain F where F: "\<And>i x. i \<in> Basis \<Longrightarrow> \<bar>f' x \<bullet> i\<bar> \<le> norm x * F i"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1798
    by metis
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1799
  have "norm (f' x) \<le> norm x * sum F Basis" for x
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1800
  proof -
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1801
    have "norm (f' x) \<le> (\<Sum>i\<in>Basis. \<bar>f' x \<bullet> i\<bar>)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1802
      by (rule norm_le_l1)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1803
    also have "... \<le> (\<Sum>i\<in>Basis. norm x * F i)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1804
      by (metis F sum_mono)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1805
    also have "... = norm x * sum F Basis"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1806
      by (simp add: sum_distrib_left)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1807
    finally show ?thesis .
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1808
  qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1809
  then show ?lhs
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1810
    by (force simp: bounded_linear_def bounded_linear_axioms_def \<open>linear f'\<close>)
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1811
qed (simp add: bounded_linear_inner_left_comp)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1812
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1813
subsection\<^marker>\<open>tag unimportant\<close> \<open>Continuous Extension\<close>
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1814
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1815
definition clamp :: "'a::euclidean_space \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> 'a" where
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1816
  "clamp a b x = (if (\<forall>i\<in>Basis. a \<bullet> i \<le> b \<bullet> i)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1817
    then (\<Sum>i\<in>Basis. (if x\<bullet>i < a\<bullet>i then a\<bullet>i else if x\<bullet>i \<le> b\<bullet>i then x\<bullet>i else b\<bullet>i) *\<^sub>R i)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1818
    else a)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1819
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1820
lemma clamp_in_interval[simp]:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1821
  assumes "\<And>i. i \<in> Basis \<Longrightarrow> a \<bullet> i \<le> b \<bullet> i"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1822
  shows "clamp a b x \<in> cbox a b"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1823
  unfolding clamp_def
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1824
  using box_ne_empty(1)[of a b] assms by (auto simp: cbox_def)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1825
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1826
lemma clamp_cancel_cbox[simp]:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1827
  fixes x a b :: "'a::euclidean_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1828
  assumes x: "x \<in> cbox a b"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1829
  shows "clamp a b x = x"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1830
  using assms
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1831
  by (auto simp: clamp_def mem_box intro!: euclidean_eqI[where 'a='a])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1832
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1833
lemma clamp_empty_interval:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1834
  assumes "i \<in> Basis" "a \<bullet> i > b \<bullet> i"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1835
  shows "clamp a b = (\<lambda>_. a)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1836
  using assms
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1837
  by (force simp: clamp_def[abs_def] split: if_splits intro!: ext)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1838
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1839
lemma dist_clamps_le_dist_args:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1840
  fixes x :: "'a::euclidean_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1841
  shows "dist (clamp a b y) (clamp a b x) \<le> dist y x"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1842
proof cases
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1843
  assume le: "(\<forall>i\<in>Basis. a \<bullet> i \<le> b \<bullet> i)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1844
  then have "(\<Sum>i\<in>Basis. (dist (clamp a b y \<bullet> i) (clamp a b x \<bullet> i))\<^sup>2) \<le>
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1845
    (\<Sum>i\<in>Basis. (dist (y \<bullet> i) (x \<bullet> i))\<^sup>2)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1846
    by (auto intro!: sum_mono simp: clamp_def dist_real_def abs_le_square_iff[symmetric])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1847
  then show ?thesis
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1848
    by (auto intro: real_sqrt_le_mono
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1849
      simp: euclidean_dist_l2[where y=x] euclidean_dist_l2[where y="clamp a b x"] L2_set_def)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1850
qed (auto simp: clamp_def)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1851
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1852
lemma clamp_continuous_at:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1853
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::metric_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1854
    and x :: 'a
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1855
  assumes f_cont: "continuous_on (cbox a b) f"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1856
  shows "continuous (at x) (\<lambda>x. f (clamp a b x))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1857
proof cases
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1858
  assume le: "(\<forall>i\<in>Basis. a \<bullet> i \<le> b \<bullet> i)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1859
  show ?thesis
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1860
    unfolding continuous_at_eps_delta
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1861
  proof safe
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1862
    fix x :: 'a
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1863
    fix e :: real
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1864
    assume "e > 0"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1865
    moreover have "clamp a b x \<in> cbox a b"
71172
nipkow
parents: 71033
diff changeset
  1866
      by (simp add: le)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1867
    moreover note f_cont[simplified continuous_on_iff]
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1868
    ultimately
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1869
    obtain d where d: "0 < d"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1870
      "\<And>x'. x' \<in> cbox a b \<Longrightarrow> dist x' (clamp a b x) < d \<Longrightarrow> dist (f x') (f (clamp a b x)) < e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1871
      by force
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1872
    show "\<exists>d>0. \<forall>x'. dist x' x < d \<longrightarrow> dist (f (clamp a b x')) (f (clamp a b x)) < e"
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1873
      using le
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1874
      by (auto intro!: d clamp_in_interval dist_clamps_le_dist_args[THEN le_less_trans])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1875
  qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1876
qed (auto simp: clamp_empty_interval)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1877
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1878
lemma clamp_continuous_on:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1879
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::metric_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1880
  assumes f_cont: "continuous_on (cbox a b) f"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1881
  shows "continuous_on S (\<lambda>x. f (clamp a b x))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1882
  using assms
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1883
  by (auto intro: continuous_at_imp_continuous_on clamp_continuous_at)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1884
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1885
lemma clamp_bounded:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1886
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::metric_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1887
  assumes bounded: "bounded (f ` (cbox a b))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1888
  shows "bounded (range (\<lambda>x. f (clamp a b x)))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1889
proof cases
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1890
  assume le: "(\<forall>i\<in>Basis. a \<bullet> i \<le> b \<bullet> i)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1891
  from bounded obtain c where f_bound: "\<forall>x\<in>f ` cbox a b. dist undefined x \<le> c"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1892
    by (auto simp: bounded_any_center[where a=undefined])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1893
  then show ?thesis
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1894
    by (metis bounded bounded_subset clamp_in_interval image_mono image_subsetI le range_composition)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1895
qed (auto simp: clamp_empty_interval image_def)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1896
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1897
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1898
definition ext_cont :: "('a::euclidean_space \<Rightarrow> 'b::metric_space) \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> 'a \<Rightarrow> 'b"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1899
  where "ext_cont f a b = (\<lambda>x. f (clamp a b x))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1900
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1901
lemma ext_cont_cancel_cbox[simp]:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1902
  fixes x a b :: "'a::euclidean_space"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1903
  assumes x: "x \<in> cbox a b"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1904
  shows "ext_cont f a b x = f x"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1905
  using assms by (simp add: ext_cont_def)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1906
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1907
lemma continuous_on_ext_cont[continuous_intros]:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1908
  "continuous_on (cbox a b) f \<Longrightarrow> continuous_on S (ext_cont f a b)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1909
  by (auto intro!: clamp_continuous_on simp: ext_cont_def)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1910
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1911
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1912
subsection \<open>Separability\<close>
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1913
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1914
lemma univ_second_countable_sequence:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1915
  obtains B :: "nat \<Rightarrow> 'a::euclidean_space set"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1916
    where "inj B" "\<And>n. open(B n)" "\<And>S. open S \<Longrightarrow> \<exists>k. S = \<Union>{B n |n. n \<in> k}"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1917
proof -
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1918
  obtain \<B> :: "'a set set"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1919
  where "countable \<B>"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1920
    and opn: "\<And>C. C \<in> \<B> \<Longrightarrow> open C"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1921
    and Un: "\<And>S. open S \<Longrightarrow> \<exists>U. U \<subseteq> \<B> \<and> S = \<Union>U"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1922
    using univ_second_countable by blast
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1923
  have *: "infinite (range (\<lambda>n. ball (0::'a) (inverse(Suc n))))"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1924
    by (simp add: inj_on_def ball_eq_ball_iff Infinite_Set.range_inj_infinite)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1925
  have "infinite \<B>"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1926
  proof
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1927
    assume "finite \<B>"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1928
    then have "finite (Union ` (Pow \<B>))"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1929
      by simp
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1930
    moreover have "range (\<lambda>n. ball 0 (inverse (real (Suc n)))) \<subseteq> \<Union> ` Pow \<B>"
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1931
      by (metis (no_types, lifting) PowI image_eqI image_subset_iff Un [OF open_ball])
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1932
    ultimately show False
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1933
      by (metis finite_subset *)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1934
  qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1935
  obtain f :: "nat \<Rightarrow> 'a set" where "\<B> = range f" "inj f"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1936
    by (blast intro: countable_as_injective_image [OF \<open>countable \<B>\<close> \<open>infinite \<B>\<close>])
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1937
  have *: "\<exists>k. S = \<Union>{f n |n. n \<in> k}" if "open S" for S
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1938
    using Un [OF that]
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1939
    apply clarify
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1940
    apply (rule_tac x="f-`U" in exI)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1941
    using \<open>inj f\<close> \<open>\<B> = range f\<close> apply force
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1942
    done
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1943
  show ?thesis
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1944
    using "*" \<open>\<B> = range f\<close> \<open>inj f\<close> opn that by force
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1945
qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1946
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1947
proposition separable:
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1948
  fixes S :: "'a::{metric_space, second_countable_topology} set"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1949
  obtains T where "countable T" "T \<subseteq> S" "S \<subseteq> closure T"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1950
proof -
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1951
  obtain \<B> :: "'a set set"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1952
    where "countable \<B>"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1953
      and "{} \<notin> \<B>"
69922
4a9167f377b0 new material about topology, etc.; also fixes for yesterday's
paulson <lp15@cam.ac.uk>
parents: 69918
diff changeset
  1954
      and ope: "\<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: 69918
diff changeset
  1955
      and if_ope: "\<And>T. openin(top_of_set S) T \<Longrightarrow> \<exists>\<U>. \<U> \<subseteq> \<B> \<and> T = \<Union>\<U>"
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1956
    by (meson subset_second_countable)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1957
  then obtain f where f: "\<And>C. C \<in> \<B> \<Longrightarrow> f C \<in> C"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1958
    by (metis equals0I)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1959
  show ?thesis
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1960
  proof
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1961
    show "countable (f ` \<B>)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1962
      by (simp add: \<open>countable \<B>\<close>)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1963
    show "f ` \<B> \<subseteq> S"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1964
      using ope f openin_imp_subset by blast
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1965
    show "S \<subseteq> closure (f ` \<B>)"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1966
    proof (clarsimp simp: closure_approachable)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1967
      fix x and e::real
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1968
      assume "x \<in> S" "0 < e"
69922
4a9167f377b0 new material about topology, etc.; also fixes for yesterday's
paulson <lp15@cam.ac.uk>
parents: 69918
diff changeset
  1969
      have "openin (top_of_set S) (S \<inter> ball x e)"
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1970
        by (simp add: openin_Int_open)
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1971
      with if_ope obtain \<U> where  \<U>: "\<U> \<subseteq> \<B>" "S \<inter> ball x e = \<Union>\<U>"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1972
        by meson
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1973
      show "\<exists>C \<in> \<B>. dist (f C) x < e"
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1974
      proof (cases "\<U> = {}")
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1975
        case True
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1976
        then show ?thesis
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1977
          using \<open>0 < e\<close>  \<U> \<open>x \<in> S\<close> by auto
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1978
      next
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1979
        case False
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1980
        then show ?thesis
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  1981
          by (metis IntI Union_iff \<U> \<open>0 < e\<close> \<open>x \<in> S\<close> dist_commute dist_self f inf_le2 mem_ball subset_eq)
69615
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1982
      qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1983
    qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1984
  qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1985
qed
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1986
e502cd4d7062 moved material from Connected.thy to more appropriate places
immler
parents: 69613
diff changeset
  1987
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  1988
subsection\<^marker>\<open>tag unimportant\<close> \<open>Diameter\<close>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1989
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1990
lemma diameter_cball [simp]:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1991
  fixes a :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1992
  shows "diameter(cball a r) = (if r < 0 then 0 else 2*r)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1993
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1994
  have "diameter(cball a r) = 2*r" if "r \<ge> 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1995
  proof (rule order_antisym)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1996
    show "diameter (cball a r) \<le> 2*r"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1997
    proof (rule diameter_le)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1998
      fix x y assume "x \<in> cball a r" "y \<in> cball a r"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  1999
      then have "norm (x - a) \<le> r" "norm (a - y) \<le> r"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2000
        by (auto simp: dist_norm norm_minus_commute)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2001
      then have "norm (x - y) \<le> r+r"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2002
        using norm_diff_triangle_le by blast
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2003
      then show "norm (x - y) \<le> 2*r" by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2004
    qed (simp add: that)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2005
    have "2*r = dist (a + r *\<^sub>R (SOME i. i \<in> Basis)) (a - r *\<^sub>R (SOME i. i \<in> Basis))"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2006
      using \<open>0 \<le> r\<close> that by (simp add: dist_norm flip: scaleR_2)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2007
    also have "... \<le> diameter (cball a r)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2008
      apply (rule diameter_bounded_bound)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2009
      using that by (auto simp: dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2010
    finally show "2*r \<le> diameter (cball a r)" .
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2011
  qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2012
  then show ?thesis by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2013
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2014
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2015
lemma diameter_ball [simp]:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2016
  fixes a :: "'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2017
  shows "diameter(ball a r) = (if r < 0 then 0 else 2*r)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2018
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2019
  have "diameter(ball a r) = 2*r" if "r > 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2020
    by (metis bounded_ball diameter_closure closure_ball diameter_cball less_eq_real_def linorder_not_less that)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2021
  then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2022
    by (simp add: diameter_def)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2023
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2024
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2025
lemma diameter_closed_interval [simp]: "diameter {a..b} = (if b < a then 0 else b-a)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2026
proof -
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2027
  have "{a..b} = cball ((a+b)/2) ((b-a)/2)"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2028
    using atLeastAtMost_eq_cball by blast
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2029
  then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2030
    by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2031
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2032
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2033
lemma diameter_open_interval [simp]: "diameter {a<..<b} = (if b < a then 0 else b-a)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2034
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2035
  have "{a <..< b} = ball ((a+b)/2) ((b-a)/2)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2036
    using greaterThanLessThan_eq_ball by blast
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2037
  then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2038
    by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2039
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2040
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2041
lemma diameter_cbox:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2042
  fixes a b::"'a::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2043
  shows "(\<forall>i \<in> Basis. a \<bullet> i \<le> b \<bullet> i) \<Longrightarrow> diameter (cbox a b) = dist a b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2044
  by (force simp: diameter_def intro!: cSup_eq_maximum L2_set_mono
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2045
     simp: euclidean_dist_l2[where 'a='a] cbox_def dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2046
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2047
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  2048
subsection\<^marker>\<open>tag unimportant\<close>\<open>Relating linear images to open/closed/interior/closure/connected\<close>
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  2049
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2050
proposition open_surjective_linear_image:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2051
  fixes f :: "'a::real_normed_vector \<Rightarrow> 'b::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2052
  assumes "open A" "linear f" "surj f"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2053
    shows "open(f ` A)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2054
unfolding open_dist
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2055
proof clarify
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2056
  fix x
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2057
  assume "x \<in> A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2058
  have "bounded (inv f ` Basis)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2059
    by (simp add: finite_imp_bounded)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2060
  with bounded_pos obtain B where "B > 0" and B: "\<And>x. x \<in> inv f ` Basis \<Longrightarrow> norm x \<le> B"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2061
    by metis
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2062
  obtain e where "e > 0" and e: "\<And>z. dist z x < e \<Longrightarrow> z \<in> A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2063
    by (metis open_dist \<open>x \<in> A\<close> \<open>open A\<close>)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2064
  define \<delta> where "\<delta> \<equiv> e / B / DIM('b)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2065
  show "\<exists>e>0. \<forall>y. dist y (f x) < e \<longrightarrow> y \<in> f ` A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2066
  proof (intro exI conjI)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2067
    show "\<delta> > 0"
70817
dd675800469d dedicated fact collections for algebraic simplification rules potentially splitting goals
haftmann
parents: 70802
diff changeset
  2068
      using \<open>e > 0\<close> \<open>B > 0\<close>  by (simp add: \<delta>_def field_split_simps)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2069
    have "y \<in> f ` A" if "dist y (f x) * (B * real DIM('b)) < e" for y
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2070
    proof -
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2071
      define u where "u \<equiv> y - f x"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2072
      show ?thesis
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2073
      proof (rule image_eqI)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2074
        show "y = f (x + (\<Sum>i\<in>Basis. (u \<bullet> i) *\<^sub>R inv f i))"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2075
          apply (simp add: linear_add linear_sum linear.scaleR \<open>linear f\<close> surj_f_inv_f \<open>surj f\<close>)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2076
          apply (simp add: euclidean_representation u_def)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2077
          done
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2078
        have "dist (x + (\<Sum>i\<in>Basis. (u \<bullet> i) *\<^sub>R inv f i)) x \<le> (\<Sum>i\<in>Basis. norm ((u \<bullet> i) *\<^sub>R inv f i))"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2079
          by (simp add: dist_norm sum_norm_le)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2080
        also have "... = (\<Sum>i\<in>Basis. \<bar>u \<bullet> i\<bar> * norm (inv f i))"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2081
          by simp
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2082
        also have "... \<le> (\<Sum>i\<in>Basis. \<bar>u \<bullet> i\<bar>) * B"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2083
          by (simp add: B sum_distrib_right sum_mono mult_left_mono)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2084
        also have "... \<le> DIM('b) * dist y (f x) * B"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2085
          apply (rule mult_right_mono [OF sum_bounded_above])
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2086
          using \<open>0 < B\<close> by (auto simp: Basis_le_norm dist_norm u_def)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2087
        also have "... < e"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2088
          by (metis mult.commute mult.left_commute that)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2089
        finally show "x + (\<Sum>i\<in>Basis. (u \<bullet> i) *\<^sub>R inv f i) \<in> A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2090
          by (rule e)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2091
      qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2092
    qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2093
    then show "\<forall>y. dist y (f x) < \<delta> \<longrightarrow> y \<in> f ` A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2094
      using \<open>e > 0\<close> \<open>B > 0\<close>
71172
nipkow
parents: 71033
diff changeset
  2095
      by (auto simp: \<delta>_def field_split_simps)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2096
  qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2097
qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2098
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2099
corollary open_bijective_linear_image_eq:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2100
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2101
  assumes "linear f" "bij f"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2102
    shows "open(f ` A) \<longleftrightarrow> open A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2103
proof
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2104
  assume "open(f ` A)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2105
  then show "open A"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2106
    by (metis assms bij_is_inj continuous_open_vimage inj_vimage_image_eq linear_continuous_at linear_linear)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2107
next
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2108
  assume "open A"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2109
  then show "open(f ` A)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2110
    by (simp add: assms bij_is_surj open_surjective_linear_image)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2111
qed
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2112
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2113
corollary interior_bijective_linear_image:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2114
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2115
  assumes "linear f" "bij f"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2116
  shows "interior (f ` S) = f ` interior S" 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2117
  by (smt (verit) assms bij_is_inj inj_image_subset_iff interior_maximal interior_subset 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2118
      open_bijective_linear_image_eq open_interior subset_antisym subset_imageE)
69611
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2119
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2120
lemma interior_injective_linear_image:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2121
  fixes f :: "'a::euclidean_space \<Rightarrow> 'a::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2122
  assumes "linear f" "inj f"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2123
   shows "interior(f ` S) = f ` (interior S)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2124
  by (simp add: linear_injective_imp_surjective assms bijI interior_bijective_linear_image)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2125
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2126
lemma interior_surjective_linear_image:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2127
  fixes f :: "'a::euclidean_space \<Rightarrow> 'a::euclidean_space"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2128
  assumes "linear f" "surj f"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2129
   shows "interior(f ` S) = f ` (interior S)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2130
  by (simp add: assms interior_injective_linear_image linear_surjective_imp_injective)
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2131
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2132
lemma interior_negations:
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2133
  fixes S :: "'a::euclidean_space set"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2134
  shows "interior(uminus ` S) = image uminus (interior S)"
42cc3609fedf moved some material from Connected.thy to more appropriate places
immler
parents: 69544
diff changeset
  2135
  by (simp add: bij_uminus interior_bijective_linear_image linear_uminus)
56189
c4daa97ac57a removed dependencies on theory Ordered_Euclidean_Space
immler
parents: 56188
diff changeset
  2136
69617
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2137
lemma connected_linear_image:
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2138
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::real_normed_vector"
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2139
  assumes "linear f" and "connected s"
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2140
  shows "connected (f ` s)"
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2141
using connected_continuous_image assms linear_continuous_on linear_conv_bounded_linear by blast
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2142
63ee37c519a3 reduced dependencies of Connected.thy
immler
parents: 69615
diff changeset
  2143
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  2144
subsection\<^marker>\<open>tag unimportant\<close> \<open>"Isometry" (up to constant bounds) of Injective Linear Map\<close>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2145
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2146
proposition injective_imp_isometric:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2147
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2148
  assumes s: "closed s" "subspace s"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2149
    and f: "bounded_linear f" "\<forall>x\<in>s. f x = 0 \<longrightarrow> x = 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2150
  shows "\<exists>e>0. \<forall>x\<in>s. norm (f x) \<ge> e * norm x"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2151
proof (cases "s \<subseteq> {0::'a}")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2152
  case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2153
  have "norm x \<le> norm (f x)" if "x \<in> s" for x
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2154
  proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2155
    from True that have "x = 0" by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2156
    then show ?thesis by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2157
  qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2158
  then show ?thesis
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2159
    by (auto intro!: exI[where x=1])
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2160
next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2161
  case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2162
  interpret f: bounded_linear f by fact
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2163
  from False obtain a where a: "a \<noteq> 0" "a \<in> s"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2164
    by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2165
  from False have "s \<noteq> {}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2166
    by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2167
  let ?S = "{f x| x. x \<in> s \<and> norm x = norm a}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2168
  let ?S' = "{x::'a. x\<in>s \<and> norm x = norm a}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2169
  let ?S'' = "{x::'a. norm x = norm a}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2170
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2171
  have "?S'' = frontier (cball 0 (norm a))"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2172
    by (simp add: sphere_def dist_norm)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2173
  then have "compact ?S''" by (metis compact_cball compact_frontier)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2174
  moreover have "?S' = s \<inter> ?S''" by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2175
  ultimately have "compact ?S'"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2176
    using closed_Int_compact[of s ?S''] using s(1) by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2177
  moreover have *:"f ` ?S' = ?S" by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2178
  ultimately have "compact ?S"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2179
    using compact_continuous_image[OF linear_continuous_on[OF f(1)], of ?S'] by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2180
  then have "closed ?S"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2181
    using compact_imp_closed by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2182
  moreover from a have "?S \<noteq> {}" by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2183
  ultimately obtain b' where "b'\<in>?S" "\<forall>y\<in>?S. norm b' \<le> norm y"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2184
    using distance_attains_inf[of ?S 0] unfolding dist_0_norm by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2185
  then obtain b where "b\<in>s"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2186
    and ba: "norm b = norm a"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2187
    and b: "\<forall>x\<in>{x \<in> s. norm x = norm a}. norm (f b) \<le> norm (f x)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2188
    unfolding *[symmetric] unfolding image_iff by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2189
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2190
  let ?e = "norm (f b) / norm b"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2191
  have "norm b > 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2192
    using ba and a and norm_ge_zero by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2193
  moreover have "norm (f b) > 0"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2194
    using f(2)[THEN bspec[where x=b], OF \<open>b\<in>s\<close>]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2195
    using \<open>norm b >0\<close> by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2196
  ultimately have "0 < norm (f b) / norm b" by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2197
  moreover
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2198
  have "norm (f b) / norm b * norm x \<le> norm (f x)" if "x\<in>s" for x
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2199
  proof (cases "x = 0")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2200
    case True
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2201
    then show "norm (f b) / norm b * norm x \<le> norm (f x)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2202
      by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2203
  next
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2204
    case False
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2205
    with \<open>a \<noteq> 0\<close> have *: "0 < norm a / norm x"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2206
      unfolding zero_less_norm_iff[symmetric] by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2207
    have "\<forall>x\<in>s. c *\<^sub>R x \<in> s" for c
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2208
      using s[unfolded subspace_def] by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2209
    with \<open>x \<in> s\<close> \<open>x \<noteq> 0\<close> have "(norm a / norm x) *\<^sub>R x \<in> {x \<in> s. norm x = norm a}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2210
      by simp
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2211
    with \<open>x \<noteq> 0\<close> \<open>a \<noteq> 0\<close> show "norm (f b) / norm b * norm x \<le> norm (f x)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2212
      using b[THEN bspec[where x="(norm a / norm x) *\<^sub>R x"]]
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2213
      unfolding f.scaleR and ba
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2214
      by (auto simp: mult.commute pos_le_divide_eq pos_divide_le_eq)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2215
  qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2216
  ultimately show ?thesis by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2217
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2218
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2219
proposition closed_injective_image_subspace:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2220
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2221
  assumes "subspace s" "bounded_linear f" "\<forall>x\<in>s. f x = 0 \<longrightarrow> x = 0" "closed s"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2222
  shows "closed(f ` s)"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2223
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2224
  obtain e where "e > 0" and e: "\<forall>x\<in>s. e * norm x \<le> norm (f x)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2225
    using assms injective_imp_isometric by blast
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2226
  with assms show ?thesis
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2227
    by (meson complete_eq_closed complete_isometric_image)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2228
qed
71255
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2229
                               
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2230
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2231
lemma closure_bounded_linear_image_subset:
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2232
  assumes f: "bounded_linear f"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2233
  shows "f ` closure S \<subseteq> closure (f ` S)"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2234
  using linear_continuous_on [OF f] closed_closure closure_subset
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2235
  by (rule image_closure_subset)
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2236
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2237
lemma closure_linear_image_subset:
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2238
  fixes f :: "'m::euclidean_space \<Rightarrow> 'n::real_normed_vector"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2239
  assumes "linear f"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2240
  shows "f ` (closure S) \<subseteq> closure (f ` S)"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2241
  using assms unfolding linear_conv_bounded_linear
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2242
  by (rule closure_bounded_linear_image_subset)
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2243
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2244
lemma closed_injective_linear_image:
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2245
    fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2246
    assumes S: "closed S" and f: "linear f" "inj f"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2247
    shows "closed (f ` S)"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2248
proof -
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2249
  obtain g where g: "linear g" "g \<circ> f = id"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2250
    using linear_injective_left_inverse [OF f] by blast
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2251
  then have confg: "continuous_on (range f) g"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2252
    using linear_continuous_on linear_conv_bounded_linear by blast
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2253
  have [simp]: "g ` f ` S = S"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2254
    using g by (simp add: image_comp)
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2255
  have cgf: "closed (g ` f ` S)"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2256
    by (simp add: \<open>g \<circ> f = id\<close> S image_comp)
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2257
  have [simp]: "(range f \<inter> g -` S) = f ` S"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2258
    using g unfolding o_def id_def image_def by auto metis+
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2259
  show ?thesis
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2260
  proof (rule closedin_closed_trans [of "range f"])
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2261
    show "closedin (top_of_set (range f)) (f ` S)"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2262
      using continuous_closedin_preimage [OF confg cgf] by simp
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2263
    show "closed (range f)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2264
      using closed_injective_image_subspace f linear_conv_bounded_linear 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2265
          linear_injective_0 subspace_UNIV by blast
71255
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2266
  qed
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2267
qed
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2268
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2269
lemma closed_injective_linear_image_eq:
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2270
    fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2271
    assumes f: "linear f" "inj f"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2272
      shows "(closed(image f s) \<longleftrightarrow> closed s)"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2273
  by (metis closed_injective_linear_image closure_eq closure_linear_image_subset closure_subset_eq f(1) f(2) inj_image_subset_iff)
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2274
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2275
lemma closure_injective_linear_image:
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2276
    fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2277
    shows "\<lbrakk>linear f; inj f\<rbrakk> \<Longrightarrow> f ` (closure S) = closure (f ` S)"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2278
  by (simp add: closed_injective_linear_image closure_linear_image_subset 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2279
        closure_minimal closure_subset image_mono subset_antisym)
71255
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2280
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2281
lemma closure_bounded_linear_image:
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2282
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2283
  assumes "linear f" "bounded S"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2284
    shows "f ` (closure S) = closure (f ` S)"  (is "?lhs = ?rhs")
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2285
proof
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2286
  show "?lhs \<subseteq> ?rhs"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2287
    using assms closure_linear_image_subset by blast
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2288
  show "?rhs \<subseteq> ?lhs"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2289
    using assms by (meson closure_minimal closure_subset compact_closure compact_eq_bounded_closed
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2290
                      compact_continuous_image image_mono linear_continuous_on linear_linear)
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2291
qed
71255
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2292
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2293
lemma closure_scaleR:
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2294
  fixes S :: "'a::real_normed_vector set"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2295
  shows "((*\<^sub>R) c) ` (closure S) = closure (((*\<^sub>R) c) ` S)"  (is "?lhs = ?rhs")
71255
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2296
proof
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2297
  show "?lhs \<subseteq> ?rhs"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2298
    using bounded_linear_scaleR_right by (rule closure_bounded_linear_image_subset)
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2299
  show "?rhs \<subseteq> ?lhs"
71255
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2300
    by (intro closure_minimal image_mono closure_subset closed_scaling closed_closure)
4258ee13f5d4 moved lemmas
nipkow
parents: 71172
diff changeset
  2301
qed
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2302
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2303
70136
f03a01a18c6e modernized tags: default scope excludes proof;
wenzelm
parents: 70086
diff changeset
  2304
subsection\<^marker>\<open>tag unimportant\<close> \<open>Some properties of a canonical subspace\<close>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2305
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2306
lemma closed_substandard: "closed {x::'a::euclidean_space. \<forall>i\<in>Basis. P i \<longrightarrow> x\<bullet>i = 0}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2307
  (is "closed ?A")
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2308
proof -
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2309
  let ?D = "{i\<in>Basis. P i}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2310
  have "closed (\<Inter>i\<in>?D. {x::'a. x\<bullet>i = 0})"
71172
nipkow
parents: 71033
diff changeset
  2311
    by (simp add: closed_INT closed_Collect_eq continuous_on_inner)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2312
  also have "(\<Inter>i\<in>?D. {x::'a. x\<bullet>i = 0}) = ?A"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2313
    by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2314
  finally show "closed ?A" .
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2315
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2316
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2317
lemma closed_subspace:
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2318
  fixes S :: "'a::euclidean_space set"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2319
  assumes "subspace S"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2320
  shows "closed S"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2321
proof -
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2322
  have "dim S \<le> card (Basis :: 'a set)"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2323
    using dim_subset_UNIV by auto
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2324
  with obtain_subset_with_card_n 
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2325
  obtain d :: "'a set" where cd: "card d = dim S" and d: "d \<subseteq> Basis"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2326
    by metis
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2327
  let ?t = "{x::'a. \<forall>i\<in>Basis. i \<notin> d \<longrightarrow> x\<bullet>i = 0}"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2328
  have "\<exists>f. linear f \<and> f ` {x::'a. \<forall>i\<in>Basis. i \<notin> d \<longrightarrow> x \<bullet> i = 0} = S \<and>
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2329
      inj_on f {x::'a. \<forall>i\<in>Basis. i \<notin> d \<longrightarrow> x \<bullet> i = 0}"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2330
    using dim_substandard[of d] cd d assms
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2331
    by (intro subspace_isomorphism[OF subspace_substandard[of "\<lambda>i. i \<notin> d"]]) (auto simp: inner_Basis)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2332
  then obtain f where f:
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2333
      "linear f"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2334
      "f ` {x. \<forall>i\<in>Basis. i \<notin> d \<longrightarrow> x \<bullet> i = 0} = S"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2335
      "inj_on f {x. \<forall>i\<in>Basis. i \<notin> d \<longrightarrow> x \<bullet> i = 0}"
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2336
    by blast
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2337
  interpret f: bounded_linear f
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2338
    using f by (simp add: linear_conv_bounded_linear)
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2339
  have "x \<in> ?t \<Longrightarrow> f x = 0 \<Longrightarrow> x = 0" for x
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2340
    using f.zero d f(3)[THEN inj_onD, of x 0] by auto
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2341
  then show ?thesis
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2342
    using closed_injective_image_subspace[of ?t f] closed_substandard subspace_substandard
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2343
    using f(2) f.bounded_linear_axioms by force
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2344
qed
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2345
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2346
lemma complete_subspace: "subspace S \<Longrightarrow> complete S"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2347
  for S :: "'a::euclidean_space set"
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2348
  using complete_eq_closed closed_subspace by auto
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2349
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2350
lemma closed_span [iff]: "closed (span S)"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2351
  for S :: "'a::euclidean_space set"
71172
nipkow
parents: 71033
diff changeset
  2352
  by (simp add: closed_subspace)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2353
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2354
lemma dim_closure [simp]: "dim (closure S) = dim S" (is "?dc = ?d")
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2355
  for S :: "'a::euclidean_space set"
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2356
  by (metis closed_span closure_minimal closure_subset dim_eq_span span_eq_dim span_superset subset_le_dim)
69613
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2357
1331e57b54c6 moved material from Connected.thy to more appropriate places
immler
parents: 69611
diff changeset
  2358
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2359
subsection \<open>Set Distance\<close>
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2360
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2361
lemma setdist_compact_closed:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2362
  fixes A :: "'a::heine_borel set"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2363
  assumes "compact A" "closed B"
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2364
    and "A \<noteq> {}" "B \<noteq> {}"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2365
  shows "\<exists>x \<in> A. \<exists>y \<in> B. dist x y = setdist A B"
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2366
  by (metis assms infdist_attains_inf setdist_attains_inf setdist_sym)
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2367
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2368
lemma setdist_closed_compact:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2369
  fixes S :: "'a::heine_borel set"
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2370
  assumes S: "closed S" and T: "compact T"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2371
      and "S \<noteq> {}" "T \<noteq> {}"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2372
    shows "\<exists>x \<in> S. \<exists>y \<in> T. dist x y = setdist S T"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2373
  using setdist_compact_closed [OF T S \<open>T \<noteq> {}\<close> \<open>S \<noteq> {}\<close>]
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2374
  by (metis dist_commute setdist_sym)
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2375
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2376
lemma setdist_eq_0_compact_closed:
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2377
  assumes S: "compact S" and T: "closed T"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2378
    shows "setdist S T = 0 \<longleftrightarrow> S = {} \<or> T = {} \<or> S \<inter> T \<noteq> {}"
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2379
proof (cases "S = {} \<or> T = {}")
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2380
  case False
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2381
  then show ?thesis
76836
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2382
    by (metis S T disjoint_iff in_closed_iff_infdist_zero setdist_attains_inf setdist_eq_0I setdist_sym)
30182f9e1818 Big simplifications of old proofs
paulson <lp15@cam.ac.uk>
parents: 76834
diff changeset
  2383
qed auto
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2384
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2385
corollary setdist_gt_0_compact_closed:
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2386
  assumes S: "compact S" and T: "closed T"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2387
    shows "setdist S T > 0 \<longleftrightarrow> (S \<noteq> {} \<and> T \<noteq> {} \<and> S \<inter> T = {})"
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2388
  using setdist_pos_le [of S T] setdist_eq_0_compact_closed [OF assms] by linarith
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2389
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2390
lemma setdist_eq_0_closed_compact:
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2391
  assumes S: "closed S" and T: "compact T"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2392
    shows "setdist S T = 0 \<longleftrightarrow> S = {} \<or> T = {} \<or> S \<inter> T \<noteq> {}"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2393
  using setdist_eq_0_compact_closed [OF T S]
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2394
  by (metis Int_commute setdist_sym)
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2395
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2396
lemma setdist_eq_0_bounded:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2397
  fixes S :: "'a::heine_borel set"
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2398
  assumes "bounded S \<or> bounded T"
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2399
  shows "setdist S T = 0 \<longleftrightarrow> S = {} \<or> T = {} \<or> closure S \<inter> closure T \<noteq> {}"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2400
proof (cases "S = {} \<or> T = {}")
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2401
  case False
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2402
  then show ?thesis
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2403
    using setdist_eq_0_compact_closed [of "closure S" "closure T"]
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2404
          setdist_eq_0_closed_compact [of "closure S" "closure T"] assms
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2405
    by (force simp:  bounded_closure compact_eq_bounded_closed)
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2406
qed force
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2407
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2408
lemma setdist_eq_0_sing_1:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2409
  "setdist {x} S = 0 \<longleftrightarrow> S = {} \<or> x \<in> closure S"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2410
  by (metis in_closure_iff_infdist_zero infdist_def infdist_eq_setdist)
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2411
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2412
lemma setdist_eq_0_sing_2:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2413
  "setdist S {x} = 0 \<longleftrightarrow> S = {} \<or> x \<in> closure S"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2414
  by (metis setdist_eq_0_sing_1 setdist_sym)
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2415
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2416
lemma setdist_neq_0_sing_1:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2417
  "\<lbrakk>setdist {x} S = a; a \<noteq> 0\<rbrakk> \<Longrightarrow> S \<noteq> {} \<and> x \<notin> closure S"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2418
  by (metis setdist_closure_2 setdist_empty2 setdist_eq_0I singletonI)
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2419
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2420
lemma setdist_neq_0_sing_2:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2421
  "\<lbrakk>setdist S {x} = a; a \<noteq> 0\<rbrakk> \<Longrightarrow> S \<noteq> {} \<and> x \<notin> closure S"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2422
  by (simp add: setdist_neq_0_sing_1 setdist_sym)
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2423
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2424
lemma setdist_sing_in_set:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2425
   "x \<in> S \<Longrightarrow> setdist {x} S = 0"
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2426
  by (simp add: setdist_eq_0I)
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2427
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2428
lemma setdist_eq_0_closed:
69918
eddcc7c726f3 new material;' strengthened material; moved proofs out of Function_Topology in order to lessen its dependencies
paulson <lp15@cam.ac.uk>
parents: 69750
diff changeset
  2429
   "closed S \<Longrightarrow> (setdist {x} S = 0 \<longleftrightarrow> S = {} \<or> x \<in> S)"
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2430
by (simp add: setdist_eq_0_sing_1)
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2431
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2432
lemma setdist_eq_0_closedin:
69922
4a9167f377b0 new material about topology, etc.; also fixes for yesterday's
paulson <lp15@cam.ac.uk>
parents: 69918
diff changeset
  2433
  shows "\<lbrakk>closedin (top_of_set U) S; x \<in> U\<rbrakk>
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2434
         \<Longrightarrow> (setdist {x} S = 0 \<longleftrightarrow> S = {} \<or> x \<in> S)"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2435
  by (auto simp: closedin_limpt setdist_eq_0_sing_1 closure_def)
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2436
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2437
lemma setdist_gt_0_closedin:
69922
4a9167f377b0 new material about topology, etc.; also fixes for yesterday's
paulson <lp15@cam.ac.uk>
parents: 69918
diff changeset
  2438
  shows "\<lbrakk>closedin (top_of_set U) S; x \<in> U; S \<noteq> {}; x \<notin> S\<rbrakk>
69618
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2439
         \<Longrightarrow> setdist {x} S > 0"
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2440
  using less_eq_real_def setdist_eq_0_closedin by fastforce
2be1baf40351 moved setdist to more appropriate places
immler
parents: 69617
diff changeset
  2441
80034
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2442
text \<open>A consequence of the results above\<close>
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2443
lemma compact_minkowski_sum_cball:
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2444
  fixes A :: "'a :: heine_borel set"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2445
  assumes "compact A"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2446
  shows   "compact (\<Union>x\<in>A. cball x r)"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2447
proof (cases "A = {}")
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2448
  case False
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2449
  show ?thesis
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2450
  unfolding compact_eq_bounded_closed
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2451
  proof safe
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2452
    have "open (-(\<Union>x\<in>A. cball x r))"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2453
      unfolding open_dist
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2454
    proof safe
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2455
      fix x assume x: "x \<notin> (\<Union>x\<in>A. cball x r)"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2456
      have "\<exists>x'\<in>{x}. \<exists>y\<in>A. dist x' y = setdist {x} A"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2457
        using \<open>A \<noteq> {}\<close> assms
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2458
        by (intro setdist_compact_closed) (auto simp: compact_imp_closed)
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2459
      then obtain y where y: "y \<in> A" "dist x y = setdist {x} A"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2460
        by blast
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2461
      with x have "setdist {x} A > r"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2462
        by (auto simp: dist_commute)
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2463
      moreover have "False" if "dist z x < setdist {x} A - r" "u \<in> A" "z \<in> cball u r" for z u
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2464
        by (smt (verit, del_insts) mem_cball setdist_Lipschitz setdist_sing_in_set that)
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2465
      ultimately
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2466
      show "\<exists>e>0. \<forall>y. dist y x < e \<longrightarrow> y \<in> - (\<Union>x\<in>A. cball x r)"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2467
        by (force intro!: exI[of _ "setdist {x} A - r"])
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2468
    qed
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2469
    thus "closed (\<Union>x\<in>A. cball x r)"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2470
      using closed_open by blast
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2471
  next
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2472
    from assms have "bounded A"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2473
      by (simp add: compact_imp_bounded)
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2474
    then obtain x c where c: "\<And>y. y \<in> A \<Longrightarrow> dist x y \<le> c"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2475
      unfolding bounded_def by blast
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2476
    have "\<forall>y\<in>(\<Union>x\<in>A. cball x r). dist x y \<le> c + r"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2477
    proof safe
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2478
      fix y z assume *: "y \<in> A" "z \<in> cball y r"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2479
      thus "dist x z \<le> c + r"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2480
        using * c[of y] cball_trans mem_cball by blast
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2481
    qed
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2482
    thus "bounded (\<Union>x\<in>A. cball x r)"
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2483
      unfolding bounded_def by blast
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2484
  qed
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2485
qed auto
95b4fb2b5359 New material and a bit of refactoring
paulson <lp15@cam.ac.uk>
parents: 77490
diff changeset
  2486
81128
5b201b24d99b tuned whitespace, to simplify hypersearch;
wenzelm
parents: 80914
diff changeset
  2487
no_notation eucl_less  (infix \<open><e\<close> 50)
54775
2d3df8633dad prefer box over greaterThanLessThan on euclidean_space
immler
parents: 54489
diff changeset
  2488
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
  2489
end