src/HOL/Multivariate_Analysis/Euclidean_Space.thy
changeset 44128 e6c6ca74d81b
parent 43968 1fe23cfca01f
child 44129 286bd57858b9
--- a/src/HOL/Multivariate_Analysis/Euclidean_Space.thy	Tue Aug 09 12:50:22 2011 -0700
+++ b/src/HOL/Multivariate_Analysis/Euclidean_Space.thy	Tue Aug 09 13:09:35 2011 -0700
@@ -1731,8 +1731,10 @@
 
 end
 
-interpretation euclidean_component: additive "\<lambda>x. euclidean_component x i"
-proof qed (simp add: euclidean_component_def inner_right.add)
+interpretation euclidean_component:
+  bounded_linear "\<lambda>x. euclidean_component x i"
+  unfolding euclidean_component_def
+  by (rule inner.bounded_linear_right)
 
 subsection{* Euclidean Spaces as Typeclass *}