src/HOL/Multivariate_Analysis/Integration.thy
changeset 36318 3567d0571932
parent 36244 009b0ee1b838
child 36334 068a01b4bc56
--- a/src/HOL/Multivariate_Analysis/Integration.thy	Fri Apr 23 22:48:07 2010 +0200
+++ b/src/HOL/Multivariate_Analysis/Integration.thy	Fri Apr 23 23:33:48 2010 +0200
@@ -3327,7 +3327,7 @@
   using additive_tagged_division_1[OF _ assms(2), of "f o dest_vec1"]
   unfolding o_def vec1_dest_vec1 using assms(1) by auto
 
-lemma split_minus[simp]:"(\<lambda>(x, k). ?f x k) x - (\<lambda>(x, k). ?g x k) x = (\<lambda>(x, k). ?f x k - ?g x k) x"
+lemma split_minus[simp]:"(\<lambda>(x, k). f x k) x - (\<lambda>(x, k). g x k) x = (\<lambda>(x, k). f x k - g x k) x"
   unfolding split_def by(rule refl)
 
 lemma norm_triangle_le_sub: "norm x + norm y \<le> e \<Longrightarrow> norm (x - y) \<le> e"