src/HOL/Analysis/Linear_Algebra.thy
changeset 73648 1bd3463e30b8
parent 71120 f4579e6800d7
child 73795 8893e0ed263a
equal deleted inserted replaced
73647:a037f01aedab 73648:1bd3463e30b8
  1873     and f :: "'d::t2_space \<Rightarrow> 'a"
  1873     and f :: "'d::t2_space \<Rightarrow> 'a"
  1874   assumes "continuous_on S f" "continuous_on S g" "bilinear h"
  1874   assumes "continuous_on S f" "continuous_on S g" "bilinear h"
  1875   shows "continuous_on S (\<lambda>x. h (f x) (g x))"
  1875   shows "continuous_on S (\<lambda>x. h (f x) (g x))"
  1876   using assms by (simp add: continuous_on_eq_continuous_within bilinear_continuous_compose)
  1876   using assms by (simp add: continuous_on_eq_continuous_within bilinear_continuous_compose)
  1877 
  1877 
  1878 
       
  1879 end
  1878 end