src/HOL/Real/HahnBanach/NormedSpace.thy
changeset 14254 342634f38451
parent 13547 bf399f3bd7dc
child 16417 9bc16273c2d4
--- a/src/HOL/Real/HahnBanach/NormedSpace.thy	Fri Oct 31 06:54:22 2003 +0100
+++ b/src/HOL/Real/HahnBanach/NormedSpace.thy	Thu Nov 06 14:18:05 2003 +0100
@@ -23,6 +23,8 @@
     and abs_homogenous [iff?]: "x \<in> V \<Longrightarrow> \<parallel>a \<cdot> x\<parallel> = \<bar>a\<bar> * \<parallel>x\<parallel>"
     and subadditive [iff?]: "x \<in> V \<Longrightarrow> y \<in> V \<Longrightarrow> \<parallel>x + y\<parallel> \<le> \<parallel>x\<parallel> + \<parallel>y\<parallel>"
 
+declare seminorm.intro [intro?]
+
 lemma (in seminorm) diff_subadditive:
   includes vectorspace
   shows "x \<in> V \<Longrightarrow> y \<in> V \<Longrightarrow> \<parallel>x - y\<parallel> \<le> \<parallel>x\<parallel> + \<parallel>y\<parallel>"
@@ -71,6 +73,8 @@
 
 locale normed_vectorspace = vectorspace + norm
 
+declare normed_vectorspace.intro [intro?]
+
 lemma (in normed_vectorspace) gt_zero [intro?]:
   "x \<in> V \<Longrightarrow> x \<noteq> 0 \<Longrightarrow> 0 < \<parallel>x\<parallel>"
 proof -