src/HOL/Multivariate_Analysis/Linear_Algebra.thy
changeset 63148 6a767355d1a9
parent 63114 27afe7af7379
child 63170 eae6549dbea2
--- a/src/HOL/Multivariate_Analysis/Linear_Algebra.thy	Wed May 25 13:13:35 2016 +0200
+++ b/src/HOL/Multivariate_Analysis/Linear_Algebra.thy	Wed May 25 16:01:42 2016 +0200
@@ -978,8 +978,8 @@
     using \<open>independent B'\<close>
     by (rule independentD_unique[OF _ X(2) X(1)]) (auto intro: X simp: X(3)[symmetric])
 
-  def f' \<equiv> "\<lambda>y. if y \<in> B then f y else 0"
-  def g \<equiv> "\<lambda>y. \<Sum>x|X y x \<noteq> 0. X y x *\<^sub>R f' x"
+  define f' where "f' y = (if y \<in> B then f y else 0)" for y
+  define g where "g y = (\<Sum>x|X y x \<noteq> 0. X y x *\<^sub>R f' x)" for y
 
   have g_f': "x \<in> B' \<Longrightarrow> g x = f' x" for x
     by (auto simp: g_def X_B')