author | kleing |
Tue, 13 May 2003 08:59:21 +0200 | |
changeset 14024 | 213dcc39358f |
parent 13966 | 2160abf7cfe7 |
child 14051 | 4b61bbb0dcab |
permissions | -rw-r--r-- |
13966
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
1 |
(* Title: HOL/Real/ex/BinEx.thy |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
2 |
ID: $Id$ |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
4 |
Copyright 1999 University of Cambridge |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
5 |
*) |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
6 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
7 |
header {* Binary arithmetic examples *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
8 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
9 |
theory BinEx = Real: |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
10 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
11 |
text {* |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
12 |
Examples of performing binary arithmetic by simplification This time |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
13 |
we use the reals, though the representation is just of integers. |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
14 |
*} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
15 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
16 |
text {* \medskip Addition *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
17 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
18 |
lemma "(1359::real) + -2468 = -1109" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
19 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
20 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
21 |
lemma "(93746::real) + -46375 = 47371" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
22 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
23 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
24 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
25 |
text {* \medskip Negation *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
26 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
27 |
lemma "- (65745::real) = -65745" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
28 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
29 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
30 |
lemma "- (-54321::real) = 54321" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
31 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
32 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
33 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
34 |
text {* \medskip Multiplication *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
35 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
36 |
lemma "(-84::real) * 51 = -4284" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
37 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
38 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
39 |
lemma "(255::real) * 255 = 65025" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
40 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
41 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
42 |
lemma "(1359::real) * -2468 = -3354012" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
43 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
44 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
45 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
46 |
text {* \medskip Inequalities *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
47 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
48 |
lemma "(89::real) * 10 \<noteq> 889" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
49 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
50 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
51 |
lemma "(13::real) < 18 - 4" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
52 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
53 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
54 |
lemma "(-345::real) < -242 + -100" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
55 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
56 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
57 |
lemma "(13557456::real) < 18678654" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
58 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
59 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
60 |
lemma "(999999::real) \<le> (1000001 + 1) - 2" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
61 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
62 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
63 |
lemma "(1234567::real) \<le> 1234567" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
64 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
65 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
66 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
67 |
text {* \medskip Powers *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
68 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
69 |
lemma "2 ^ 15 = (32768::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
70 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
71 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
72 |
lemma "-3 ^ 7 = (-2187::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
73 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
74 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
75 |
lemma "13 ^ 7 = (62748517::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
76 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
77 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
78 |
lemma "3 ^ 15 = (14348907::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
79 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
80 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
81 |
lemma "-5 ^ 11 = (-48828125::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
82 |
by simp |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
83 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
84 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
85 |
text {* \medskip Tests *} |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
86 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
87 |
lemma "(x + y = x) = (y = (0::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
88 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
89 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
90 |
lemma "(x + y = y) = (x = (0::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
91 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
92 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
93 |
lemma "(x + y = (0::real)) = (x = -y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
94 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
95 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
96 |
lemma "(x + y = (0::real)) = (y = -x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
97 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
98 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
99 |
lemma "((x + y) < (x + z)) = (y < (z::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
100 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
101 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
102 |
lemma "((x + z) < (y + z)) = (x < (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
103 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
104 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
105 |
lemma "(\<not> x < y) = (y \<le> (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
106 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
107 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
108 |
lemma "\<not> (x < y \<and> y < (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
109 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
110 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
111 |
lemma "(x::real) < y ==> \<not> y < x" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
112 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
113 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
114 |
lemma "((x::real) \<noteq> y) = (x < y \<or> y < x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
115 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
116 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
117 |
lemma "(\<not> x \<le> y) = (y < (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
118 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
119 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
120 |
lemma "x \<le> y \<or> y \<le> (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
121 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
122 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
123 |
lemma "x \<le> y \<or> y < (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
124 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
125 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
126 |
lemma "x < y \<or> y \<le> (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
127 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
128 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
129 |
lemma "x \<le> (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
130 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
131 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
132 |
lemma "((x::real) \<le> y) = (x < y \<or> x = y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
133 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
134 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
135 |
lemma "((x::real) \<le> y \<and> y \<le> x) = (x = y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
136 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
137 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
138 |
lemma "\<not>(x < y \<and> y \<le> (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
139 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
140 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
141 |
lemma "\<not>(x \<le> y \<and> y < (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
142 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
143 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
144 |
lemma "(-x < (0::real)) = (0 < x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
145 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
146 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
147 |
lemma "((0::real) < -x) = (x < 0)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
148 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
149 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
150 |
lemma "(-x \<le> (0::real)) = (0 \<le> x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
151 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
152 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
153 |
lemma "((0::real) \<le> -x) = (x \<le> 0)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
154 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
155 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
156 |
lemma "(x::real) = y \<or> x < y \<or> y < x" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
157 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
158 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
159 |
lemma "(x::real) = 0 \<or> 0 < x \<or> 0 < -x" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
160 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
161 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
162 |
lemma "(0::real) \<le> x \<or> 0 \<le> -x" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
163 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
164 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
165 |
lemma "((x::real) + y \<le> x + z) = (y \<le> z)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
166 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
167 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
168 |
lemma "((x::real) + z \<le> y + z) = (x \<le> y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
169 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
170 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
171 |
lemma "(w::real) < x \<and> y < z ==> w + y < x + z" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
172 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
173 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
174 |
lemma "(w::real) \<le> x \<and> y \<le> z ==> w + y \<le> x + z" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
175 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
176 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
177 |
lemma "(0::real) \<le> x \<and> 0 \<le> y ==> 0 \<le> x + y" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
178 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
179 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
180 |
lemma "(0::real) < x \<and> 0 < y ==> 0 < x + y" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
181 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
182 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
183 |
lemma "(-x < y) = (0 < x + (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
184 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
185 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
186 |
lemma "(x < -y) = (x + y < (0::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
187 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
188 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
189 |
lemma "(y < x + -z) = (y + z < (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
190 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
191 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
192 |
lemma "(x + -y < z) = (x < z + (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
193 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
194 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
195 |
lemma "x \<le> y ==> x < y + (1::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
196 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
197 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
198 |
lemma "(x - y) + y = (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
199 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
200 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
201 |
lemma "y + (x - y) = (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
202 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
203 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
204 |
lemma "x - x = (0::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
205 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
206 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
207 |
lemma "(x - y = 0) = (x = (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
208 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
209 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
210 |
lemma "((0::real) \<le> x + x) = (0 \<le> x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
211 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
212 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
213 |
lemma "(-x \<le> x) = ((0::real) \<le> x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
214 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
215 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
216 |
lemma "(x \<le> -x) = (x \<le> (0::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
217 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
218 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
219 |
lemma "(-x = (0::real)) = (x = 0)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
220 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
221 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
222 |
lemma "-(x - y) = y - (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
223 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
224 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
225 |
lemma "((0::real) < x - y) = (y < x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
226 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
227 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
228 |
lemma "((0::real) \<le> x - y) = (y \<le> x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
229 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
230 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
231 |
lemma "(x + y) - x = (y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
232 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
233 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
234 |
lemma "(-x = y) = (x = (-y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
235 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
236 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
237 |
lemma "x < (y::real) ==> \<not>(x = y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
238 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
239 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
240 |
lemma "(x \<le> x + y) = ((0::real) \<le> y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
241 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
242 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
243 |
lemma "(y \<le> x + y) = ((0::real) \<le> x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
244 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
245 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
246 |
lemma "(x < x + y) = ((0::real) < y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
247 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
248 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
249 |
lemma "(y < x + y) = ((0::real) < x)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
250 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
251 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
252 |
lemma "(x - y) - x = (-y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
253 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
254 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
255 |
lemma "(x + y < z) = (x < z - (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
256 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
257 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
258 |
lemma "(x - y < z) = (x < z + (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
259 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
260 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
261 |
lemma "(x < y - z) = (x + z < (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
262 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
263 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
264 |
lemma "(x \<le> y - z) = (x + z \<le> (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
265 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
266 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
267 |
lemma "(x - y \<le> z) = (x \<le> z + (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
268 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
269 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
270 |
lemma "(-x < -y) = (y < (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
271 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
272 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
273 |
lemma "(-x \<le> -y) = (y \<le> (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
274 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
275 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
276 |
lemma "(a + b) - (c + d) = (a - c) + (b - (d::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
277 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
278 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
279 |
lemma "(0::real) - x = -x" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
280 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
281 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
282 |
lemma "x - (0::real) = x" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
283 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
284 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
285 |
lemma "w \<le> x \<and> y < z ==> w + y < x + (z::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
286 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
287 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
288 |
lemma "w < x \<and> y \<le> z ==> w + y < x + (z::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
289 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
290 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
291 |
lemma "(0::real) \<le> x \<and> 0 < y ==> 0 < x + (y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
292 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
293 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
294 |
lemma "(0::real) < x \<and> 0 \<le> y ==> 0 < x + y" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
295 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
296 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
297 |
lemma "-x - y = -(x + (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
298 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
299 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
300 |
lemma "x - (-y) = x + (y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
301 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
302 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
303 |
lemma "-x - -y = y - (x::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
304 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
305 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
306 |
lemma "(a - b) + (b - c) = a - (c::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
307 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
308 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
309 |
lemma "(x = y - z) = (x + z = (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
310 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
311 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
312 |
lemma "(x - y = z) = (x = z + (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
313 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
314 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
315 |
lemma "x - (x - y) = (y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
316 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
317 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
318 |
lemma "x - (x + y) = -(y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
319 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
320 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
321 |
lemma "x = y ==> x \<le> (y::real)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
322 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
323 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
324 |
lemma "(0::real) < x ==> \<not>(x = 0)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
325 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
326 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
327 |
lemma "(x + y) * (x - y) = (x * x) - (y * y)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
328 |
oops |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
329 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
330 |
lemma "(-x = -y) = (x = (y::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
331 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
332 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
333 |
lemma "(-x < -y) = (y < (x::real))" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
334 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
335 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
336 |
lemma "!!a::real. a \<le> b ==> c \<le> d ==> x + y < z ==> a + c \<le> b + d" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
337 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
338 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
339 |
lemma "!!a::real. a < b ==> c < d ==> a - d \<le> b + (-c)" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
340 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
341 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
342 |
lemma "!!a::real. a \<le> b ==> b + b \<le> c ==> a + a \<le> c" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
343 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
344 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
345 |
lemma "!!a::real. a + b \<le> i + j ==> a \<le> b ==> i \<le> j ==> a + a \<le> j + j" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
346 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
347 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
348 |
lemma "!!a::real. a + b < i + j ==> a < b ==> i < j ==> a + a < j + j" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
349 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
350 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
351 |
lemma "!!a::real. a + b + c \<le> i + j + k \<and> a \<le> b \<and> b \<le> c \<and> i \<le> j \<and> j \<le> k --> a + a + a \<le> k + k + k" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
352 |
by arith |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
353 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
354 |
lemma "!!a::real. a + b + c + d \<le> i + j + k + l ==> a \<le> b ==> b \<le> c |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
355 |
==> c \<le> d ==> i \<le> j ==> j \<le> k ==> k \<le> l ==> a \<le> l" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
356 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
357 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
358 |
lemma "!!a::real. a + b + c + d \<le> i + j + k + l ==> a \<le> b ==> b \<le> c |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
359 |
==> c \<le> d ==> i \<le> j ==> j \<le> k ==> k \<le> l ==> a + a + a + a \<le> l + l + l + l" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
360 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
361 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
362 |
lemma "!!a::real. a + b + c + d \<le> i + j + k + l ==> a \<le> b ==> b \<le> c |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
363 |
==> c \<le> d ==> i \<le> j ==> j \<le> k ==> k \<le> l ==> a + a + a + a + a \<le> l + l + l + l + i" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
364 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
365 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
366 |
lemma "!!a::real. a + b + c + d \<le> i + j + k + l ==> a \<le> b ==> b \<le> c |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
367 |
==> c \<le> d ==> i \<le> j ==> j \<le> k ==> k \<le> l ==> a + a + a + a + a + a \<le> l + l + l + l + i + l" |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
368 |
by (tactic "fast_arith_tac 1") |
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
369 |
|
2160abf7cfe7
removal of the image HOL-Real and merging of HOL-Real-ex with HOL-Complex-ex
paulson
parents:
diff
changeset
|
370 |
end |