src/HOL/Real/HahnBanach/Linearform.thy
changeset 11701 3d51fbf81c17
parent 10687 c186279eecea
child 12018 ec054019c910
--- a/src/HOL/Real/HahnBanach/Linearform.thy	Fri Oct 05 21:50:37 2001 +0200
+++ b/src/HOL/Real/HahnBanach/Linearform.thy	Fri Oct 05 21:52:39 2001 +0200
@@ -37,8 +37,8 @@
   \<Longrightarrow> f (- x) = - f x"
 proof -
   assume "is_linearform V f"  "is_vectorspace V"  "x \<in> V"
-  have "f (- x) = f ((- #1) \<cdot> x)" by (simp! add: negate_eq1)
-  also have "... = (- #1) * (f x)" by (rule linearform_mult)
+  have "f (- x) = f ((- Numeral1) \<cdot> x)" by (simp! add: negate_eq1)
+  also have "... = (- Numeral1) * (f x)" by (rule linearform_mult)
   also have "... = - (f x)" by (simp!)
   finally show ?thesis .
 qed
@@ -58,14 +58,14 @@
 text {* Every linear form yields @{text 0} for the @{text 0} vector. *}
 
 lemma linearform_zero [intro?, simp]:
-  "is_vectorspace V \<Longrightarrow> is_linearform V f \<Longrightarrow> f 0 = #0"
+  "is_vectorspace V \<Longrightarrow> is_linearform V f \<Longrightarrow> f 0 = Numeral0"
 proof -
   assume "is_vectorspace V"  "is_linearform V f"
   have "f 0 = f (0 - 0)" by (simp!)
   also have "... = f 0 - f 0"
     by (rule linearform_diff) (simp!)+
-  also have "... = #0" by simp
-  finally show "f 0 = #0" .
+  also have "... = Numeral0" by simp
+  finally show "f 0 = Numeral0" .
 qed
 
 end