diff -r 23a8c5ac35f8 -r 69916a850301 src/HOL/Hahn_Banach/Hahn_Banach.thy --- a/src/HOL/Hahn_Banach/Hahn_Banach.thy Sat Oct 17 01:05:59 2009 +0200 +++ b/src/HOL/Hahn_Banach/Hahn_Banach.thy Sat Oct 17 14:43:18 2009 +0200 @@ -202,7 +202,7 @@ proof (rule graph_extI) fix t assume t: "t \ H" from E HE t have "(SOME (y, a). t = y + a \ x' \ y \ H) = (t, 0)" - using `x' \ H` `x' \ E` `x' \ 0` by (rule decomp_H'_H) + using `x' \ H` `x' \ E` `x' \ 0` by (rule decomp_H'_H) with h'_def show "h t = h' t" by (simp add: Let_def) next from HH' show "H \ H'" .. @@ -216,7 +216,7 @@ proof assume eq: "graph H h = graph H' h'" have "x' \ H'" - unfolding H'_def + unfolding H'_def proof from H show "0 \ H" by (rule vectorspace.zero) from x'E show "x' \ lin x'" by (rule x_lin_x) @@ -236,10 +236,10 @@ show "graph H' h' \ norm_pres_extensions E p F f" proof (rule norm_pres_extensionI2) show "linearform H' h'" - using h'_def H'_def HE linearform `x' \ H` `x' \ E` `x' \ 0` E - by (rule h'_lf) + using h'_def H'_def HE linearform `x' \ H` `x' \ E` `x' \ 0` E + by (rule h'_lf) show "H' \ E" - unfolding H'_def + unfolding H'_def proof show "H \ E" by fact show "vectorspace E" by fact @@ -256,12 +256,12 @@ by (simp add: Let_def) also have "(x, 0) = (SOME (y, a). x = y + a \ x' \ y \ H)" - using E HE + using E HE proof (rule decomp_H'_H [symmetric]) from FH x show "x \ H" .. from x' show "x' \ 0" . - show "x' \ H" by fact - show "x' \ E" by fact + show "x' \ H" by fact + show "x' \ E" by fact qed also have "(let (y, a) = (SOME (y, a). x = y + a \ x' \ y \ H) @@ -271,9 +271,9 @@ from FH' show "F \ H'" .. qed show "\x \ H'. h' x \ p x" - using h'_def H'_def `x' \ H` `x' \ E` `x' \ 0` E HE - `seminorm E p` linearform and hp xi - by (rule h'_norm_pres) + using h'_def H'_def `x' \ H` `x' \ E` `x' \ 0` E HE + `seminorm E p` linearform and hp xi + by (rule h'_norm_pres) qed qed ultimately show ?thesis .. @@ -483,23 +483,23 @@ show "\f\\F \ \g\\E" proof (rule normed_vectorspace_with_fn_norm.fn_norm_least - [OF normed_vectorspace_with_fn_norm.intro, - OF F_norm, folded B_def fn_norm_def]) + [OF normed_vectorspace_with_fn_norm.intro, + OF F_norm, folded B_def fn_norm_def]) show "\x \ F. \f x\ \ \g\\E * \x\" proof - fix x assume x: "x \ F" - from a x have "g x = f x" .. - then have "\f x\ = \g x\" by (simp only:) - also from g_cont - have "\ \ \g\\E * \x\" - proof (rule fn_norm_le_cong [OF _ linearformE, folded B_def fn_norm_def]) - from FE x show "x \ E" .. - qed - finally show "\f x\ \ \g\\E * \x\" . + fix x assume x: "x \ F" + from a x have "g x = f x" .. + then have "\f x\ = \g x\" by (simp only:) + also from g_cont + have "\ \ \g\\E * \x\" + proof (rule fn_norm_le_cong [OF _ linearformE, folded B_def fn_norm_def]) + from FE x show "x \ E" .. + qed + finally show "\f x\ \ \g\\E * \x\" . qed show "0 \ \g\\E" - using g_cont - by (rule fn_norm_ge_zero [of g, folded B_def fn_norm_def]) + using g_cont + by (rule fn_norm_ge_zero [of g, folded B_def fn_norm_def]) show "continuous F norm f" by fact qed qed