src/HOL/Hyperreal/FrechetDeriv.thy
changeset 28823 dcbef866c9e2
parent 27611 2c01c0bdb385
child 28866 30cd9d89a0fb
--- a/src/HOL/Hyperreal/FrechetDeriv.thy	Mon Nov 17 17:00:27 2008 +0100
+++ b/src/HOL/Hyperreal/FrechetDeriv.thy	Mon Nov 17 17:00:55 2008 +0100
@@ -31,7 +31,7 @@
 
 lemma bounded_linear_zero:
   "bounded_linear (\<lambda>x::'a::real_normed_vector. 0::'b::real_normed_vector)"
-proof (unfold_locales)
+proof
   show "(0::'b) = 0 + 0" by simp
   fix r show "(0::'b) = scaleR r 0" by simp
   have "\<forall>x::'a. norm (0::'b) \<le> norm x * 0" by simp
@@ -43,7 +43,7 @@
 
 lemma bounded_linear_ident:
   "bounded_linear (\<lambda>x::'a::real_normed_vector. x)"
-proof (unfold_locales)
+proof
   fix x y :: 'a show "x + y = x + y" by simp
   fix r and x :: 'a show "scaleR r x = scaleR r x" by simp
   have "\<forall>x::'a. norm x \<le> norm x * 1" by simp