src/HOL/Real/HahnBanach/FunctionNorm.thy
author paulson
Fri, 15 Sep 2000 12:39:57 +0200
changeset 9969 4753185f1dd2
parent 9503 3324cbbecef8
child 9998 09bf8fcd1c6e
permissions -rw-r--r--
renamed (most of...) the select rules
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
     1
(*  Title:      HOL/Real/HahnBanach/FunctionNorm.thy
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
     2
    ID:         $Id$
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
     3
    Author:     Gertrud Bauer, TU Munich
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
     4
*)
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
     5
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
     6
header {* The norm of a function *}
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
     7
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
     8
theory FunctionNorm = NormedSpace + FunctionOrder:
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
     9
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    10
subsection {* Continuous linear forms*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    11
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    12
text{* A linear form $f$ on a normed vector space $(V, \norm{\cdot})$
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    13
is \emph{continuous}, iff it is bounded, i.~e.
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    14
\[\Ex {c\in R}{\All {x\in V} {|f\ap x| \leq c \cdot \norm x}}\]
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    15
In our application no other functions than linear forms are considered,
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    16
so we can define continuous linear forms as bounded linear forms:
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    17
*}
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    18
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    19
constdefs
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    20
  is_continuous ::
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    21
  "['a::{plus, minus, zero} set, 'a => real, 'a => real] => bool" 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    22
  "is_continuous V norm f == 
9503
wenzelm
parents: 9408
diff changeset
    23
    is_linearform V f \<and> (\<exists>c. \<forall>x \<in> V. |f x| <= c * norm x)"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    24
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    25
lemma continuousI [intro]: 
9503
wenzelm
parents: 9408
diff changeset
    26
  "[| is_linearform V f; !! x. x \<in> V ==> |f x| <= c * norm x |] 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    27
  ==> is_continuous V norm f"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    28
proof (unfold is_continuous_def, intro exI conjI ballI)
9503
wenzelm
parents: 9408
diff changeset
    29
  assume r: "!! x. x \<in> V ==> |f x| <= c * norm x" 
wenzelm
parents: 9408
diff changeset
    30
  fix x assume "x \<in> V" show "|f x| <= c * norm x" by (rule r)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    31
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    32
  
9408
d3d56e1d2ec1 classical atts now intro! / intro / intro?;
wenzelm
parents: 9394
diff changeset
    33
lemma continuous_linearform [intro?]: 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    34
  "is_continuous V norm f ==> is_linearform V f"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    35
  by (unfold is_continuous_def) force
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    36
9408
d3d56e1d2ec1 classical atts now intro! / intro / intro?;
wenzelm
parents: 9394
diff changeset
    37
lemma continuous_bounded [intro?]:
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    38
  "is_continuous V norm f 
9503
wenzelm
parents: 9408
diff changeset
    39
  ==> \<exists>c. \<forall>x \<in> V. |f x| <= c * norm x"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    40
  by (unfold is_continuous_def) force
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    41
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    42
subsection{* The norm of a linear form *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    43
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    44
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    45
text{* The least real number $c$ for which holds
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    46
\[\All {x\in V}{|f\ap x| \leq c \cdot \norm x}\]
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    47
is called the \emph{norm} of $f$.
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    48
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    49
For non-trivial vector spaces $V \neq \{\zero\}$ the norm can be defined as 
7927
b50446a33c16 update by Gertrud Bauer;
wenzelm
parents: 7917
diff changeset
    50
\[\fnorm {f} =\sup_{x\neq\zero}\frac{|f\ap x|}{\norm x} \] 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    51
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    52
For the case $V = \{\zero\}$ the supremum would be taken from an
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    53
empty set. Since $\bbbR$ is unbounded, there would be no supremum.  To
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    54
avoid this situation it must be guaranteed that there is an element in
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    55
this set. This element must be ${} \ge 0$ so that
7927
b50446a33c16 update by Gertrud Bauer;
wenzelm
parents: 7917
diff changeset
    56
$\idt{function{\dsh}norm}$ has the norm properties. Furthermore it
b50446a33c16 update by Gertrud Bauer;
wenzelm
parents: 7917
diff changeset
    57
does not have to change the norm in all other cases, so it must be
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    58
$0$, as all other elements of are ${} \ge 0$.
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    59
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    60
Thus we define the set $B$ the supremum is taken from as
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    61
\[
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    62
\{ 0 \} \Union \left\{ \frac{|f\ap x|}{\norm x} \dt x\neq \zero \And x\in F\right\}
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    63
 \]
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    64
*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    65
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    66
constdefs
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    67
  B :: "[ 'a set, 'a => real, 'a::{plus, minus, zero} => real ] => real set"
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
    68
  "B V norm f == 
9503
wenzelm
parents: 9408
diff changeset
    69
  {#0} \<union> {|f x| * rinv (norm x) | x. x \<noteq> 0 \<and> x \<in> V}"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    70
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    71
text{* $n$ is the function norm of $f$, iff 
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    72
$n$ is the supremum of $B$. 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    73
*}
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    74
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    75
constdefs 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    76
  is_function_norm :: 
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    77
  " ['a::{minus,plus,zero}  => real, 'a set, 'a => real] => real => bool"
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    78
  "is_function_norm f V norm fn == is_Sup UNIV (B V norm f) fn"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    79
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    80
text{* $\idt{function{\dsh}norm}$ is equal to the supremum of $B$, 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    81
if the supremum exists. Otherwise it is undefined. *}
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    82
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    83
constdefs 
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    84
  function_norm :: " ['a::{minus,plus,zero} => real, 'a set, 'a => real] => real"
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    85
  "function_norm f V norm == Sup UNIV (B V norm f)"
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    86
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    87
syntax   
9503
wenzelm
parents: 9408
diff changeset
    88
  function_norm :: " ['a => real, 'a set, 'a => real] => real" ("\<parallel>_\<parallel>_,_")
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
    89
9503
wenzelm
parents: 9408
diff changeset
    90
lemma B_not_empty: "#0 \<in> B V norm f"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    91
  by (unfold B_def, force)
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    92
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    93
text {* The following lemma states that every continuous linear form
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    94
on a normed space $(V, \norm{\cdot})$ has a function norm. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    95
9408
d3d56e1d2ec1 classical atts now intro! / intro / intro?;
wenzelm
parents: 9394
diff changeset
    96
lemma ex_fnorm [intro?]: 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
    97
  "[| is_normed_vectorspace V norm; is_continuous V norm f|]
9503
wenzelm
parents: 9408
diff changeset
    98
     ==> is_function_norm f V norm \<parallel>f\<parallel>V,norm" 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    99
proof (unfold function_norm_def is_function_norm_def 
9969
4753185f1dd2 renamed (most of...) the select rules
paulson
parents: 9503
diff changeset
   100
  is_continuous_def Sup_def, elim conjE, rule someI2EX)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   101
  assume "is_normed_vectorspace V norm"
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   102
  assume "is_linearform V f" 
9503
wenzelm
parents: 9408
diff changeset
   103
  and e: "\<exists>c. \<forall>x \<in> V. |f x| <= c * norm x"
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   104
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   105
  txt {* The existence of the supremum is shown using the 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   106
  completeness of the reals. Completeness means, that
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   107
  every non-empty bounded set of reals has a 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   108
  supremum. *}
9503
wenzelm
parents: 9408
diff changeset
   109
  show  "\<exists>a. is_Sup UNIV (B V norm f) a" 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   110
  proof (unfold is_Sup_def, rule reals_complete)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   111
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   112
    txt {* First we have to show that $B$ is non-empty: *} 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   113
9503
wenzelm
parents: 9408
diff changeset
   114
    show "\<exists>X. X \<in> B V norm f" 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   115
    proof (intro exI)
9503
wenzelm
parents: 9408
diff changeset
   116
      show "#0 \<in> (B V norm f)" by (unfold B_def, force)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   117
    qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   118
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   119
    txt {* Then we have to show that $B$ is bounded: *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   120
9503
wenzelm
parents: 9408
diff changeset
   121
    from e show "\<exists>Y. isUb UNIV (B V norm f) Y"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   122
    proof
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   123
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   124
      txt {* We know that $f$ is bounded by some value $c$. *}  
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   125
  
9503
wenzelm
parents: 9408
diff changeset
   126
      fix c assume a: "\<forall>x \<in> V. |f x| <= c * norm x"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   127
      def b == "max c #0"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   128
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   129
      show "?thesis"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   130
      proof (intro exI isUbI setleI ballI, unfold B_def, 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   131
	elim UnE CollectE exE conjE singletonE)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   132
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   133
        txt{* To proof the thesis, we have to show that there is 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   134
        some constant $b$, such that $y \leq b$ for all $y\in B$. 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   135
        Due to the definition of $B$ there are two cases for
9379
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   136
        $y\in B$. If $y = 0$ then $y \leq \idt{max}\ap c\ap 0$: *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   137
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   138
	fix y assume "y = (#0::real)"
9394
wenzelm
parents: 9379
diff changeset
   139
        show "y <= b" by (simp! add: le_maxI2)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   140
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   141
        txt{* The second case is 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   142
        $y = {|f\ap x|}/{\norm x}$ for some 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   143
        $x\in V$ with $x \neq \zero$. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   144
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   145
      next
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   146
	fix x y
9503
wenzelm
parents: 9408
diff changeset
   147
        assume "x \<in> V" "x \<noteq> 0" (***
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   148
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   149
         have ge: "#0 <= rinv (norm x)";
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   150
          by (rule real_less_imp_le, rule real_rinv_gt_zero, 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   151
                rule normed_vs_norm_gt_zero); ( ***
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7567
diff changeset
   152
          proof (rule real_less_imp_le);
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   153
            show "#0 < rinv (norm x)";
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
   154
            proof (rule real_rinv_gt_zero);
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   155
              show "#0 < norm x"; ..;
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
   156
            qed;
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   157
          qed; *** )
9503
wenzelm
parents: 9408
diff changeset
   158
        have nz: "norm x \<noteq> #0" 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   159
          by (rule not_sym, rule lt_imp_not_eq, 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   160
              rule normed_vs_norm_gt_zero) (***
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   161
          proof (rule not_sym);
9503
wenzelm
parents: 9408
diff changeset
   162
            show "#0 \<noteq> norm x"; 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   163
            proof (rule lt_imp_not_eq);
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   164
              show "#0 < norm x"; ..;
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   165
            qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   166
          qed; ***)***)
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   167
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   168
        txt {* The thesis follows by a short calculation using the 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   169
        fact that $f$ is bounded. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   170
    
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   171
        assume "y = |f x| * rinv (norm x)"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   172
        also have "... <= c * norm x * rinv (norm x)"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   173
        proof (rule real_mult_le_le_mono2)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   174
          show "#0 <= rinv (norm x)"
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   175
            by (rule real_less_imp_le, rule real_rinv_gt_zero1, 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   176
                rule normed_vs_norm_gt_zero)
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   177
          from a show "|f x| <= c * norm x" ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   178
        qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   179
        also have "... = c * (norm x * rinv (norm x))" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   180
          by (rule real_mult_assoc)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   181
        also have "(norm x * rinv (norm x)) = (#1::real)" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   182
        proof (rule real_mult_inv_right1)
9503
wenzelm
parents: 9408
diff changeset
   183
          show nz: "norm x \<noteq> #0" 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   184
            by (rule not_sym, rule lt_imp_not_eq, 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   185
              rule normed_vs_norm_gt_zero)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   186
        qed
9394
wenzelm
parents: 9379
diff changeset
   187
        also have "c * ... <= b " by (simp! add: le_maxI1)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   188
	finally show "y <= b" .
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   189
      qed simp
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   190
    qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   191
  qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   192
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   193
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   194
text {* The norm of a continuous function is always $\geq 0$. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   195
9408
d3d56e1d2ec1 classical atts now intro! / intro / intro?;
wenzelm
parents: 9394
diff changeset
   196
lemma fnorm_ge_zero [intro?]: 
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   197
  "[| is_continuous V norm f; is_normed_vectorspace V norm |]
9503
wenzelm
parents: 9408
diff changeset
   198
   ==> #0 <= \<parallel>f\<parallel>V,norm"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   199
proof -
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   200
  assume c: "is_continuous V norm f" 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   201
     and n: "is_normed_vectorspace V norm"
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   202
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   203
  txt {* The function norm is defined as the supremum of $B$. 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   204
  So it is $\geq 0$ if all elements in $B$ are $\geq 0$, provided
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   205
  the supremum exists and $B$ is not empty. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   206
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   207
  show ?thesis 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   208
  proof (unfold function_norm_def, rule sup_ub1)
9503
wenzelm
parents: 9408
diff changeset
   209
    show "\<forall>x \<in> (B V norm f). #0 <= x" 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   210
    proof (intro ballI, unfold B_def,
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   211
           elim UnE singletonE CollectE exE conjE) 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   212
      fix x r
9503
wenzelm
parents: 9408
diff changeset
   213
      assume "x \<in> V" "x \<noteq> 0" 
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   214
        and r: "r = |f x| * rinv (norm x)"
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   215
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   216
      have ge: "#0 <= |f x|" by (simp! only: abs_ge_zero)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   217
      have "#0 <= rinv (norm x)" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   218
        by (rule real_less_imp_le, rule real_rinv_gt_zero1, rule)(***
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7567
diff changeset
   219
        proof (rule real_less_imp_le);
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   220
          show "#0 < rinv (norm x)"; 
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
   221
          proof (rule real_rinv_gt_zero);
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   222
            show "#0 < norm x"; ..;
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
   223
          qed;
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   224
        qed; ***)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   225
      with ge show "#0 <= r"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   226
       by (simp only: r, rule real_le_mult_order1a)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   227
    qed (simp!)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   228
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   229
    txt {* Since $f$ is continuous the function norm exists: *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   230
9503
wenzelm
parents: 9408
diff changeset
   231
    have "is_function_norm f V norm \<parallel>f\<parallel>V,norm" ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   232
    thus "is_Sup UNIV (B V norm f) (Sup UNIV (B V norm f))" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   233
      by (unfold is_function_norm_def function_norm_def)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   234
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   235
    txt {* $B$ is non-empty by construction: *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   236
9503
wenzelm
parents: 9408
diff changeset
   237
    show "#0 \<in> B V norm f" by (rule B_not_empty)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   238
  qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   239
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   240
  
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   241
text{* \medskip The fundamental property of function norms is: 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   242
\begin{matharray}{l}
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   243
| f\ap x | \leq {\fnorm {f}} \cdot {\norm x}  
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   244
\end{matharray}
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   245
*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   246
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   247
lemma norm_fx_le_norm_f_norm_x: 
9503
wenzelm
parents: 9408
diff changeset
   248
  "[| is_continuous V norm f; is_normed_vectorspace V norm; x \<in> V |] 
wenzelm
parents: 9408
diff changeset
   249
    ==> |f x| <= \<parallel>f\<parallel>V,norm * norm x"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   250
proof - 
9503
wenzelm
parents: 9408
diff changeset
   251
  assume "is_normed_vectorspace V norm" "x \<in> V" 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   252
  and c: "is_continuous V norm f"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   253
  have v: "is_vectorspace V" ..
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   254
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   255
 txt{* The proof is by case analysis on $x$. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   256
 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   257
  show ?thesis
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   258
  proof cases
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   259
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   260
    txt {* For the case $x = \zero$ the thesis follows
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   261
    from the linearity of $f$: for every linear function
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   262
    holds $f\ap \zero = 0$. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   263
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   264
    assume "x = 0"
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   265
    have "|f x| = |f 0|" by (simp!)
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   266
    also from v continuous_linearform have "f 0 = #0" ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   267
    also note abs_zero
9503
wenzelm
parents: 9408
diff changeset
   268
    also have "#0 <= \<parallel>f\<parallel>V,norm * norm x"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   269
    proof (rule real_le_mult_order1a)
9503
wenzelm
parents: 9408
diff changeset
   270
      show "#0 <= \<parallel>f\<parallel>V,norm" ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   271
      show "#0 <= norm x" ..
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   272
    qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   273
    finally 
9503
wenzelm
parents: 9408
diff changeset
   274
    show "|f x| <= \<parallel>f\<parallel>V,norm * norm x" .
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   275
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   276
  next
9503
wenzelm
parents: 9408
diff changeset
   277
    assume "x \<noteq> 0"
9379
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   278
    have n: "#0 < norm x" ..
9503
wenzelm
parents: 9408
diff changeset
   279
    hence nz: "norm x \<noteq> #0" 
9379
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   280
      by (simp only: lt_imp_not_eq)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   281
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   282
    txt {* For the case $x\neq \zero$ we derive the following
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   283
    fact from the definition of the function norm:*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   284
9503
wenzelm
parents: 9408
diff changeset
   285
    have l: "|f x| * rinv (norm x) <= \<parallel>f\<parallel>V,norm"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   286
    proof (unfold function_norm_def, rule sup_ub)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   287
      from ex_fnorm [OF _ c]
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   288
      show "is_Sup UNIV (B V norm f) (Sup UNIV (B V norm f))"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   289
         by (simp! add: is_function_norm_def function_norm_def)
9503
wenzelm
parents: 9408
diff changeset
   290
      show "|f x| * rinv (norm x) \<in> B V norm f" 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   291
        by (unfold B_def, intro UnI2 CollectI exI [of _ x]
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   292
            conjI, simp)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   293
    qed
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   294
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   295
    txt {* The thesis now follows by a short calculation: *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   296
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   297
    have "|f x| = |f x| * #1" by (simp!)
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   298
    also from nz have "#1 = rinv (norm x) * norm x" 
9379
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   299
      by (simp add: real_mult_inv_left1)
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   300
    also have "|f x| * ... = |f x| * rinv (norm x) * norm x"
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   301
      by (simp! add: real_mult_assoc)
9503
wenzelm
parents: 9408
diff changeset
   302
    also from n l have "... <= \<parallel>f\<parallel>V,norm * norm x"
9379
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   303
      by (simp add: real_mult_le_le_mono2)
9503
wenzelm
parents: 9408
diff changeset
   304
    finally show "|f x| <= \<parallel>f\<parallel>V,norm * norm x" .
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   305
  qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   306
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   307
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   308
text{* \medskip The function norm is the least positive real number for 
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   309
which the following inequation holds:
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   310
\begin{matharray}{l}
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   311
| f\ap x | \leq c \cdot {\norm x}  
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   312
\end{matharray} 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   313
*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   314
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   315
lemma fnorm_le_ub: 
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   316
  "[| is_continuous V norm f; is_normed_vectorspace V norm; 
9503
wenzelm
parents: 9408
diff changeset
   317
     \<forall>x \<in> V. |f x| <= c * norm x; #0 <= c |]
wenzelm
parents: 9408
diff changeset
   318
  ==> \<parallel>f\<parallel>V,norm <= c"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   319
proof (unfold function_norm_def)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   320
  assume "is_normed_vectorspace V norm" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   321
  assume c: "is_continuous V norm f"
9503
wenzelm
parents: 9408
diff changeset
   322
  assume fb: "\<forall>x \<in> V. |f x| <= c * norm x"
9379
21cfeae6659d tuded presentation;
bauerg
parents: 9374
diff changeset
   323
    and "#0 <= c"
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   324
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   325
  txt {* Suppose the inequation holds for some $c\geq 0$.
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   326
  If $c$ is an upper bound of $B$, then $c$ is greater 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   327
  than the function norm since the function norm is the
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   328
  least upper bound.
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   329
  *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   330
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   331
  show "Sup UNIV (B V norm f) <= c" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   332
  proof (rule sup_le_ub)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   333
    from ex_fnorm [OF _ c] 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   334
    show "is_Sup UNIV (B V norm f) (Sup UNIV (B V norm f))" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   335
      by (simp! add: is_function_norm_def function_norm_def) 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   336
  
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   337
    txt {* $c$ is an upper bound of $B$, i.e. every
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   338
    $y\in B$ is less than $c$. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   339
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   340
    show "isUb UNIV (B V norm f) c"  
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   341
    proof (intro isUbI setleI ballI)
9503
wenzelm
parents: 9408
diff changeset
   342
      fix y assume "y \<in> B V norm f"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   343
      thus le: "y <= c"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   344
      proof (unfold B_def, elim UnE CollectE exE conjE singletonE)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   345
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   346
       txt {* The first case for $y\in B$ is $y=0$. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   347
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   348
        assume "y = #0"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   349
        show "y <= c" by (force!)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   350
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   351
        txt{* The second case is 
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7927
diff changeset
   352
        $y = {|f\ap x|}/{\norm x}$ for some 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   353
        $x\in V$ with $x \neq \zero$. *}  
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   354
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   355
      next
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   356
	fix x 
9503
wenzelm
parents: 9408
diff changeset
   357
        assume "x \<in> V" "x \<noteq> 0" 
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   358
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   359
        have lz: "#0 < norm x" 
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   360
          by (simp! add: normed_vs_norm_gt_zero)
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
   361
          
9503
wenzelm
parents: 9408
diff changeset
   362
        have nz: "norm x \<noteq> #0" 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   363
        proof (rule not_sym)
9503
wenzelm
parents: 9408
diff changeset
   364
          from lz show "#0 \<noteq> norm x"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   365
            by (simp! add: order_less_imp_not_eq)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   366
        qed
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
   367
            
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   368
	from lz have "#0 < rinv (norm x)"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   369
	  by (simp! add: real_rinv_gt_zero1)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   370
	hence rinv_gez: "#0 <= rinv (norm x)"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   371
          by (rule real_less_imp_le)
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   372
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   373
	assume "y = |f x| * rinv (norm x)" 
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   374
	also from rinv_gez have "... <= c * norm x * rinv (norm x)"
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   375
	  proof (rule real_mult_le_le_mono2)
9374
153853af318b - xsymbols for
bauerg
parents: 9035
diff changeset
   376
	    show "|f x| <= c * norm x" by (rule bspec)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   377
	  qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   378
	also have "... <= c" by (simp add: nz real_mult_assoc)
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   379
	finally show ?thesis .
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   380
      qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   381
    qed force
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   382
  qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   383
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   384
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   385
end