src/HOL/Real/HahnBanach/Linearform.thy
changeset 9408 d3d56e1d2ec1
parent 9374 153853af318b
child 10687 c186279eecea
--- a/src/HOL/Real/HahnBanach/Linearform.thy	Sun Jul 23 11:59:21 2000 +0200
+++ b/src/HOL/Real/HahnBanach/Linearform.thy	Sun Jul 23 12:01:05 2000 +0200
@@ -22,15 +22,15 @@
  ==> is_linearform V f"
  by (unfold is_linearform_def) force
 
-lemma linearform_add [intro??]: 
+lemma linearform_add [intro?]: 
   "[| is_linearform V f; x \<in> V; y \<in> V |] ==> f (x + y) = f x + f y"
   by (unfold is_linearform_def) fast
 
-lemma linearform_mult [intro??]: 
+lemma linearform_mult [intro?]: 
   "[| is_linearform V f; x \<in> V |] ==>  f (a \<cdot> x) = a * (f x)" 
   by (unfold is_linearform_def) fast
 
-lemma linearform_neg [intro??]:
+lemma linearform_neg [intro?]:
   "[|  is_vectorspace V; is_linearform V f; x \<in> V|] 
   ==> f (- x) = - f x"
 proof - 
@@ -41,7 +41,7 @@
   finally show ?thesis .
 qed
 
-lemma linearform_diff [intro??]: 
+lemma linearform_diff [intro?]: 
   "[| is_vectorspace V; is_linearform V f; x \<in> V; y \<in> V |] 
   ==> f (x - y) = f x - f y"  
 proof -
@@ -55,7 +55,7 @@
 
 text{* Every linear form yields $0$ for the $\zero$ vector.*}
 
-lemma linearform_zero [intro??, simp]: 
+lemma linearform_zero [intro?, simp]: 
   "[| is_vectorspace V; is_linearform V f |] ==> f 0 = #0"
 proof - 
   assume "is_vectorspace V" "is_linearform V f"