src/HOL/Real/HahnBanach/HahnBanach.thy
changeset 28823 dcbef866c9e2
parent 27612 d3eb431db035
child 29234 60f7fb56f8cd
--- a/src/HOL/Real/HahnBanach/HahnBanach.thy	Mon Nov 17 17:00:27 2008 +0100
+++ b/src/HOL/Real/HahnBanach/HahnBanach.thy	Mon Nov 17 17:00:55 2008 +0100
@@ -369,8 +369,8 @@
   interpret subspace [F E] by fact
   interpret linearform [F f] by fact
   interpret continuous [F norm f] by fact
-  have E: "vectorspace E" by unfold_locales
-  have F: "vectorspace F" by rule unfold_locales
+  have E: "vectorspace E" by intro_locales
+  have F: "vectorspace F" by rule intro_locales
   have F_norm: "normed_vectorspace F norm"
     using FE E_norm by (rule subspace_normed_vs)
   have ge_zero: "0 \<le> \<parallel>f\<parallel>\<hyphen>F"