src/HOL/Multivariate_Analysis/Operator_Norm.thy
author paulson <lp15@cam.ac.uk>
Fri, 07 Mar 2014 12:35:06 +0000
changeset 55967 5dadc93ff3df
parent 54263 c4159fe6fa46
child 56223 7696903b9e61
permissions -rw-r--r--
a few new lemmas
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
41959
b460124855b8 tuned headers;
wenzelm
parents: 38642
diff changeset
     1
(*  Title:      HOL/Multivariate_Analysis/Operator_Norm.thy
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     2
    Author:     Amine Chaieb, University of Cambridge
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     3
*)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     4
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     5
header {* Operator Norm *}
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     6
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     7
theory Operator_Norm
44133
691c52e900ca split Linear_Algebra.thy from Euclidean_Space.thy
huffman
parents: 41959
diff changeset
     8
imports Linear_Algebra
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
     9
begin
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    10
54263
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    11
definition "onorm f = (SUP x:{x. norm x = 1}. norm (f x))"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    12
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    13
lemma norm_bound_generalize:
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    14
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    15
  assumes lf: "linear f"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    16
  shows "(\<forall>x. norm x = 1 \<longrightarrow> norm (f x) \<le> b) \<longleftrightarrow> (\<forall>x. norm (f x) \<le> b * norm x)"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    17
  (is "?lhs \<longleftrightarrow> ?rhs")
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    18
proof
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    19
  assume H: ?rhs
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    20
  {
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    21
    fix x :: "'a"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    22
    assume x: "norm x = 1"
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    23
    from H[rule_format, of x] x have "norm (f x) \<le> b"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    24
      by simp
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    25
  }
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    26
  then show ?lhs by blast
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    27
next
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    28
  assume H: ?lhs
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    29
  have bp: "b \<ge> 0"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    30
    apply -
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    31
    apply (rule order_trans [OF norm_ge_zero])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    32
    apply (rule H[rule_format, of "SOME x::'a. x \<in> Basis"])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    33
    apply (auto intro: SOME_Basis norm_Basis)
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    34
    done
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    35
  {
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    36
    fix x :: "'a"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    37
    {
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    38
      assume "x = 0"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    39
      then have "norm (f x) \<le> b * norm x"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    40
        by (simp add: linear_0[OF lf] bp)
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    41
    }
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    42
    moreover
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    43
    {
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    44
      assume x0: "x \<noteq> 0"
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    45
      then have n0: "norm x \<noteq> 0"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    46
        by (metis norm_eq_zero)
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    47
      let ?c = "1/ norm x"
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    48
      have "norm (?c *\<^sub>R x) = 1"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    49
        using x0 by (simp add: n0)
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    50
      with H have "norm (f (?c *\<^sub>R x)) \<le> b"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    51
        by blast
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    52
      then have "?c * norm (f x) \<le> b"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    53
        by (simp add: linear_cmul[OF lf])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    54
      then have "norm (f x) \<le> b * norm x"
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    55
        using n0 norm_ge_zero[of x]
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    56
        by (auto simp add: field_simps)
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    57
    }
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    58
    ultimately have "norm (f x) \<le> b * norm x"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    59
      by blast
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    60
  }
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    61
  then show ?rhs by blast
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    62
qed
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    63
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    64
lemma onorm:
37489
44e42d392c6e Introduce a type class for euclidean spaces, port most lemmas from real^'n to this type class.
hoelzl
parents: 36593
diff changeset
    65
  fixes f:: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    66
  assumes lf: "linear f"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    67
  shows "norm (f x) \<le> onorm f * norm x"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    68
    and "\<forall>x. norm (f x) \<le> b * norm x \<Longrightarrow> onorm f \<le> b"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    69
proof -
54263
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    70
  let ?S = "(\<lambda>x. norm (f x))`{x. norm x = 1}"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    71
  have "norm (f (SOME i. i \<in> Basis)) \<in> ?S"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    72
    by (auto intro!: exI[of _ "SOME i. i \<in> Basis"] norm_Basis SOME_Basis)
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    73
  then have Se: "?S \<noteq> {}"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    74
    by auto
54263
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    75
  from linear_bounded[OF lf] have b: "bdd_above ?S"
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    76
    unfolding norm_bound_generalize[OF lf, symmetric] by auto
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    77
  then show "norm (f x) \<le> onorm f * norm x"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    78
    apply -
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    79
    apply (rule spec[where x = x])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    80
    unfolding norm_bound_generalize[OF lf, symmetric]
54263
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    81
    apply (auto simp: onorm_def intro!: cSUP_upper)
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    82
    done
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    83
  show "\<forall>x. norm (f x) \<le> b * norm x \<Longrightarrow> onorm f \<le> b"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    84
    unfolding norm_bound_generalize[OF lf, symmetric]
54263
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
    85
    using Se by (auto simp: onorm_def intro!: cSUP_least b)
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    86
qed
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    87
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    88
lemma onorm_pos_le:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    89
  fixes f :: "'n::euclidean_space \<Rightarrow> 'm::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    90
  assumes lf: "linear f"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    91
  shows "0 \<le> onorm f"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    92
  using order_trans[OF norm_ge_zero onorm(1)[OF lf, of "SOME i. i \<in> Basis"]]
50526
899c9c4e4a4c Remove the indexed basis from the definition of euclidean spaces and only use the set of Basis vectors
hoelzl
parents: 44133
diff changeset
    93
  by (simp add: SOME_Basis)
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    94
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
    95
lemma onorm_eq_0:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    96
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
    97
  assumes lf: "linear f"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    98
  shows "onorm f = 0 \<longleftrightarrow> (\<forall>x. f x = 0)"
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
    99
  using onorm[OF lf]
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   100
  apply (auto simp add: onorm_pos_le)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   101
  apply atomize
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   102
  apply (erule allE[where x="0::real"])
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   103
  using onorm_pos_le[OF lf]
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   104
  apply arith
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   105
  done
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   106
54263
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
   107
lemma onorm_const: "onorm (\<lambda>x::'a::euclidean_space. y::'b::euclidean_space) = norm y"
c4159fe6fa46 move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
hoelzl
parents: 53688
diff changeset
   108
  using SOME_Basis by (auto simp add: onorm_def intro!: cSUP_const norm_Basis)
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   109
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   110
lemma onorm_pos_lt:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   111
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   112
  assumes lf: "linear f"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   113
  shows "0 < onorm f \<longleftrightarrow> \<not> (\<forall>x. f x = 0)"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   114
  unfolding onorm_eq_0[OF lf, symmetric]
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   115
  using onorm_pos_le[OF lf] by arith
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   116
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   117
lemma onorm_compose:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   118
  fixes f :: "'n::euclidean_space \<Rightarrow> 'm::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   119
    and g :: "'k::euclidean_space \<Rightarrow> 'n::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   120
  assumes lf: "linear f"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   121
    and lg: "linear g"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   122
  shows "onorm (f \<circ> g) \<le> onorm f * onorm g"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   123
    apply (rule onorm(2)[OF linear_compose[OF lg lf], rule_format])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   124
    unfolding o_def
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   125
    apply (subst mult_assoc)
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   126
    apply (rule order_trans)
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   127
    apply (rule onorm(1)[OF lf])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   128
    apply (rule mult_left_mono)
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   129
    apply (rule onorm(1)[OF lg])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   130
    apply (rule onorm_pos_le[OF lf])
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   131
    done
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   132
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   133
lemma onorm_neg_lemma:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   134
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   135
  assumes lf: "linear f"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   136
  shows "onorm (\<lambda>x. - f x) \<le> onorm f"
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   137
  using onorm[OF linear_compose_neg[OF lf]] onorm[OF lf]
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   138
  unfolding norm_minus_cancel by metis
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   139
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   140
lemma onorm_neg:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   141
  fixes f :: "'a::euclidean_space \<Rightarrow> 'b::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   142
  assumes lf: "linear f"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   143
  shows "onorm (\<lambda>x. - f x) = onorm f"
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   144
  using onorm_neg_lemma[OF lf] onorm_neg_lemma[OF linear_compose_neg[OF lf]]
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   145
  by simp
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   146
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   147
lemma onorm_triangle:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   148
  fixes f g :: "'n::euclidean_space \<Rightarrow> 'm::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   149
  assumes lf: "linear f"
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   150
    and lg: "linear g"
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   151
  shows "onorm (\<lambda>x. f x + g x) \<le> onorm f + onorm g"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   152
  apply(rule onorm(2)[OF linear_compose_add[OF lf lg], rule_format])
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   153
  apply (rule order_trans)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   154
  apply (rule norm_triangle_ineq)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   155
  apply (simp add: distrib)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   156
  apply (rule add_mono)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   157
  apply (rule onorm(1)[OF lf])
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   158
  apply (rule onorm(1)[OF lg])
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   159
  done
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   160
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   161
lemma onorm_triangle_le:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   162
  fixes f :: "'n::euclidean_space \<Rightarrow> 'm::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   163
  assumes "linear f"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   164
    and "linear g"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   165
    and "onorm f + onorm g \<le> e"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   166
  shows "onorm (\<lambda>x. f x + g x) \<le> e"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   167
  apply (rule order_trans)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   168
  apply (rule onorm_triangle)
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   169
  apply (rule assms)+
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   170
  done
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   171
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   172
lemma onorm_triangle_lt:
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   173
  fixes f g :: "'n::euclidean_space \<Rightarrow> 'm::euclidean_space"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   174
  assumes "linear f"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   175
    and "linear g"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   176
    and "onorm f + onorm g < e"
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   177
  shows "onorm (\<lambda>x. f x + g x) < e"
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   178
  apply (rule order_le_less_trans)
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   179
  apply (rule onorm_triangle)
53688
63892cfef47f tuned proofs;
wenzelm
parents: 53253
diff changeset
   180
  apply (rule assms)+
53253
220f306f5c4e tuned proofs;
wenzelm
parents: 51475
diff changeset
   181
  done
36581
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   182
bbea7f52e8e1 move operator norm stuff to new theory file
huffman
parents:
diff changeset
   183
end