author | wenzelm |
Tue, 03 Sep 2013 11:29:01 +0200 | |
changeset 53375 | 78693e46a237 |
parent 53015 | a1119cf551e8 |
child 53938 | eb93cca4589a |
permissions | -rw-r--r-- |
41959 | 1 |
(* Title: HOL/Library/Inner_Product.thy |
2 |
Author: Brian Huffman |
|
29993 | 3 |
*) |
4 |
||
5 |
header {* Inner Product Spaces and the Gradient Derivative *} |
|
6 |
||
7 |
theory Inner_Product |
|
51642
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
8 |
imports "~~/src/HOL/Complex_Main" |
29993 | 9 |
begin |
10 |
||
11 |
subsection {* Real inner product spaces *} |
|
12 |
||
31492
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
13 |
text {* |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
14 |
Temporarily relax type constraints for @{term "open"}, |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
15 |
@{term dist}, and @{term norm}. |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
16 |
*} |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
17 |
|
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
18 |
setup {* Sign.add_const_constraint |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
19 |
(@{const_name "open"}, SOME @{typ "'a::open set \<Rightarrow> bool"}) *} |
31446 | 20 |
|
21 |
setup {* Sign.add_const_constraint |
|
22 |
(@{const_name dist}, SOME @{typ "'a::dist \<Rightarrow> 'a \<Rightarrow> real"}) *} |
|
23 |
||
24 |
setup {* Sign.add_const_constraint |
|
25 |
(@{const_name norm}, SOME @{typ "'a::norm \<Rightarrow> real"}) *} |
|
26 |
||
31492
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
27 |
class real_inner = real_vector + sgn_div_norm + dist_norm + open_dist + |
29993 | 28 |
fixes inner :: "'a \<Rightarrow> 'a \<Rightarrow> real" |
29 |
assumes inner_commute: "inner x y = inner y x" |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
30 |
and inner_add_left: "inner (x + y) z = inner x z + inner y z" |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
31 |
and inner_scaleR_left [simp]: "inner (scaleR r x) y = r * (inner x y)" |
29993 | 32 |
and inner_ge_zero [simp]: "0 \<le> inner x x" |
33 |
and inner_eq_zero_iff [simp]: "inner x x = 0 \<longleftrightarrow> x = 0" |
|
34 |
and norm_eq_sqrt_inner: "norm x = sqrt (inner x x)" |
|
35 |
begin |
|
36 |
||
37 |
lemma inner_zero_left [simp]: "inner 0 x = 0" |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
38 |
using inner_add_left [of 0 0 x] by simp |
29993 | 39 |
|
40 |
lemma inner_minus_left [simp]: "inner (- x) y = - inner x y" |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
41 |
using inner_add_left [of x "- x" y] by simp |
29993 | 42 |
|
43 |
lemma inner_diff_left: "inner (x - y) z = inner x z - inner y z" |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
44 |
by (simp add: diff_minus inner_add_left) |
29993 | 45 |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
46 |
lemma inner_setsum_left: "inner (\<Sum>x\<in>A. f x) y = (\<Sum>x\<in>A. inner (f x) y)" |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
47 |
by (cases "finite A", induct set: finite, simp_all add: inner_add_left) |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
48 |
|
29993 | 49 |
text {* Transfer distributivity rules to right argument. *} |
50 |
||
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
51 |
lemma inner_add_right: "inner x (y + z) = inner x y + inner x z" |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
52 |
using inner_add_left [of y z x] by (simp only: inner_commute) |
29993 | 53 |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
54 |
lemma inner_scaleR_right [simp]: "inner x (scaleR r y) = r * (inner x y)" |
29993 | 55 |
using inner_scaleR_left [of r y x] by (simp only: inner_commute) |
56 |
||
57 |
lemma inner_zero_right [simp]: "inner x 0 = 0" |
|
58 |
using inner_zero_left [of x] by (simp only: inner_commute) |
|
59 |
||
60 |
lemma inner_minus_right [simp]: "inner x (- y) = - inner x y" |
|
61 |
using inner_minus_left [of y x] by (simp only: inner_commute) |
|
62 |
||
63 |
lemma inner_diff_right: "inner x (y - z) = inner x y - inner x z" |
|
64 |
using inner_diff_left [of y z x] by (simp only: inner_commute) |
|
65 |
||
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
66 |
lemma inner_setsum_right: "inner x (\<Sum>y\<in>A. f y) = (\<Sum>y\<in>A. inner x (f y))" |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
67 |
using inner_setsum_left [of f A x] by (simp only: inner_commute) |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
68 |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
69 |
lemmas inner_add [algebra_simps] = inner_add_left inner_add_right |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
70 |
lemmas inner_diff [algebra_simps] = inner_diff_left inner_diff_right |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
71 |
lemmas inner_scaleR = inner_scaleR_left inner_scaleR_right |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
72 |
|
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
73 |
text {* Legacy theorem names *} |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
74 |
lemmas inner_left_distrib = inner_add_left |
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
75 |
lemmas inner_right_distrib = inner_add_right |
29993 | 76 |
lemmas inner_distrib = inner_left_distrib inner_right_distrib |
77 |
||
78 |
lemma inner_gt_zero_iff [simp]: "0 < inner x x \<longleftrightarrow> x \<noteq> 0" |
|
79 |
by (simp add: order_less_le) |
|
80 |
||
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
81 |
lemma power2_norm_eq_inner: "(norm x)\<^sup>2 = inner x x" |
29993 | 82 |
by (simp add: norm_eq_sqrt_inner) |
83 |
||
30046 | 84 |
lemma Cauchy_Schwarz_ineq: |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
85 |
"(inner x y)\<^sup>2 \<le> inner x x * inner y y" |
29993 | 86 |
proof (cases) |
87 |
assume "y = 0" |
|
88 |
thus ?thesis by simp |
|
89 |
next |
|
90 |
assume y: "y \<noteq> 0" |
|
91 |
let ?r = "inner x y / inner y y" |
|
92 |
have "0 \<le> inner (x - scaleR ?r y) (x - scaleR ?r y)" |
|
93 |
by (rule inner_ge_zero) |
|
94 |
also have "\<dots> = inner x x - inner y x * ?r" |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
95 |
by (simp add: inner_diff) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
96 |
also have "\<dots> = inner x x - (inner x y)\<^sup>2 / inner y y" |
29993 | 97 |
by (simp add: power2_eq_square inner_commute) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
98 |
finally have "0 \<le> inner x x - (inner x y)\<^sup>2 / inner y y" . |
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
99 |
hence "(inner x y)\<^sup>2 / inner y y \<le> inner x x" |
29993 | 100 |
by (simp add: le_diff_eq) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
101 |
thus "(inner x y)\<^sup>2 \<le> inner x x * inner y y" |
29993 | 102 |
by (simp add: pos_divide_le_eq y) |
103 |
qed |
|
104 |
||
30046 | 105 |
lemma Cauchy_Schwarz_ineq2: |
29993 | 106 |
"\<bar>inner x y\<bar> \<le> norm x * norm y" |
107 |
proof (rule power2_le_imp_le) |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
108 |
have "(inner x y)\<^sup>2 \<le> inner x x * inner y y" |
30046 | 109 |
using Cauchy_Schwarz_ineq . |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
110 |
thus "\<bar>inner x y\<bar>\<^sup>2 \<le> (norm x * norm y)\<^sup>2" |
29993 | 111 |
by (simp add: power_mult_distrib power2_norm_eq_inner) |
112 |
show "0 \<le> norm x * norm y" |
|
113 |
unfolding norm_eq_sqrt_inner |
|
114 |
by (intro mult_nonneg_nonneg real_sqrt_ge_zero inner_ge_zero) |
|
115 |
qed |
|
116 |
||
117 |
subclass real_normed_vector |
|
118 |
proof |
|
119 |
fix a :: real and x y :: 'a |
|
120 |
show "norm x = 0 \<longleftrightarrow> x = 0" |
|
121 |
unfolding norm_eq_sqrt_inner by simp |
|
122 |
show "norm (x + y) \<le> norm x + norm y" |
|
123 |
proof (rule power2_le_imp_le) |
|
124 |
have "inner x y \<le> norm x * norm y" |
|
30046 | 125 |
by (rule order_trans [OF abs_ge_self Cauchy_Schwarz_ineq2]) |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
126 |
thus "(norm (x + y))\<^sup>2 \<le> (norm x + norm y)\<^sup>2" |
29993 | 127 |
unfolding power2_sum power2_norm_eq_inner |
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
128 |
by (simp add: inner_add inner_commute) |
29993 | 129 |
show "0 \<le> norm x + norm y" |
44126 | 130 |
unfolding norm_eq_sqrt_inner by simp |
29993 | 131 |
qed |
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
132 |
have "sqrt (a\<^sup>2 * inner x x) = \<bar>a\<bar> * sqrt (inner x x)" |
29993 | 133 |
by (simp add: real_sqrt_mult_distrib) |
134 |
then show "norm (a *\<^sub>R x) = \<bar>a\<bar> * norm x" |
|
135 |
unfolding norm_eq_sqrt_inner |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
136 |
by (simp add: power2_eq_square mult_assoc) |
29993 | 137 |
qed |
138 |
||
139 |
end |
|
140 |
||
31492
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
141 |
text {* |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
142 |
Re-enable constraints for @{term "open"}, |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
143 |
@{term dist}, and @{term norm}. |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
144 |
*} |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
145 |
|
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
146 |
setup {* Sign.add_const_constraint |
5400beeddb55
replace 'topo' with 'open'; add extra type constraint for 'open'
huffman
parents:
31446
diff
changeset
|
147 |
(@{const_name "open"}, SOME @{typ "'a::topological_space set \<Rightarrow> bool"}) *} |
31446 | 148 |
|
149 |
setup {* Sign.add_const_constraint |
|
150 |
(@{const_name dist}, SOME @{typ "'a::metric_space \<Rightarrow> 'a \<Rightarrow> real"}) *} |
|
151 |
||
152 |
setup {* Sign.add_const_constraint |
|
153 |
(@{const_name norm}, SOME @{typ "'a::real_normed_vector \<Rightarrow> real"}) *} |
|
154 |
||
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
155 |
lemma bounded_bilinear_inner: |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
156 |
"bounded_bilinear (inner::'a::real_inner \<Rightarrow> 'a \<Rightarrow> real)" |
29993 | 157 |
proof |
158 |
fix x y z :: 'a and r :: real |
|
159 |
show "inner (x + y) z = inner x z + inner y z" |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
160 |
by (rule inner_add_left) |
29993 | 161 |
show "inner x (y + z) = inner x y + inner x z" |
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
162 |
by (rule inner_add_right) |
29993 | 163 |
show "inner (scaleR r x) y = scaleR r (inner x y)" |
164 |
unfolding real_scaleR_def by (rule inner_scaleR_left) |
|
165 |
show "inner x (scaleR r y) = scaleR r (inner x y)" |
|
166 |
unfolding real_scaleR_def by (rule inner_scaleR_right) |
|
167 |
show "\<exists>K. \<forall>x y::'a. norm (inner x y) \<le> norm x * norm y * K" |
|
168 |
proof |
|
169 |
show "\<forall>x y::'a. norm (inner x y) \<le> norm x * norm y * 1" |
|
30046 | 170 |
by (simp add: Cauchy_Schwarz_ineq2) |
29993 | 171 |
qed |
172 |
qed |
|
173 |
||
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
174 |
lemmas tendsto_inner [tendsto_intros] = |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
175 |
bounded_bilinear.tendsto [OF bounded_bilinear_inner] |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
176 |
|
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
177 |
lemmas isCont_inner [simp] = |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
178 |
bounded_bilinear.isCont [OF bounded_bilinear_inner] |
29993 | 179 |
|
51642
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
180 |
lemmas FDERIV_inner [FDERIV_intros] = |
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
181 |
bounded_bilinear.FDERIV [OF bounded_bilinear_inner] |
29993 | 182 |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
183 |
lemmas bounded_linear_inner_left = |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
184 |
bounded_bilinear.bounded_linear_left [OF bounded_bilinear_inner] |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
185 |
|
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
186 |
lemmas bounded_linear_inner_right = |
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
187 |
bounded_bilinear.bounded_linear_right [OF bounded_bilinear_inner] |
44233 | 188 |
|
51642
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
189 |
lemmas FDERIV_inner_right [FDERIV_intros] = |
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
190 |
bounded_linear.FDERIV [OF bounded_linear_inner_right] |
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
191 |
|
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
192 |
lemmas FDERIV_inner_left [FDERIV_intros] = |
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
193 |
bounded_linear.FDERIV [OF bounded_linear_inner_left] |
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
194 |
|
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
195 |
lemma differentiable_inner [simp]: |
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
196 |
"f differentiable x in s \<Longrightarrow> g differentiable x in s \<Longrightarrow> (\<lambda>x. inner (f x) (g x)) differentiable x in s" |
400ec5ae7f8f
move FrechetDeriv from the Library to HOL/Deriv; base DERIV on FDERIV and both derivatives allow a restricted support set; FDERIV is now an abbreviation of has_derivative
hoelzl
parents:
51002
diff
changeset
|
197 |
unfolding isDiff_def by (blast intro: FDERIV_inner) |
29993 | 198 |
|
199 |
subsection {* Class instances *} |
|
200 |
||
201 |
instantiation real :: real_inner |
|
202 |
begin |
|
203 |
||
204 |
definition inner_real_def [simp]: "inner = op *" |
|
205 |
||
206 |
instance proof |
|
207 |
fix x y z r :: real |
|
208 |
show "inner x y = inner y x" |
|
209 |
unfolding inner_real_def by (rule mult_commute) |
|
210 |
show "inner (x + y) z = inner x z + inner y z" |
|
49962
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
webertj
parents:
44902
diff
changeset
|
211 |
unfolding inner_real_def by (rule distrib_right) |
29993 | 212 |
show "inner (scaleR r x) y = r * inner x y" |
213 |
unfolding inner_real_def real_scaleR_def by (rule mult_assoc) |
|
214 |
show "0 \<le> inner x x" |
|
215 |
unfolding inner_real_def by simp |
|
216 |
show "inner x x = 0 \<longleftrightarrow> x = 0" |
|
217 |
unfolding inner_real_def by simp |
|
218 |
show "norm x = sqrt (inner x x)" |
|
219 |
unfolding inner_real_def by simp |
|
220 |
qed |
|
221 |
||
222 |
end |
|
223 |
||
224 |
instantiation complex :: real_inner |
|
225 |
begin |
|
226 |
||
227 |
definition inner_complex_def: |
|
228 |
"inner x y = Re x * Re y + Im x * Im y" |
|
229 |
||
230 |
instance proof |
|
231 |
fix x y z :: complex and r :: real |
|
232 |
show "inner x y = inner y x" |
|
233 |
unfolding inner_complex_def by (simp add: mult_commute) |
|
234 |
show "inner (x + y) z = inner x z + inner y z" |
|
49962
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
webertj
parents:
44902
diff
changeset
|
235 |
unfolding inner_complex_def by (simp add: distrib_right) |
29993 | 236 |
show "inner (scaleR r x) y = r * inner x y" |
49962
a8cc904a6820
Renamed {left,right}_distrib to distrib_{right,left}.
webertj
parents:
44902
diff
changeset
|
237 |
unfolding inner_complex_def by (simp add: distrib_left) |
29993 | 238 |
show "0 \<le> inner x x" |
44126 | 239 |
unfolding inner_complex_def by simp |
29993 | 240 |
show "inner x x = 0 \<longleftrightarrow> x = 0" |
241 |
unfolding inner_complex_def |
|
242 |
by (simp add: add_nonneg_eq_0_iff complex_Re_Im_cancel_iff) |
|
243 |
show "norm x = sqrt (inner x x)" |
|
244 |
unfolding inner_complex_def complex_norm_def |
|
245 |
by (simp add: power2_eq_square) |
|
246 |
qed |
|
247 |
||
248 |
end |
|
249 |
||
44902
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
250 |
lemma complex_inner_1 [simp]: "inner 1 x = Re x" |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
251 |
unfolding inner_complex_def by simp |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
252 |
|
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
253 |
lemma complex_inner_1_right [simp]: "inner x 1 = Re x" |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
254 |
unfolding inner_complex_def by simp |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
255 |
|
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
256 |
lemma complex_inner_ii_left [simp]: "inner ii x = Im x" |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
257 |
unfolding inner_complex_def by simp |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
258 |
|
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
259 |
lemma complex_inner_ii_right [simp]: "inner x ii = Im x" |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
260 |
unfolding inner_complex_def by simp |
9ba11d41cd1f
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
huffman
parents:
44282
diff
changeset
|
261 |
|
29993 | 262 |
|
263 |
subsection {* Gradient derivative *} |
|
264 |
||
265 |
definition |
|
266 |
gderiv :: |
|
267 |
"['a::real_inner \<Rightarrow> real, 'a, 'a] \<Rightarrow> bool" |
|
268 |
("(GDERIV (_)/ (_)/ :> (_))" [1000, 1000, 60] 60) |
|
269 |
where |
|
270 |
"GDERIV f x :> D \<longleftrightarrow> FDERIV f x :> (\<lambda>h. inner h D)" |
|
271 |
||
272 |
lemma gderiv_deriv [simp]: "GDERIV f x :> D \<longleftrightarrow> DERIV f x :> D" |
|
273 |
by (simp only: gderiv_def deriv_fderiv inner_real_def) |
|
274 |
||
275 |
lemma GDERIV_DERIV_compose: |
|
276 |
"\<lbrakk>GDERIV f x :> df; DERIV g (f x) :> dg\<rbrakk> |
|
277 |
\<Longrightarrow> GDERIV (\<lambda>x. g (f x)) x :> scaleR dg df" |
|
278 |
unfolding gderiv_def deriv_fderiv |
|
279 |
apply (drule (1) FDERIV_compose) |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
280 |
apply (simp add: mult_ac) |
29993 | 281 |
done |
282 |
||
283 |
lemma FDERIV_subst: "\<lbrakk>FDERIV f x :> df; df = d\<rbrakk> \<Longrightarrow> FDERIV f x :> d" |
|
284 |
by simp |
|
285 |
||
286 |
lemma GDERIV_subst: "\<lbrakk>GDERIV f x :> df; df = d\<rbrakk> \<Longrightarrow> GDERIV f x :> d" |
|
287 |
by simp |
|
288 |
||
289 |
lemma GDERIV_const: "GDERIV (\<lambda>x. k) x :> 0" |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
290 |
unfolding gderiv_def inner_zero_right by (rule FDERIV_const) |
29993 | 291 |
|
292 |
lemma GDERIV_add: |
|
293 |
"\<lbrakk>GDERIV f x :> df; GDERIV g x :> dg\<rbrakk> |
|
294 |
\<Longrightarrow> GDERIV (\<lambda>x. f x + g x) x :> df + dg" |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
295 |
unfolding gderiv_def inner_add_right by (rule FDERIV_add) |
29993 | 296 |
|
297 |
lemma GDERIV_minus: |
|
298 |
"GDERIV f x :> df \<Longrightarrow> GDERIV (\<lambda>x. - f x) x :> - df" |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
299 |
unfolding gderiv_def inner_minus_right by (rule FDERIV_minus) |
29993 | 300 |
|
301 |
lemma GDERIV_diff: |
|
302 |
"\<lbrakk>GDERIV f x :> df; GDERIV g x :> dg\<rbrakk> |
|
303 |
\<Longrightarrow> GDERIV (\<lambda>x. f x - g x) x :> df - dg" |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
304 |
unfolding gderiv_def inner_diff_right by (rule FDERIV_diff) |
29993 | 305 |
|
306 |
lemma GDERIV_scaleR: |
|
307 |
"\<lbrakk>DERIV f x :> df; GDERIV g x :> dg\<rbrakk> |
|
308 |
\<Longrightarrow> GDERIV (\<lambda>x. scaleR (f x) (g x)) x |
|
309 |
:> (scaleR (f x) dg + scaleR df (g x))" |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
310 |
unfolding gderiv_def deriv_fderiv inner_add_right inner_scaleR_right |
29993 | 311 |
apply (rule FDERIV_subst) |
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
312 |
apply (erule (1) FDERIV_scaleR) |
29993 | 313 |
apply (simp add: mult_ac) |
314 |
done |
|
315 |
||
316 |
lemma GDERIV_mult: |
|
317 |
"\<lbrakk>GDERIV f x :> df; GDERIV g x :> dg\<rbrakk> |
|
318 |
\<Longrightarrow> GDERIV (\<lambda>x. f x * g x) x :> scaleR (f x) dg + scaleR (g x) df" |
|
319 |
unfolding gderiv_def |
|
320 |
apply (rule FDERIV_subst) |
|
321 |
apply (erule (1) FDERIV_mult) |
|
31590
776d6a4c1327
declare inner_add, inner_diff [algebra_simps]; declare inner_scaleR [simp]
huffman
parents:
31492
diff
changeset
|
322 |
apply (simp add: inner_add mult_ac) |
29993 | 323 |
done |
324 |
||
325 |
lemma GDERIV_inverse: |
|
326 |
"\<lbrakk>GDERIV f x :> df; f x \<noteq> 0\<rbrakk> |
|
53015
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents:
51642
diff
changeset
|
327 |
\<Longrightarrow> GDERIV (\<lambda>x. inverse (f x)) x :> - (inverse (f x))\<^sup>2 *\<^sub>R df" |
29993 | 328 |
apply (erule GDERIV_DERIV_compose) |
329 |
apply (erule DERIV_inverse [folded numeral_2_eq_2]) |
|
330 |
done |
|
331 |
||
332 |
lemma GDERIV_norm: |
|
333 |
assumes "x \<noteq> 0" shows "GDERIV (\<lambda>x. norm x) x :> sgn x" |
|
334 |
proof - |
|
335 |
have 1: "FDERIV (\<lambda>x. inner x x) x :> (\<lambda>h. inner x h + inner h x)" |
|
44282
f0de18b62d63
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman
parents:
44233
diff
changeset
|
336 |
by (intro FDERIV_inner FDERIV_ident) |
29993 | 337 |
have 2: "(\<lambda>h. inner x h + inner h x) = (\<lambda>h. inner h (scaleR 2 x))" |
39302
d7728f65b353
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
nipkow
parents:
39198
diff
changeset
|
338 |
by (simp add: fun_eq_iff inner_commute) |
29993 | 339 |
have "0 < inner x x" using `x \<noteq> 0` by simp |
340 |
then have 3: "DERIV sqrt (inner x x) :> (inverse (sqrt (inner x x)) / 2)" |
|
341 |
by (rule DERIV_real_sqrt) |
|
342 |
have 4: "(inverse (sqrt (inner x x)) / 2) *\<^sub>R 2 *\<^sub>R x = sgn x" |
|
343 |
by (simp add: sgn_div_norm norm_eq_sqrt_inner) |
|
344 |
show ?thesis |
|
345 |
unfolding norm_eq_sqrt_inner |
|
346 |
apply (rule GDERIV_subst [OF _ 4]) |
|
347 |
apply (rule GDERIV_DERIV_compose [where g=sqrt and df="scaleR 2 x"]) |
|
348 |
apply (subst gderiv_def) |
|
349 |
apply (rule FDERIV_subst [OF _ 2]) |
|
350 |
apply (rule 1) |
|
351 |
apply (rule 3) |
|
352 |
done |
|
353 |
qed |
|
354 |
||
355 |
lemmas FDERIV_norm = GDERIV_norm [unfolded gderiv_def] |
|
356 |
||
357 |
end |