src/HOL/Analysis/Convex_Euclidean_Space.thy
changeset 63938 f6ce08859d4c
parent 63928 d81fb5b46a5c
child 63945 444eafb6e864
--- a/src/HOL/Analysis/Convex_Euclidean_Space.thy	Wed Sep 21 16:59:51 2016 +0100
+++ b/src/HOL/Analysis/Convex_Euclidean_Space.thy	Thu Sep 22 15:44:47 2016 +0100
@@ -1,5 +1,5 @@
-(*  Title:      HOL/Analysis/Convex_Euclidean_Space.thy
-    Authors: Robert Himmelmann, TU Muenchen; Bogdan Grechuk, University of Edinburgh; LCP
+(*  Author:     L C Paulson, University of Cambridge
+    Authors: Robert Himmelmann, TU Muenchen; Bogdan Grechuk, University of Edinburgh
 *)
 
 section \<open>Convex sets, functions and related things\<close>
@@ -219,7 +219,7 @@
     from gxy have th0: "g (x - y) = 0"
       by (simp add: linear_diff[OF g(1)])
     have th1: "x - y \<in> span B" using x' y'
-      by (metis span_sub)
+      by (metis span_diff)
     have "x = y" using g0[OF th1 th0] by simp
   }
   then have giS: "inj_on g S" unfolding inj_on_def by blast
@@ -2267,7 +2267,7 @@
     apply (rule subset_le_dim)
     unfolding subset_eq
     using \<open>a\<in>s\<close>
-    apply (auto simp add:span_superset span_sub)
+    apply (auto simp add:span_superset span_diff)
     done
   also have "\<dots> < dim s + 1" by auto
   also have "\<dots> \<le> card (s - {a})"