diff -r a0e6bda62b7b -r 3d51fbf81c17 src/HOL/Real/HahnBanach/HahnBanach.thy --- a/src/HOL/Real/HahnBanach/HahnBanach.thy Fri Oct 05 21:50:37 2001 +0200 +++ b/src/HOL/Real/HahnBanach/HahnBanach.thy Fri Oct 05 21:52:39 2001 +0200 @@ -201,7 +201,7 @@ proof (rule graph_extI) fix t assume "t \ H" have "(SOME (y, a). t = y + a \ x' \ y \ H) - = (t, #0)" + = (t, Numeral0)" 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 \ F" have "f x = h x" .. - also have " ... = h x + #0 * xi" by simp + also have " ... = h x + Numeral0 * xi" by simp also - have "... = (let (y, a) = (x, #0) in h y + a * xi)" + have "... = (let (y, a) = (x, Numeral0) in h y + a * xi)" by (simp add: Let_def) also have - "(x, #0) = (SOME (y, a). x = y + a \ x' \ y \ H)" + "(x, Numeral0) = (SOME (y, a). x = y + a \ x' \ y \ H)" by (rule decomp_H'_H [symmetric]) (simp! add: x')+ also have "(let (y, a) = (SOME (y, a). x = y + a \ x' \ y \ H) @@ -372,10 +372,10 @@ txt {* @{text p} is positive definite: *} -show "#0 \ p x" +show "Numeral0 \ p x" proof (unfold p_def, rule real_le_mult_order1a) - from f_cont f_norm show "#0 \ \f\F,norm" .. - show "#0 \ norm x" .. + from f_cont f_norm show "Numeral0 \ \f\F,norm" .. + show "Numeral0 \ norm x" .. qed txt {* @{text p} is absolutely homogenous: *} @@ -402,7 +402,7 @@ also have "... \ \f\F,norm * (norm x + norm y)" proof (rule real_mult_le_le_mono1a) - from f_cont f_norm show "#0 \ \f\F,norm" .. + from f_cont f_norm show "Numeral0 \ \f\F,norm" .. show "norm (x + y) \ norm x + norm y" .. qed also have "... = \f\F,norm * norm x @@ -489,7 +489,7 @@ with g_cont e_norm show "?L \ ?R" proof (rule fnorm_le_ub) - from f_cont f_norm show "#0 \ \f\F,norm" .. + from f_cont f_norm show "Numeral0 \ \f\F,norm" .. qed txt{* The other direction is achieved by a similar @@ -509,7 +509,7 @@ qed thus "?R \ ?L" proof (rule fnorm_le_ub [OF f_cont f_norm]) - from g_cont show "#0 \ \g\E,norm" .. + from g_cont show "Numeral0 \ \g\E,norm" .. qed qed qed