src/HOL/Analysis/Linear_Algebra.thy
changeset 70999 5b753486c075
parent 70817 dd675800469d
child 71040 9d2753406c60
equal deleted inserted replaced
70988:38ade730f6df 70999:5b753486c075
   643   then interpret f: bounded_linear f .
   643   then interpret f: bounded_linear f .
   644   show "linear f" ..
   644   show "linear f" ..
   645 qed
   645 qed
   646 
   646 
   647 lemmas linear_linear = linear_conv_bounded_linear[symmetric]
   647 lemmas linear_linear = linear_conv_bounded_linear[symmetric]
       
   648 
       
   649 lemma inj_linear_imp_inv_bounded_linear:
       
   650   fixes f::"'a::euclidean_space \<Rightarrow> 'a"
       
   651   shows "\<lbrakk>bounded_linear f; inj f\<rbrakk> \<Longrightarrow> bounded_linear (inv f)"
       
   652   by (simp add: inj_linear_imp_inv_linear linear_linear)
   648 
   653 
   649 lemma linear_bounded_pos:
   654 lemma linear_bounded_pos:
   650   fixes f :: "'a::euclidean_space \<Rightarrow> 'b::real_normed_vector"
   655   fixes f :: "'a::euclidean_space \<Rightarrow> 'b::real_normed_vector"
   651   assumes lf: "linear f"
   656   assumes lf: "linear f"
   652  obtains B where "B > 0" "\<And>x. norm (f x) \<le> B * norm x"
   657  obtains B where "B > 0" "\<And>x. norm (f x) \<le> B * norm x"