diff -r d01983034ded -r 247615bfffb8 src/HOL/Real/HahnBanach/FunctionNorm.thy --- a/src/HOL/Real/HahnBanach/FunctionNorm.thy Thu May 06 20:43:30 2004 +0200 +++ b/src/HOL/Real/HahnBanach/FunctionNorm.thy Fri May 07 12:16:57 2004 +0200 @@ -137,7 +137,7 @@ by (rule real_mult_assoc) also from gt have "\x\ \ 0" by simp - hence "\x\ * inverse \x\ = 1" by (simp add: real_mult_inv_right1) + hence "\x\ * inverse \x\ = 1" by simp also have "c * 1 \ b" by (simp add: b_def le_maxI1) finally show "y \ b" . qed @@ -199,13 +199,11 @@ then have "\f x\ = \f 0\" by simp also have "f 0 = 0" .. also have "\\\ = 0" by simp - also have "\ \ \f\\V * \x\" - proof (rule real_le_mult_order1a) - show "0 \ \f\\V" + also have a: "0 \ \f\\V" by (unfold B_def fn_norm_def) (rule fn_norm_ge_zero [OF _ continuous.intro]) - show "0 \ norm x" .. - qed + have "0 \ norm x" .. + with a have "0 \ \f\\V * \x\" by (simp add: zero_le_mult_iff) finally show "\f x\ \ \f\\V * \x\" . next assume "x \ 0"