src/HOL/Real/HahnBanach/FunctionNorm.thy
author wenzelm
Thu, 14 Jun 2007 00:22:45 +0200
changeset 23378 1d138d6bb461
parent 22931 11cc1ccad58e
child 27611 2c01c0bdb385
permissions -rw-r--r--
tuned proofs: avoid implicit prems;
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
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 15206
diff changeset
     8
theory FunctionNorm imports NormedSpace FunctionOrder begin
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
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    12
text {*
11472
wenzelm
parents: 10752
diff changeset
    13
  A linear form @{text f} on a normed vector space @{text "(V, \<parallel>\<cdot>\<parallel>)"}
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    14
  is \emph{continuous}, iff it is bounded, i.e.
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    15
  \begin{center}
11472
wenzelm
parents: 10752
diff changeset
    16
  @{text "\<exists>c \<in> R. \<forall>x \<in> V. \<bar>f x\<bar> \<le> c \<cdot> \<parallel>x\<parallel>"}
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    17
  \end{center}
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    18
  In our application no other functions than linear forms are
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    19
  considered, so we can define continuous linear forms as bounded
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    20
  linear forms:
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    21
*}
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    22
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    23
locale continuous = var V + norm_syntax + linearform +
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    24
  assumes bounded: "\<exists>c. \<forall>x \<in> V. \<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    25
14254
342634f38451 Isar/Locales: <loc>.intro and <loc>.axioms no longer intro? and elim? by
ballarin
parents: 14214
diff changeset
    26
declare continuous.intro [intro?] continuous_axioms.intro [intro?]
342634f38451 Isar/Locales: <loc>.intro and <loc>.axioms no longer intro? and elim? by
ballarin
parents: 14214
diff changeset
    27
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    28
lemma continuousI [intro]:
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    29
  includes norm_syntax + linearform
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    30
  assumes r: "\<And>x. x \<in> V \<Longrightarrow> \<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    31
  shows "continuous V norm f"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    32
proof
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
    33
  show "linearform V f" by fact
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    34
  from r have "\<exists>c. \<forall>x\<in>V. \<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>" by blast
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    35
  then show "continuous_axioms V norm f" ..
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    36
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    37
11472
wenzelm
parents: 10752
diff changeset
    38
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    39
subsection {* The norm of a linear form *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    40
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    41
text {*
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    42
  The least real number @{text c} for which holds
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    43
  \begin{center}
11472
wenzelm
parents: 10752
diff changeset
    44
  @{text "\<forall>x \<in> V. \<bar>f x\<bar> \<le> c \<cdot> \<parallel>x\<parallel>"}
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    45
  \end{center}
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    46
  is called the \emph{norm} of @{text f}.
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    47
11472
wenzelm
parents: 10752
diff changeset
    48
  For non-trivial vector spaces @{text "V \<noteq> {0}"} the norm can be
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    49
  defined as
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    50
  \begin{center}
11472
wenzelm
parents: 10752
diff changeset
    51
  @{text "\<parallel>f\<parallel> = \<sup>x \<noteq> 0. \<bar>f x\<bar> / \<parallel>x\<parallel>"}
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    52
  \end{center}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    53
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    54
  For the case @{text "V = {0}"} the supremum would be taken from an
11472
wenzelm
parents: 10752
diff changeset
    55
  empty set. Since @{text \<real>} is unbounded, there would be no supremum.
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    56
  To avoid this situation it must be guaranteed that there is an
11472
wenzelm
parents: 10752
diff changeset
    57
  element in this set. This element must be @{text "{} \<ge> 0"} so that
13547
wenzelm
parents: 13524
diff changeset
    58
  @{text fn_norm} has the norm properties. Furthermore it does not
wenzelm
parents: 13524
diff changeset
    59
  have to change the norm in all other cases, so it must be @{text 0},
wenzelm
parents: 13524
diff changeset
    60
  as all other elements are @{text "{} \<ge> 0"}.
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    61
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    62
  Thus we define the set @{text B} where the supremum is taken from as
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    63
  follows:
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    64
  \begin{center}
11472
wenzelm
parents: 10752
diff changeset
    65
  @{text "{0} \<union> {\<bar>f x\<bar> / \<parallel>x\<parallel>. x \<noteq> 0 \<and> x \<in> F}"}
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    66
  \end{center}
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    67
13547
wenzelm
parents: 13524
diff changeset
    68
  @{text fn_norm} is equal to the supremum of @{text B}, if the
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    69
  supremum exists (otherwise it is undefined).
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
    70
*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    71
13547
wenzelm
parents: 13524
diff changeset
    72
locale fn_norm = norm_syntax +
wenzelm
parents: 13524
diff changeset
    73
  fixes B defines "B V f \<equiv> {0} \<union> {\<bar>f x\<bar> / \<parallel>x\<parallel> | x. x \<noteq> 0 \<and> x \<in> V}"
wenzelm
parents: 13524
diff changeset
    74
  fixes fn_norm ("\<parallel>_\<parallel>\<hyphen>_" [0, 1000] 999)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    75
  defines "\<parallel>f\<parallel>\<hyphen>V \<equiv> \<Squnion>(B V f)"
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    76
13547
wenzelm
parents: 13524
diff changeset
    77
lemma (in fn_norm) B_not_empty [intro]: "0 \<in> B V f"
wenzelm
parents: 13524
diff changeset
    78
  by (simp add: B_def)
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    79
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    80
text {*
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    81
  The following lemma states that every continuous linear form on a
11472
wenzelm
parents: 10752
diff changeset
    82
  normed space @{text "(V, \<parallel>\<cdot>\<parallel>)"} has a function norm.
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    83
*}
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    84
15206
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    85
(* Alternative statement of the lemma as
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    86
     lemma (in fn_norm)
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    87
       includes normed_vectorspace + continuous
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    88
       shows "lub (B V f) (\<parallel>f\<parallel>\<hyphen>V)"
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    89
   is not possible:
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    90
   fn_norm contrains parameter norm to type "'a::zero => real",
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    91
   normed_vectorspace and continuous contrain this parameter to
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    92
   "'a::{minus, plus, zero} => real, which is less general.
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    93
*)
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    94
09d78ec709c7 Modified locales: improved implementation of "includes".
ballarin
parents: 14710
diff changeset
    95
lemma (in normed_vectorspace) fn_norm_works:
13547
wenzelm
parents: 13524
diff changeset
    96
  includes fn_norm + continuous
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    97
  shows "lub (B V f) (\<parallel>f\<parallel>\<hyphen>V)"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
    98
proof -
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
    99
  txt {* The existence of the supremum is shown using the
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   100
    completeness of the reals. Completeness means, that every
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   101
    non-empty bounded set of reals has a supremum. *}
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   102
  have "\<exists>a. lub (B V f) a"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   103
  proof (rule real_complete)
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   104
    txt {* First we have to show that @{text B} is non-empty: *}
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   105
    have "0 \<in> B V f" ..
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   106
    thus "\<exists>x. x \<in> B V f" ..
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   107
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   108
    txt {* Then we have to show that @{text B} is bounded: *}
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   109
    show "\<exists>c. \<forall>y \<in> B V f. y \<le> c"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   110
    proof -
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   111
      txt {* We know that @{text f} is bounded by some value @{text c}. *}
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   112
      from bounded obtain c where c: "\<forall>x \<in> V. \<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>" ..
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   113
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   114
      txt {* To prove the thesis, we have to show that there is some
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   115
        @{text b}, such that @{text "y \<le> b"} for all @{text "y \<in>
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   116
        B"}. Due to the definition of @{text B} there are two cases. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   117
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   118
      def b \<equiv> "max c 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   119
      have "\<forall>y \<in> B V f. y \<le> b"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   120
      proof
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   121
        fix y assume y: "y \<in> B V f"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   122
        show "y \<le> b"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   123
        proof cases
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   124
          assume "y = 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   125
          thus ?thesis by (unfold b_def) arith
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   126
        next
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   127
          txt {* The second case is @{text "y = \<bar>f x\<bar> / \<parallel>x\<parallel>"} for some
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   128
            @{text "x \<in> V"} with @{text "x \<noteq> 0"}. *}
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   129
          assume "y \<noteq> 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   130
          with y obtain x where y_rep: "y = \<bar>f x\<bar> * inverse \<parallel>x\<parallel>"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   131
              and x: "x \<in> V" and neq: "x \<noteq> 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   132
            by (auto simp add: B_def real_divide_def)
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   133
          from x neq have gt: "0 < \<parallel>x\<parallel>" ..
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   134
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   135
          txt {* The thesis follows by a short calculation using the
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   136
            fact that @{text f} is bounded. *}
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   137
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   138
          note y_rep
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   139
          also have "\<bar>f x\<bar> * inverse \<parallel>x\<parallel> \<le> (c * \<parallel>x\<parallel>) * inverse \<parallel>x\<parallel>"
14334
6137d24eef79 tweaking of lemmas in RealDef, RealOrd
paulson
parents: 14254
diff changeset
   140
          proof (rule mult_right_mono)
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   141
            from c x show "\<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>" ..
14334
6137d24eef79 tweaking of lemmas in RealDef, RealOrd
paulson
parents: 14254
diff changeset
   142
            from gt have "0 < inverse \<parallel>x\<parallel>" 
6137d24eef79 tweaking of lemmas in RealDef, RealOrd
paulson
parents: 14254
diff changeset
   143
              by (rule positive_imp_inverse_positive)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   144
            thus "0 \<le> inverse \<parallel>x\<parallel>" by (rule order_less_imp_le)
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   145
          qed
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   146
          also have "\<dots> = c * (\<parallel>x\<parallel> * inverse \<parallel>x\<parallel>)"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   147
            by (rule real_mult_assoc)
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   148
          also
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   149
          from gt have "\<parallel>x\<parallel> \<noteq> 0" by simp
14710
247615bfffb8 replaced Aux.thy by RealLemmas.thy
bauerg
parents: 14334
diff changeset
   150
          hence "\<parallel>x\<parallel> * inverse \<parallel>x\<parallel> = 1" by simp 
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   151
          also have "c * 1 \<le> b" by (simp add: b_def le_maxI1)
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   152
          finally show "y \<le> b" .
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   153
        qed
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   154
      qed
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   155
      thus ?thesis ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   156
    qed
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   157
  qed
13547
wenzelm
parents: 13524
diff changeset
   158
  then show ?thesis by (unfold fn_norm_def) (rule the_lubI_ex)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   159
qed
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   160
13547
wenzelm
parents: 13524
diff changeset
   161
lemma (in normed_vectorspace) fn_norm_ub [iff?]:
wenzelm
parents: 13524
diff changeset
   162
  includes fn_norm + continuous
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   163
  assumes b: "b \<in> B V f"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   164
  shows "b \<le> \<parallel>f\<parallel>\<hyphen>V"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   165
proof -
13547
wenzelm
parents: 13524
diff changeset
   166
  have "lub (B V f) (\<parallel>f\<parallel>\<hyphen>V)"
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   167
    unfolding B_def fn_norm_def
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   168
    using `continuous V norm f` by (rule fn_norm_works)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   169
  from this and b show ?thesis ..
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   170
qed
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   171
13547
wenzelm
parents: 13524
diff changeset
   172
lemma (in normed_vectorspace) fn_norm_leastB:
wenzelm
parents: 13524
diff changeset
   173
  includes fn_norm + continuous
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   174
  assumes b: "\<And>b. b \<in> B V f \<Longrightarrow> b \<le> y"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   175
  shows "\<parallel>f\<parallel>\<hyphen>V \<le> y"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   176
proof -
13547
wenzelm
parents: 13524
diff changeset
   177
  have "lub (B V f) (\<parallel>f\<parallel>\<hyphen>V)"
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   178
    unfolding B_def fn_norm_def
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   179
    using `continuous V norm f` by (rule fn_norm_works)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   180
  from this and b show ?thesis ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   181
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   182
11472
wenzelm
parents: 10752
diff changeset
   183
text {* The norm of a continuous function is always @{text "\<ge> 0"}. *}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   184
13547
wenzelm
parents: 13524
diff changeset
   185
lemma (in normed_vectorspace) fn_norm_ge_zero [iff]:
wenzelm
parents: 13524
diff changeset
   186
  includes fn_norm + continuous
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   187
  shows "0 \<le> \<parallel>f\<parallel>\<hyphen>V"
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   188
proof -
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   189
  txt {* The function norm is defined as the supremum of @{text B}.
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   190
    So it is @{text "\<ge> 0"} if all elements in @{text B} are @{text "\<ge>
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   191
    0"}, provided the supremum exists and @{text B} is not empty. *}
13547
wenzelm
parents: 13524
diff changeset
   192
  have "lub (B V f) (\<parallel>f\<parallel>\<hyphen>V)"
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   193
    unfolding B_def fn_norm_def
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   194
    using `continuous V norm f` by (rule fn_norm_works)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   195
  moreover have "0 \<in> B V f" ..
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   196
  ultimately show ?thesis ..
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   197
qed
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   198
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   199
text {*
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   200
  \medskip The fundamental property of function norms is:
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   201
  \begin{center}
11472
wenzelm
parents: 10752
diff changeset
   202
  @{text "\<bar>f x\<bar> \<le> \<parallel>f\<parallel> \<cdot> \<parallel>x\<parallel>"}
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   203
  \end{center}
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   204
*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   205
13547
wenzelm
parents: 13524
diff changeset
   206
lemma (in normed_vectorspace) fn_norm_le_cong:
wenzelm
parents: 13524
diff changeset
   207
  includes fn_norm + continuous + linearform
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   208
  assumes x: "x \<in> V"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   209
  shows "\<bar>f x\<bar> \<le> \<parallel>f\<parallel>\<hyphen>V * \<parallel>x\<parallel>"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   210
proof cases
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   211
  assume "x = 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   212
  then have "\<bar>f x\<bar> = \<bar>f 0\<bar>" by simp
19984
29bb4659f80a Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents: 19931
diff changeset
   213
  also have "f 0 = 0" by rule unfold_locales
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   214
  also have "\<bar>\<dots>\<bar> = 0" by simp
14710
247615bfffb8 replaced Aux.thy by RealLemmas.thy
bauerg
parents: 14334
diff changeset
   215
  also have a: "0 \<le> \<parallel>f\<parallel>\<hyphen>V"
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   216
    unfolding B_def fn_norm_def
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   217
    using `continuous V norm f` by (rule fn_norm_ge_zero)
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   218
  from x have "0 \<le> norm x" ..
14710
247615bfffb8 replaced Aux.thy by RealLemmas.thy
bauerg
parents: 14334
diff changeset
   219
  with a have "0 \<le> \<parallel>f\<parallel>\<hyphen>V * \<parallel>x\<parallel>" by (simp add: zero_le_mult_iff)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   220
  finally show "\<bar>f x\<bar> \<le> \<parallel>f\<parallel>\<hyphen>V * \<parallel>x\<parallel>" .
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   221
next
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   222
  assume "x \<noteq> 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   223
  with x have neq: "\<parallel>x\<parallel> \<noteq> 0" by simp
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   224
  then have "\<bar>f x\<bar> = (\<bar>f x\<bar> * inverse \<parallel>x\<parallel>) * \<parallel>x\<parallel>" by simp
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   225
  also have "\<dots> \<le>  \<parallel>f\<parallel>\<hyphen>V * \<parallel>x\<parallel>"
14334
6137d24eef79 tweaking of lemmas in RealDef, RealOrd
paulson
parents: 14254
diff changeset
   226
  proof (rule mult_right_mono)
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   227
    from x show "0 \<le> \<parallel>x\<parallel>" ..
13547
wenzelm
parents: 13524
diff changeset
   228
    from x and neq have "\<bar>f x\<bar> * inverse \<parallel>x\<parallel> \<in> B V f"
wenzelm
parents: 13524
diff changeset
   229
      by (auto simp add: B_def real_divide_def)
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   230
    with `continuous V norm f` show "\<bar>f x\<bar> * inverse \<parallel>x\<parallel> \<le> \<parallel>f\<parallel>\<hyphen>V"
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   231
      unfolding B_def fn_norm_def by (rule fn_norm_ub)
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   232
  qed
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   233
  finally show ?thesis .
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   234
qed
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   235
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   236
text {*
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   237
  \medskip The function norm is the least positive real number for
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   238
  which the following inequation holds:
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   239
  \begin{center}
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   240
    @{text "\<bar>f x\<bar> \<le> c \<cdot> \<parallel>x\<parallel>"}
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   241
  \end{center}
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   242
*}
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
   243
13547
wenzelm
parents: 13524
diff changeset
   244
lemma (in normed_vectorspace) fn_norm_least [intro?]:
wenzelm
parents: 13524
diff changeset
   245
  includes fn_norm + continuous
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   246
  assumes ineq: "\<forall>x \<in> V. \<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>" and ge: "0 \<le> c"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   247
  shows "\<parallel>f\<parallel>\<hyphen>V \<le> c"
13547
wenzelm
parents: 13524
diff changeset
   248
proof (rule fn_norm_leastB [folded B_def fn_norm_def])
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   249
  fix b assume b: "b \<in> B V f"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   250
  show "b \<le> c"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   251
  proof cases
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   252
    assume "b = 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   253
    with ge show ?thesis by simp
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   254
  next
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   255
    assume "b \<noteq> 0"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   256
    with b obtain x where b_rep: "b = \<bar>f x\<bar> * inverse \<parallel>x\<parallel>"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   257
        and x_neq: "x \<noteq> 0" and x: "x \<in> V"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   258
      by (auto simp add: B_def real_divide_def)
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   259
    note b_rep
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   260
    also have "\<bar>f x\<bar> * inverse \<parallel>x\<parallel> \<le> (c * \<parallel>x\<parallel>) * inverse \<parallel>x\<parallel>"
14334
6137d24eef79 tweaking of lemmas in RealDef, RealOrd
paulson
parents: 14254
diff changeset
   261
    proof (rule mult_right_mono)
23378
1d138d6bb461 tuned proofs: avoid implicit prems;
wenzelm
parents: 22931
diff changeset
   262
      have "0 < \<parallel>x\<parallel>" using x x_neq ..
13515
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   263
      then show "0 \<le> inverse \<parallel>x\<parallel>" by simp
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   264
      from ineq and x show "\<bar>f x\<bar> \<le> c * \<parallel>x\<parallel>" ..
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   265
    qed
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   266
    also have "\<dots> = c"
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   267
    proof -
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   268
      from x_neq and x have "\<parallel>x\<parallel> \<noteq> 0" by simp
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   269
      then show ?thesis by simp
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   270
    qed
a6a7025fd7e8 updated to use locales (still some rough edges);
wenzelm
parents: 12018
diff changeset
   271
    finally show ?thesis .
9035
371f023d3dbd removed explicit terminator (";");
wenzelm
parents: 9013
diff changeset
   272
  qed
22931
11cc1ccad58e tuned proofs;
wenzelm
parents: 19984
diff changeset
   273
qed (insert `continuous V norm f`, simp_all add: continuous_def)
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   274
10687
c186279eecea tuned HOL/Real/HahnBanach;
wenzelm
parents: 10606
diff changeset
   275
end