src/HOL/Real/HahnBanach/Aux.thy
author fleuriot
Thu, 01 Jun 2000 11:22:27 +0200
changeset 9013 9dd0274f76af
parent 8838 4eaa99f0d223
child 9035 371f023d3dbd
permissions -rw-r--r--
Updated files to remove 0r and 1r from theorems in descendant theories of RealBin. Some new theorems added.
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/Aux.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
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
     6
header {* Auxiliary theorems *};
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
     7
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
     8
theory Aux = Real + Zorn:;
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
     9
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    10
text {* Some existing theorems are declared as extra introduction
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    11
or elimination rules, respectively. *};
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    12
8203
2fcc6017cb72 intro/elim/dest attributes: changed ! / !! flags to ? / ??;
wenzelm
parents: 7978
diff changeset
    13
lemmas [intro??] = isLub_isUb;
2fcc6017cb72 intro/elim/dest attributes: changed ! / !! flags to ? / ??;
wenzelm
parents: 7978
diff changeset
    14
lemmas [intro??] = chainD; 
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    15
lemmas chainE2 = chainD2 [elimify];
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    16
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    17
text_raw {* \medskip *};
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7917
diff changeset
    18
text{* Lemmas about sets. *};
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    19
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    20
lemma Int_singletonD: "[| A Int B = {v}; x:A; x:B |] ==> x = v";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    21
  by (fast elim: equalityE);
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    22
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    23
lemma set_less_imp_diff_not_empty: "H < E ==> EX x0:E. x0 ~: H";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    24
 by (force simp add: psubset_eq);
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    25
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    26
text_raw {* \medskip *};
7978
1b99ee57d131 final update by Gertrud Bauer;
wenzelm
parents: 7917
diff changeset
    27
text{* Some lemmas about orders. *};
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    28
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    29
lemma lt_imp_not_eq: "x < (y::'a::order) ==> x ~= y"; 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    30
  by (rule order_less_le[RS iffD1, RS conjunct2]);
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    31
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    32
lemma le_noteq_imp_less: 
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    33
  "[| x <= (r::'a::order); x ~= r |] ==> x < r";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    34
proof -;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    35
  assume "x <= (r::'a::order)" and ne:"x ~= r";
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    36
  hence "x < r | x = r"; by (simp add: order_le_less);
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    37
  with ne; show ?thesis; by simp;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    38
qed;
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    39
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    40
text_raw {* \medskip *};
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    41
text {* Some lemmas about linear orders. *};
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
    42
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
    43
theorem linorder_linear_split: 
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
    44
"[| x < a ==> Q; x = a ==> Q; a < (x::'a::linorder) ==> Q |] ==> Q";
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    45
  by (rule linorder_less_linear [of x a, elimify]) force+;
7566
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
    46
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
    47
lemma le_max1: "x <= max x (y::'a::linorder)";
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
    48
  by (simp add: le_max_iff_disj[of x x y]);
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
    49
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
    50
lemma le_max2: "y <= max x (y::'a::linorder)"; 
c5a3f980a7af accomodate refined facts handling;
wenzelm
parents: 7535
diff changeset
    51
  by (simp add: le_max_iff_disj[of y x y]);
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    52
7917
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    53
text_raw {* \medskip *};
5e5b9813cce7 HahnBanach update by Gertrud Bauer;
wenzelm
parents: 7808
diff changeset
    54
text{* Some lemmas for the reals. *};
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    55
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    56
lemma real_add_minus_eq: "x - y = (#0::real) ==> x = y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    57
  by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    58
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    59
lemma abs_minus_one: "abs (- (#1::real)) = #1"; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    60
  by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    61
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    62
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    63
lemma real_mult_le_le_mono1a: 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    64
  "[| (#0::real) <= z; x <= y |] ==> z * x  <= z * y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    65
proof -;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    66
  assume "(#0::real) <= z" "x <= y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    67
  hence "x < y | x = y"; by (force simp add: order_le_less);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    68
  thus ?thesis;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    69
  proof (elim disjE); 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    70
   assume "x < y"; show ?thesis; by (rule real_mult_le_less_mono2) simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    71
  next; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    72
   assume "x = y"; thus ?thesis;; by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    73
  qed;
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    74
qed;
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    75
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
    76
lemma real_mult_le_le_mono2: 
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    77
  "[| (#0::real) <= z; x <= y |] ==> x * z <= y * z";
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    78
proof -;
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    79
  assume "(#0::real) <= z" "x <= y";
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    80
  hence "x < y | x = y"; by (force simp add: order_le_less);
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    81
  thus ?thesis;
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    82
  proof (elim disjE); 
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    83
   assume "x < y"; show ?thesis; by (rule real_mult_le_less_mono1) simp;
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    84
  next; 
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    85
   assume "x = y"; thus ?thesis;; by simp;
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    86
  qed;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    87
qed;
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
    88
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
    89
lemma real_mult_less_le_anti: 
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    90
  "[| z < (#0::real); x <= y |] ==> z * y <= z * x";
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
    91
proof -;
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    92
  assume "z < (#0::real)" "x <= y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    93
  hence "(#0::real) < - z"; by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    94
  hence "(#0::real) <= - z"; by (rule real_less_imp_le);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    95
  hence "x * (- z) <= y * (- z)"; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    96
    by (rule real_mult_le_le_mono2);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    97
  hence  "- (x * z) <= - (y * z)"; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    98
    by (simp only: real_minus_mult_eq2);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
    99
  thus ?thesis; by (simp only: real_mult_commute);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   100
qed;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   101
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   102
lemma real_mult_less_le_mono: 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   103
  "[| (#0::real) < z; x <= y |] ==> z * x <= z * y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   104
proof -; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   105
  assume "(#0::real) < z" "x <= y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   106
  have "(#0::real) <= z"; by (rule real_less_imp_le);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   107
  hence "x * z <= y * z"; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   108
    by (rule real_mult_le_le_mono2);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   109
  thus ?thesis; by (simp only: real_mult_commute);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   110
qed;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   111
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   112
lemma real_rinv_gt_zero1: "#0 < x ==> #0 < rinv x";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   113
proof -; 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   114
  assume "#0 < x";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   115
  have "0r < x"; by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   116
  hence "0r < rinv x"; by (rule real_rinv_gt_zero);
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   117
  thus ?thesis; by simp;
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   118
qed;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   119
9013
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   120
lemma real_mult_inv_right1: "x ~= #0 ==> x*rinv(x) = #1";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   121
   by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   122
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   123
lemma real_mult_inv_left1: "x ~= #0 ==> rinv(x)*x = #1";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   124
   by simp;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   125
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   126
lemma real_le_mult_order1a: 
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   127
      "[| (#0::real) <= x; #0 <= y |] ==> #0 <= x * y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   128
proof -;
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   129
  assume "#0 <= x" "#0 <= y";
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   130
    have "[|0r <= x; 0r <= y|] ==> 0r <= x * y";  
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   131
      by (rule real_le_mult_order);
9dd0274f76af Updated files to remove 0r and 1r from theorems in descendant theories
fleuriot
parents: 8838
diff changeset
   132
    thus ?thesis; by (simp!);
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   133
qed;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   134
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   135
lemma real_mult_diff_distrib: 
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   136
  "a * (- x - (y::real)) = - a * x - a * y";
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   137
proof -;
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   138
  have "- x - y = - x + - y"; by simp;
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   139
  also; have "a * ... = a * - x + a * - y"; 
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   140
    by (simp only: real_add_mult_distrib2);
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   141
  also; have "... = - a * x - a * y"; 
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   142
    by (simp add: real_minus_mult_eq2 [RS sym] real_minus_mult_eq1);
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   143
  finally; show ?thesis; .;
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   144
qed;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   145
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   146
lemma real_mult_diff_distrib2: "a * (x - (y::real)) = a * x - a * y";
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   147
proof -; 
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   148
  have "x - y = x + - y"; by simp;
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   149
  also; have "a * ... = a * x + a * - y"; 
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   150
    by (simp only: real_add_mult_distrib2);
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   151
  also; have "... = a * x - a * y";   
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   152
    by (simp add: real_minus_mult_eq2 [RS sym] real_minus_mult_eq1);
7656
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   153
  finally; show ?thesis; .;
2f18c0ffc348 update from Gertrud;
wenzelm
parents: 7566
diff changeset
   154
qed;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   155
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   156
lemma real_minus_le: "- (x::real) <= y ==> - y <= x";
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   157
  by simp;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   158
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   159
lemma real_diff_ineq_swap: 
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   160
  "(d::real) - b <= c + a ==> - a - b <= c - d";
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   161
  by simp;
7535
599d3414b51d The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
wenzelm
parents:
diff changeset
   162
7808
fd019ac3485f update from Gertrud;
wenzelm
parents: 7656
diff changeset
   163
end;