src/HOL/Real/HahnBanach/HahnBanach.thy
changeset 12018 ec054019c910
parent 11701 3d51fbf81c17
child 13515 a6a7025fd7e8
--- a/src/HOL/Real/HahnBanach/HahnBanach.thy	Thu Nov 01 21:12:13 2001 +0100
+++ b/src/HOL/Real/HahnBanach/HahnBanach.thy	Fri Nov 02 17:55:24 2001 +0100
@@ -201,7 +201,7 @@
               proof (rule graph_extI)
                 fix t assume "t \<in> H"
                 have "(SOME (y, a). t = y + a \<cdot> x' \<and> y \<in> H)
-                     = (t, Numeral0)"
+                     = (t, 0)"
                   by (rule decomp_H'_H) (assumption+, rule x')
                 thus "h t = h' t" by (simp! add: Let_def)
               next
@@ -255,12 +255,12 @@
               proof (rule graph_extI)
                 fix x assume "x \<in> F"
                 have "f x = h x" ..
-                also have " ... = h x + Numeral0 * xi" by simp
+                also have " ... = h x + 0 * xi" by simp
                 also
-                have "... = (let (y, a) = (x, Numeral0) in h y + a * xi)"
+                have "... = (let (y, a) = (x, 0) in h y + a * xi)"
                   by (simp add: Let_def)
                 also have
-                  "(x, Numeral0) = (SOME (y, a). x = y + a \<cdot> x' \<and> y \<in> H)"
+                  "(x, 0) = (SOME (y, a). x = y + a \<cdot> x' \<and> y \<in> H)"
                   by (rule decomp_H'_H [symmetric]) (simp! add: x')+
                 also have
                   "(let (y, a) = (SOME (y, a). x = y + a \<cdot> x' \<and> y \<in> H)
@@ -372,10 +372,10 @@
 
 txt {* @{text p} is positive definite: *}
 
-show "Numeral0 \<le> p x"
+show "0 \<le> p x"
 proof (unfold p_def, rule real_le_mult_order1a)
-  from f_cont f_norm show "Numeral0 \<le> \<parallel>f\<parallel>F,norm" ..
-  show "Numeral0 \<le> norm x" ..
+  from f_cont f_norm show "0 \<le> \<parallel>f\<parallel>F,norm" ..
+  show "0 \<le> norm x" ..
 qed
 
 txt {* @{text p} is absolutely homogenous: *}
@@ -402,7 +402,7 @@
   also
   have "... \<le> \<parallel>f\<parallel>F,norm * (norm x + norm y)"
   proof (rule real_mult_le_le_mono1a)
-    from f_cont f_norm show "Numeral0 \<le> \<parallel>f\<parallel>F,norm" ..
+    from f_cont f_norm show "0 \<le> \<parallel>f\<parallel>F,norm" ..
     show "norm (x + y) \<le> norm x + norm y" ..
   qed
   also have "... = \<parallel>f\<parallel>F,norm * norm x
@@ -489,7 +489,7 @@
 
     with g_cont e_norm show "?L \<le> ?R"
     proof (rule fnorm_le_ub)
-      from f_cont f_norm show "Numeral0 \<le> \<parallel>f\<parallel>F,norm" ..
+      from f_cont f_norm show "0 \<le> \<parallel>f\<parallel>F,norm" ..
     qed
 
     txt{* The other direction is achieved by a similar
@@ -509,7 +509,7 @@
     qed
     thus "?R \<le> ?L"
     proof (rule fnorm_le_ub [OF f_cont f_norm])
-      from g_cont show "Numeral0 \<le> \<parallel>g\<parallel>E,norm" ..
+      from g_cont show "0 \<le> \<parallel>g\<parallel>E,norm" ..
     qed
   qed
 qed