src/HOL/Integ/IntDef.ML
author paulson
Fri, 18 Sep 1998 16:04:00 +0200
changeset 5508 691c70898518
child 5540 0f16c3b66ab4
permissions -rw-r--r--
new files in Integ
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
5508
691c70898518 new files in Integ
paulson
parents:
diff changeset
     1
(*  Title:      IntDef.ML
691c70898518 new files in Integ
paulson
parents:
diff changeset
     2
    ID:         $Id$
691c70898518 new files in Integ
paulson
parents:
diff changeset
     3
    Authors:    Lawrence C Paulson, Cambridge University Computer Laboratory
691c70898518 new files in Integ
paulson
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
691c70898518 new files in Integ
paulson
parents:
diff changeset
     5
691c70898518 new files in Integ
paulson
parents:
diff changeset
     6
The integers as equivalence classes over nat*nat.
691c70898518 new files in Integ
paulson
parents:
diff changeset
     7
*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
     8
691c70898518 new files in Integ
paulson
parents:
diff changeset
     9
691c70898518 new files in Integ
paulson
parents:
diff changeset
    10
(*** Proving that intrel is an equivalence relation ***)
691c70898518 new files in Integ
paulson
parents:
diff changeset
    11
691c70898518 new files in Integ
paulson
parents:
diff changeset
    12
val eqa::eqb::prems = goal Arith.thy 
691c70898518 new files in Integ
paulson
parents:
diff changeset
    13
    "[| (x1::nat) + y2 = x2 + y1; x2 + y3 = x3 + y2 |] ==> \
691c70898518 new files in Integ
paulson
parents:
diff changeset
    14
\       x1 + y3 = x3 + y1";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    15
by (res_inst_tac [("k1","x2")] (add_left_cancel RS iffD1) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    16
by (rtac (add_left_commute RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    17
by (stac eqb 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    18
by (rtac (add_left_commute RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    19
by (stac eqa 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    20
by (rtac (add_left_commute) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    21
qed "integ_trans_lemma";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    22
691c70898518 new files in Integ
paulson
parents:
diff changeset
    23
(** Natural deduction for intrel **)
691c70898518 new files in Integ
paulson
parents:
diff changeset
    24
691c70898518 new files in Integ
paulson
parents:
diff changeset
    25
Goalw  [intrel_def] "[| x1+y2 = x2+y1|] ==> ((x1,y1),(x2,y2)): intrel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    26
by (Fast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    27
qed "intrelI";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    28
691c70898518 new files in Integ
paulson
parents:
diff changeset
    29
(*intrelE is hard to derive because fast_tac tries hyp_subst_tac so soon*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
    30
Goalw [intrel_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
    31
  "p: intrel --> (EX x1 y1 x2 y2. \
691c70898518 new files in Integ
paulson
parents:
diff changeset
    32
\                  p = ((x1,y1),(x2,y2)) & x1+y2 = x2+y1)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    33
by (Fast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    34
qed "intrelE_lemma";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    35
691c70898518 new files in Integ
paulson
parents:
diff changeset
    36
val [major,minor] = Goal
691c70898518 new files in Integ
paulson
parents:
diff changeset
    37
  "[| p: intrel;  \
691c70898518 new files in Integ
paulson
parents:
diff changeset
    38
\     !!x1 y1 x2 y2. [| p = ((x1,y1),(x2,y2));  x1+y2 = x2+y1|] ==> Q |] \
691c70898518 new files in Integ
paulson
parents:
diff changeset
    39
\  ==> Q";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    40
by (cut_facts_tac [major RS (intrelE_lemma RS mp)] 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    41
by (REPEAT (eresolve_tac [asm_rl,exE,conjE,minor] 1));
691c70898518 new files in Integ
paulson
parents:
diff changeset
    42
qed "intrelE";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    43
691c70898518 new files in Integ
paulson
parents:
diff changeset
    44
AddSIs [intrelI];
691c70898518 new files in Integ
paulson
parents:
diff changeset
    45
AddSEs [intrelE];
691c70898518 new files in Integ
paulson
parents:
diff changeset
    46
691c70898518 new files in Integ
paulson
parents:
diff changeset
    47
Goal "((x1,y1),(x2,y2)): intrel = (x1+y2 = x2+y1)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    48
by (Fast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    49
qed "intrel_iff";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    50
691c70898518 new files in Integ
paulson
parents:
diff changeset
    51
Goal "(x,x): intrel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    52
by (stac surjective_pairing 1 THEN rtac (refl RS intrelI) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    53
qed "intrel_refl";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    54
691c70898518 new files in Integ
paulson
parents:
diff changeset
    55
Goalw [equiv_def, refl_def, sym_def, trans_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
    56
    "equiv {x::(nat*nat).True} intrel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    57
by (fast_tac (claset() addSIs [intrel_refl] 
691c70898518 new files in Integ
paulson
parents:
diff changeset
    58
                        addSEs [sym, integ_trans_lemma]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    59
qed "equiv_intrel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    60
691c70898518 new files in Integ
paulson
parents:
diff changeset
    61
val equiv_intrel_iff =
691c70898518 new files in Integ
paulson
parents:
diff changeset
    62
    [TrueI, TrueI] MRS 
691c70898518 new files in Integ
paulson
parents:
diff changeset
    63
    ([CollectI, CollectI] MRS 
691c70898518 new files in Integ
paulson
parents:
diff changeset
    64
    (equiv_intrel RS eq_equiv_class_iff));
691c70898518 new files in Integ
paulson
parents:
diff changeset
    65
691c70898518 new files in Integ
paulson
parents:
diff changeset
    66
Goalw  [Integ_def,intrel_def,quotient_def] "intrel^^{(x,y)}:Integ";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    67
by (Fast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    68
qed "intrel_in_integ";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    69
691c70898518 new files in Integ
paulson
parents:
diff changeset
    70
Goal "inj_on Abs_Integ Integ";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    71
by (rtac inj_on_inverseI 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    72
by (etac Abs_Integ_inverse 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    73
qed "inj_on_Abs_Integ";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    74
691c70898518 new files in Integ
paulson
parents:
diff changeset
    75
Addsimps [equiv_intrel_iff, inj_on_Abs_Integ RS inj_on_iff,
691c70898518 new files in Integ
paulson
parents:
diff changeset
    76
          intrel_iff, intrel_in_integ, Abs_Integ_inverse];
691c70898518 new files in Integ
paulson
parents:
diff changeset
    77
691c70898518 new files in Integ
paulson
parents:
diff changeset
    78
Goal "inj(Rep_Integ)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    79
by (rtac inj_inverseI 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    80
by (rtac Rep_Integ_inverse 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    81
qed "inj_Rep_Integ";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    82
691c70898518 new files in Integ
paulson
parents:
diff changeset
    83
691c70898518 new files in Integ
paulson
parents:
diff changeset
    84
(** znat: the injection from nat to Integ **)
691c70898518 new files in Integ
paulson
parents:
diff changeset
    85
691c70898518 new files in Integ
paulson
parents:
diff changeset
    86
Goal "inj(znat)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    87
by (rtac injI 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    88
by (rewtac znat_def);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    89
by (dtac (inj_on_Abs_Integ RS inj_onD) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    90
by (REPEAT (rtac intrel_in_integ 1));
691c70898518 new files in Integ
paulson
parents:
diff changeset
    91
by (dtac eq_equiv_class 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    92
by (rtac equiv_intrel 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    93
by (Fast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    94
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
    95
by (Asm_full_simp_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
    96
qed "inj_znat";
691c70898518 new files in Integ
paulson
parents:
diff changeset
    97
691c70898518 new files in Integ
paulson
parents:
diff changeset
    98
691c70898518 new files in Integ
paulson
parents:
diff changeset
    99
(**** zminus: unary negation on Integ ****)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   100
691c70898518 new files in Integ
paulson
parents:
diff changeset
   101
Goalw [congruent_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
   102
  "congruent intrel (%p. split (%x y. intrel^^{(y,x)}) p)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   103
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   104
by (asm_simp_tac (simpset() addsimps add_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   105
qed "zminus_congruent";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   106
691c70898518 new files in Integ
paulson
parents:
diff changeset
   107
691c70898518 new files in Integ
paulson
parents:
diff changeset
   108
(*Resolve th against the corresponding facts for zminus*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   109
val zminus_ize = RSLIST [equiv_intrel, zminus_congruent];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   110
691c70898518 new files in Integ
paulson
parents:
diff changeset
   111
Goalw [zminus_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
   112
      "- Abs_Integ(intrel^^{(x,y)}) = Abs_Integ(intrel ^^ {(y,x)})";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   113
by (res_inst_tac [("f","Abs_Integ")] arg_cong 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   114
by (simp_tac (simpset() addsimps 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   115
   [intrel_in_integ RS Abs_Integ_inverse,zminus_ize UN_equiv_class]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   116
qed "zminus";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   117
691c70898518 new files in Integ
paulson
parents:
diff changeset
   118
(*by lcp*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   119
val [prem] = Goal "(!!x y. z = Abs_Integ(intrel^^{(x,y)}) ==> P) ==> P";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   120
by (res_inst_tac [("x1","z")] 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   121
    (rewrite_rule [Integ_def] Rep_Integ RS quotientE) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   122
by (dres_inst_tac [("f","Abs_Integ")] arg_cong 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   123
by (res_inst_tac [("p","x")] PairE 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   124
by (rtac prem 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   125
by (asm_full_simp_tac (simpset() addsimps [Rep_Integ_inverse]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   126
qed "eq_Abs_Integ";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   127
691c70898518 new files in Integ
paulson
parents:
diff changeset
   128
Goal "- (- z) = (z::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   129
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   130
by (asm_simp_tac (simpset() addsimps [zminus]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   131
qed "zminus_zminus";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   132
Addsimps [zminus_zminus];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   133
691c70898518 new files in Integ
paulson
parents:
diff changeset
   134
Goal "inj(uminus::int=>int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   135
by (rtac injI 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   136
by (dres_inst_tac [("f","uminus")] arg_cong 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   137
by (Asm_full_simp_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   138
qed "inj_zminus";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   139
691c70898518 new files in Integ
paulson
parents:
diff changeset
   140
Goalw [znat_def] "- ($# 0) = $# 0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   141
by (simp_tac (simpset() addsimps [zminus]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   142
qed "zminus_nat0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   143
691c70898518 new files in Integ
paulson
parents:
diff changeset
   144
Addsimps [zminus_nat0];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   145
691c70898518 new files in Integ
paulson
parents:
diff changeset
   146
691c70898518 new files in Integ
paulson
parents:
diff changeset
   147
(**** znegative: the test for negative integers ****)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   148
691c70898518 new files in Integ
paulson
parents:
diff changeset
   149
691c70898518 new files in Integ
paulson
parents:
diff changeset
   150
Goalw [znegative_def, znat_def] "~ znegative($# n)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   151
by (Simp_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   152
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   153
qed "not_znegative_znat";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   154
691c70898518 new files in Integ
paulson
parents:
diff changeset
   155
Goalw [znegative_def, znat_def] "znegative(- $# Suc(n))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   156
by (simp_tac (simpset() addsimps [zminus]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   157
qed "znegative_zminus_znat";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   158
691c70898518 new files in Integ
paulson
parents:
diff changeset
   159
Addsimps [znegative_zminus_znat, not_znegative_znat]; 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   160
691c70898518 new files in Integ
paulson
parents:
diff changeset
   161
691c70898518 new files in Integ
paulson
parents:
diff changeset
   162
(**** zadd: addition on Integ ****)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   163
691c70898518 new files in Integ
paulson
parents:
diff changeset
   164
(** Congruence property for addition **)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   165
691c70898518 new files in Integ
paulson
parents:
diff changeset
   166
Goalw [congruent2_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
   167
    "congruent2 intrel (%p1 p2.                  \
691c70898518 new files in Integ
paulson
parents:
diff changeset
   168
\         split (%x1 y1. split (%x2 y2. intrel^^{(x1+x2, y1+y2)}) p2) p1)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   169
(*Proof via congruent2_commuteI seems longer*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   170
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   171
by (asm_simp_tac (simpset() addsimps [add_assoc]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   172
(*The rest should be trivial, but rearranging terms is hard*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   173
by (res_inst_tac [("x1","x1a")] (add_left_commute RS ssubst) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   174
by (asm_simp_tac (simpset() addsimps [add_assoc RS sym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   175
qed "zadd_congruent2";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   176
691c70898518 new files in Integ
paulson
parents:
diff changeset
   177
(*Resolve th against the corresponding facts for zadd*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   178
val zadd_ize = RSLIST [equiv_intrel, zadd_congruent2];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   179
691c70898518 new files in Integ
paulson
parents:
diff changeset
   180
Goalw [zadd_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
   181
  "Abs_Integ(intrel^^{(x1,y1)}) + Abs_Integ(intrel^^{(x2,y2)}) = \
691c70898518 new files in Integ
paulson
parents:
diff changeset
   182
\  Abs_Integ(intrel^^{(x1+x2, y1+y2)})";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   183
by (asm_simp_tac
691c70898518 new files in Integ
paulson
parents:
diff changeset
   184
    (simpset() addsimps [zadd_ize UN_equiv_class2]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   185
qed "zadd";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   186
691c70898518 new files in Integ
paulson
parents:
diff changeset
   187
Goal "- (z + w) = - z + - (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   188
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   189
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   190
by (asm_simp_tac (simpset() addsimps [zminus,zadd]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   191
qed "zminus_zadd_distrib";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   192
Addsimps [zminus_zadd_distrib];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   193
691c70898518 new files in Integ
paulson
parents:
diff changeset
   194
Goal "(z::int) + w = w + z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   195
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   196
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   197
by (asm_simp_tac (simpset() addsimps (add_ac @ [zadd])) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   198
qed "zadd_commute";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   199
691c70898518 new files in Integ
paulson
parents:
diff changeset
   200
Goal "((z1::int) + z2) + z3 = z1 + (z2 + z3)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   201
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   202
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   203
by (res_inst_tac [("z","z3")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   204
by (asm_simp_tac (simpset() addsimps [zadd, add_assoc]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   205
qed "zadd_assoc";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   206
691c70898518 new files in Integ
paulson
parents:
diff changeset
   207
(*For AC rewriting*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   208
Goal "(x::int)+(y+z)=y+(x+z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   209
by (rtac (zadd_commute RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   210
by (rtac (zadd_assoc RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   211
by (rtac (zadd_commute RS arg_cong) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   212
qed "zadd_left_commute";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   213
691c70898518 new files in Integ
paulson
parents:
diff changeset
   214
(*Integer addition is an AC operator*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   215
val zadd_ac = [zadd_assoc,zadd_commute,zadd_left_commute];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   216
691c70898518 new files in Integ
paulson
parents:
diff changeset
   217
Goalw [znat_def] "($#m) + ($#n) = $# (m + n)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   218
by (simp_tac (simpset() addsimps [zadd]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   219
qed "add_znat";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   220
691c70898518 new files in Integ
paulson
parents:
diff changeset
   221
Goal "$# (Suc m) = $# 1 + ($# m)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   222
by (simp_tac (simpset() addsimps [add_znat]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   223
qed "znat_Suc";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   224
691c70898518 new files in Integ
paulson
parents:
diff changeset
   225
Goalw [znat_def] "$# 0 + z = z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   226
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   227
by (asm_simp_tac (simpset() addsimps [zadd]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   228
qed "zadd_nat0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   229
691c70898518 new files in Integ
paulson
parents:
diff changeset
   230
Goal "z + $# 0 = z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   231
by (rtac (zadd_commute RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   232
by (rtac zadd_nat0 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   233
qed "zadd_nat0_right";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   234
691c70898518 new files in Integ
paulson
parents:
diff changeset
   235
Goalw [znat_def] "z + (- z) = $# 0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   236
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   237
by (asm_simp_tac (simpset() addsimps [zminus, zadd, add_commute]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   238
qed "zadd_zminus_inverse_nat";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   239
691c70898518 new files in Integ
paulson
parents:
diff changeset
   240
Goal "(- z) + z = $# 0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   241
by (rtac (zadd_commute RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   242
by (rtac zadd_zminus_inverse_nat 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   243
qed "zadd_zminus_inverse_nat2";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   244
691c70898518 new files in Integ
paulson
parents:
diff changeset
   245
Addsimps [zadd_nat0, zadd_nat0_right,
691c70898518 new files in Integ
paulson
parents:
diff changeset
   246
	  zadd_zminus_inverse_nat, zadd_zminus_inverse_nat2];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   247
691c70898518 new files in Integ
paulson
parents:
diff changeset
   248
Goal "z + (- z + w) = (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   249
by (asm_simp_tac (simpset() addsimps [zadd_assoc RS sym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   250
qed "zadd_zminus_cancel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   251
691c70898518 new files in Integ
paulson
parents:
diff changeset
   252
Goal "(-z) + (z + w) = (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   253
by (asm_simp_tac (simpset() addsimps [zadd_assoc RS sym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   254
qed "zminus_zadd_cancel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   255
691c70898518 new files in Integ
paulson
parents:
diff changeset
   256
Addsimps [zadd_zminus_cancel, zminus_zadd_cancel];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   257
691c70898518 new files in Integ
paulson
parents:
diff changeset
   258
691c70898518 new files in Integ
paulson
parents:
diff changeset
   259
(** Lemmas **)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   260
691c70898518 new files in Integ
paulson
parents:
diff changeset
   261
Goal "(z::int) + v = z' + v' ==> z + (v + w) = z' + (v' + w)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   262
by (asm_simp_tac (simpset() addsimps [zadd_assoc RS sym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   263
qed "zadd_assoc_cong";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   264
691c70898518 new files in Integ
paulson
parents:
diff changeset
   265
Goal "(z::int) + (v + w) = v + (z + w)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   266
by (REPEAT (ares_tac [zadd_commute RS zadd_assoc_cong] 1));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   267
qed "zadd_assoc_swap";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   268
691c70898518 new files in Integ
paulson
parents:
diff changeset
   269
691c70898518 new files in Integ
paulson
parents:
diff changeset
   270
(*Need properties of subtraction?  Or use $- just as an abbreviation!*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   271
691c70898518 new files in Integ
paulson
parents:
diff changeset
   272
(**** zmult: multiplication on Integ ****)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   273
691c70898518 new files in Integ
paulson
parents:
diff changeset
   274
(** Congruence property for multiplication **)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   275
691c70898518 new files in Integ
paulson
parents:
diff changeset
   276
Goal "((k::nat) + l) + (m + n) = (k + m) + (n + l)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   277
by (simp_tac (simpset() addsimps add_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   278
qed "zmult_congruent_lemma";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   279
691c70898518 new files in Integ
paulson
parents:
diff changeset
   280
Goal "congruent2 intrel (%p1 p2.                 \
691c70898518 new files in Integ
paulson
parents:
diff changeset
   281
\               split (%x1 y1. split (%x2 y2.   \
691c70898518 new files in Integ
paulson
parents:
diff changeset
   282
\                   intrel^^{(x1*x2 + y1*y2, x1*y2 + y1*x2)}) p2) p1)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   283
by (rtac (equiv_intrel RS congruent2_commuteI) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   284
by (pair_tac "w" 2);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   285
by (rename_tac "z1 z2" 2);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   286
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   287
by (rewtac split_def);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   288
by (simp_tac (simpset() addsimps add_ac@mult_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   289
by (asm_simp_tac (simpset() delsimps [equiv_intrel_iff]
691c70898518 new files in Integ
paulson
parents:
diff changeset
   290
                           addsimps add_ac@mult_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   291
by (rtac (intrelI RS(equiv_intrel RS equiv_class_eq)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   292
by (rtac (zmult_congruent_lemma RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   293
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   294
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   295
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   296
by (asm_simp_tac (simpset() addsimps [add_mult_distrib RS sym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   297
by (asm_simp_tac (simpset() addsimps add_ac@mult_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   298
qed "zmult_congruent2";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   299
691c70898518 new files in Integ
paulson
parents:
diff changeset
   300
(*Resolve th against the corresponding facts for zmult*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   301
val zmult_ize = RSLIST [equiv_intrel, zmult_congruent2];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   302
691c70898518 new files in Integ
paulson
parents:
diff changeset
   303
Goalw [zmult_def]
691c70898518 new files in Integ
paulson
parents:
diff changeset
   304
   "Abs_Integ((intrel^^{(x1,y1)})) * Abs_Integ((intrel^^{(x2,y2)})) =   \
691c70898518 new files in Integ
paulson
parents:
diff changeset
   305
\   Abs_Integ(intrel ^^ {(x1*x2 + y1*y2, x1*y2 + y1*x2)})";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   306
by (simp_tac (simpset() addsimps [zmult_ize UN_equiv_class2]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   307
qed "zmult";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   308
691c70898518 new files in Integ
paulson
parents:
diff changeset
   309
Goal "(- z) * w = - (z * (w::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   310
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   311
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   312
by (asm_simp_tac (simpset() addsimps ([zminus, zmult] @ add_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   313
qed "zmult_zminus";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   314
691c70898518 new files in Integ
paulson
parents:
diff changeset
   315
691c70898518 new files in Integ
paulson
parents:
diff changeset
   316
Goal "(- z) * (- w) = (z * (w::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   317
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   318
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   319
by (asm_simp_tac (simpset() addsimps ([zminus, zmult] @ add_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   320
qed "zmult_zminus_zminus";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   321
691c70898518 new files in Integ
paulson
parents:
diff changeset
   322
Goal "(z::int) * w = w * z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   323
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   324
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   325
by (asm_simp_tac (simpset() addsimps ([zmult] @ add_ac @ mult_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   326
qed "zmult_commute";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   327
691c70898518 new files in Integ
paulson
parents:
diff changeset
   328
Goal "((z1::int) * z2) * z3 = z1 * (z2 * z3)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   329
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   330
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   331
by (res_inst_tac [("z","z3")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   332
by (asm_simp_tac (simpset() addsimps ([add_mult_distrib2,zmult] @ 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   333
                                     add_ac @ mult_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   334
qed "zmult_assoc";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   335
691c70898518 new files in Integ
paulson
parents:
diff changeset
   336
(*For AC rewriting*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   337
Goal "(z1::int)*(z2*z3) = z2*(z1*z3)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   338
by (rtac (zmult_commute RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   339
by (rtac (zmult_assoc RS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   340
by (rtac (zmult_commute RS arg_cong) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   341
qed "zmult_left_commute";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   342
691c70898518 new files in Integ
paulson
parents:
diff changeset
   343
(*Integer multiplication is an AC operator*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   344
val zmult_ac = [zmult_assoc, zmult_commute, zmult_left_commute];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   345
691c70898518 new files in Integ
paulson
parents:
diff changeset
   346
Goal "((z1::int) + z2) * w = (z1 * w) + (z2 * w)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   347
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   348
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   349
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   350
by (asm_simp_tac 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   351
    (simpset() addsimps ([add_mult_distrib2, zadd, zmult] @ 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   352
			 add_ac @ mult_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   353
qed "zadd_zmult_distrib";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   354
691c70898518 new files in Integ
paulson
parents:
diff changeset
   355
val zmult_commute'= read_instantiate [("z","w")] zmult_commute;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   356
691c70898518 new files in Integ
paulson
parents:
diff changeset
   357
Goal "w * (- z) = - (w * (z::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   358
by (simp_tac (simpset() addsimps [zmult_commute', zmult_zminus]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   359
qed "zmult_zminus_right";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   360
691c70898518 new files in Integ
paulson
parents:
diff changeset
   361
Goal "(w::int) * (z1 + z2) = (w * z1) + (w * z2)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   362
by (simp_tac (simpset() addsimps [zmult_commute',zadd_zmult_distrib]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   363
qed "zadd_zmult_distrib2";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   364
691c70898518 new files in Integ
paulson
parents:
diff changeset
   365
Goalw [znat_def] "$# 0 * z = $# 0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   366
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   367
by (asm_simp_tac (simpset() addsimps [zmult]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   368
qed "zmult_nat0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   369
691c70898518 new files in Integ
paulson
parents:
diff changeset
   370
Goalw [znat_def] "$# 1 * z = z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   371
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   372
by (asm_simp_tac (simpset() addsimps [zmult]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   373
qed "zmult_nat1";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   374
691c70898518 new files in Integ
paulson
parents:
diff changeset
   375
Goal "z * $# 0 = $# 0";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   376
by (rtac ([zmult_commute, zmult_nat0] MRS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   377
qed "zmult_nat0_right";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   378
691c70898518 new files in Integ
paulson
parents:
diff changeset
   379
Goal "z * $# 1 = z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   380
by (rtac ([zmult_commute, zmult_nat1] MRS trans) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   381
qed "zmult_nat1_right";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   382
691c70898518 new files in Integ
paulson
parents:
diff changeset
   383
Addsimps [zmult_nat0, zmult_nat0_right, zmult_nat1, zmult_nat1_right];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   384
691c70898518 new files in Integ
paulson
parents:
diff changeset
   385
691c70898518 new files in Integ
paulson
parents:
diff changeset
   386
Goal "(- z = w) = (z = - (w::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   387
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   388
by (rtac (zminus_zminus RS sym) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   389
by (rtac zminus_zminus 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   390
qed "zminus_exchange";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   391
691c70898518 new files in Integ
paulson
parents:
diff changeset
   392
691c70898518 new files in Integ
paulson
parents:
diff changeset
   393
(* Theorems about less and less_equal *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   394
691c70898518 new files in Integ
paulson
parents:
diff changeset
   395
(*This lemma allows direct proofs of other <-properties*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   396
Goalw [zless_def, znegative_def, zdiff_def, znat_def] 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   397
    "(w < z) = (EX n. z = w + $#(Suc n))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   398
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   399
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   400
by (Clarify_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   401
by (asm_full_simp_tac (simpset() addsimps [zadd, zminus]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   402
by (safe_tac (claset() addSDs [less_eq_Suc_add]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   403
by (res_inst_tac [("x","k")] exI 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   404
by (ALLGOALS (asm_full_simp_tac (simpset() addsimps add_ac)));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   405
qed "zless_iff_Suc_zadd";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   406
691c70898518 new files in Integ
paulson
parents:
diff changeset
   407
Goal "z < z + $# (Suc n)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   408
by (auto_tac (claset(),
691c70898518 new files in Integ
paulson
parents:
diff changeset
   409
	      simpset() addsimps [zless_iff_Suc_zadd, zadd_assoc, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   410
				  add_znat]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   411
qed "zless_zadd_Suc";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   412
691c70898518 new files in Integ
paulson
parents:
diff changeset
   413
Goal "[| z1<z2; z2<z3 |] ==> z1 < (z3::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   414
by (auto_tac (claset(),
691c70898518 new files in Integ
paulson
parents:
diff changeset
   415
	      simpset() addsimps [zless_iff_Suc_zadd, zadd_assoc, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   416
				  add_znat]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   417
qed "zless_trans";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   418
691c70898518 new files in Integ
paulson
parents:
diff changeset
   419
Goal "!!w::int. z<w ==> ~w<z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   420
by (safe_tac (claset() addSDs [zless_iff_Suc_zadd RS iffD1]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   421
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   422
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   423
by (asm_full_simp_tac (simpset() addsimps ([znat_def, zadd])) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   424
qed "zless_not_sym";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   425
691c70898518 new files in Integ
paulson
parents:
diff changeset
   426
(* [| n<m;  ~P ==> m<n |] ==> P *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   427
bind_thm ("zless_asym", (zless_not_sym RS swap));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   428
691c70898518 new files in Integ
paulson
parents:
diff changeset
   429
Goal "!!z::int. ~ z<z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   430
by (resolve_tac [zless_asym RS notI] 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   431
by (REPEAT (assume_tac 1));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   432
qed "zless_not_refl";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   433
691c70898518 new files in Integ
paulson
parents:
diff changeset
   434
(* z<z ==> R *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   435
bind_thm ("zless_irrefl", (zless_not_refl RS notE));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   436
AddSEs [zless_irrefl];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   437
691c70898518 new files in Integ
paulson
parents:
diff changeset
   438
Goal "z<w ==> w ~= (z::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   439
by (Blast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   440
qed "zless_not_refl2";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   441
691c70898518 new files in Integ
paulson
parents:
diff changeset
   442
(* s < t ==> s ~= t *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   443
bind_thm ("zless_not_refl3", zless_not_refl2 RS not_sym);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   444
691c70898518 new files in Integ
paulson
parents:
diff changeset
   445
691c70898518 new files in Integ
paulson
parents:
diff changeset
   446
(*"Less than" is a linear ordering*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   447
Goalw [zless_def, znegative_def, zdiff_def] 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   448
    "z<w | z=w | w<(z::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   449
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   450
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   451
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   452
by (asm_full_simp_tac
691c70898518 new files in Integ
paulson
parents:
diff changeset
   453
    (simpset() addsimps [zadd, zminus, Image_iff, Bex_def]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   454
by (res_inst_tac [("m1", "x+ya"), ("n1", "xa+y")] (less_linear RS disjE) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   455
by (auto_tac (claset(), simpset() addsimps add_ac));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   456
qed "zless_linear";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   457
691c70898518 new files in Integ
paulson
parents:
diff changeset
   458
Goal "!!w::int. (w ~= z) = (w<z | z<w)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   459
by (cut_facts_tac [zless_linear] 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   460
by (Blast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   461
qed "int_neq_iff";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   462
691c70898518 new files in Integ
paulson
parents:
diff changeset
   463
(*** eliminates ~= in premises ***)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   464
bind_thm("int_neqE", int_neq_iff RS iffD1 RS disjE);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   465
691c70898518 new files in Integ
paulson
parents:
diff changeset
   466
Goal "($# m = $# n) = (m = n)"; 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   467
by (fast_tac (claset() addSEs [inj_znat RS injD]) 1); 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   468
qed "znat_znat_eq"; 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   469
AddIffs [znat_znat_eq]; 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   470
691c70898518 new files in Integ
paulson
parents:
diff changeset
   471
Goal "($#m < $#n) = (m<n)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   472
by (simp_tac (simpset() addsimps [less_iff_Suc_add, zless_iff_Suc_zadd, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   473
				  add_znat]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   474
qed "zless_eq_less";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   475
Addsimps [zless_eq_less];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   476
691c70898518 new files in Integ
paulson
parents:
diff changeset
   477
691c70898518 new files in Integ
paulson
parents:
diff changeset
   478
(*** Properties of <= ***)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   479
691c70898518 new files in Integ
paulson
parents:
diff changeset
   480
Goalw [zle_def, le_def] "($#m <= $#n) = (m<=n)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   481
by (Simp_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   482
qed "zle_eq_le";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   483
Addsimps [zle_eq_le];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   484
691c70898518 new files in Integ
paulson
parents:
diff changeset
   485
Goalw [zle_def] "~(w<z) ==> z<=(w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   486
by (assume_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   487
qed "zleI";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   488
691c70898518 new files in Integ
paulson
parents:
diff changeset
   489
Goalw [zle_def] "z<=w ==> ~(w<(z::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   490
by (assume_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   491
qed "zleD";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   492
691c70898518 new files in Integ
paulson
parents:
diff changeset
   493
(*  [| z <= w;  ~ P ==> w < z |] ==> P  *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   494
bind_thm ("zleE", zleD RS swap);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   495
691c70898518 new files in Integ
paulson
parents:
diff changeset
   496
Goalw [zle_def] "(~w<=z) = (z<(w::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   497
by (Simp_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   498
qed "not_zle_iff_zless";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   499
691c70898518 new files in Integ
paulson
parents:
diff changeset
   500
Goalw [zle_def] "~ z <= w ==> w<(z::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   501
by (Fast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   502
qed "not_zleE";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   503
691c70898518 new files in Integ
paulson
parents:
diff changeset
   504
Goalw [zle_def] "z <= w ==> z < w | z=(w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   505
by (cut_facts_tac [zless_linear] 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   506
by (blast_tac (claset() addEs [zless_asym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   507
qed "zle_imp_zless_or_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   508
691c70898518 new files in Integ
paulson
parents:
diff changeset
   509
Goalw [zle_def] "z<w | z=w ==> z <= (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   510
by (cut_facts_tac [zless_linear] 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   511
by (blast_tac (claset() addEs [zless_asym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   512
qed "zless_or_eq_imp_zle";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   513
691c70898518 new files in Integ
paulson
parents:
diff changeset
   514
Goal "(x <= (y::int)) = (x < y | x=y)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   515
by (REPEAT(ares_tac [iffI, zless_or_eq_imp_zle, zle_imp_zless_or_eq] 1));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   516
qed "zle_eq_zless_or_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   517
691c70898518 new files in Integ
paulson
parents:
diff changeset
   518
Goal "w <= (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   519
by (simp_tac (simpset() addsimps [zle_eq_zless_or_eq]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   520
qed "zle_refl";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   521
691c70898518 new files in Integ
paulson
parents:
diff changeset
   522
Goalw [zle_def] "z < w ==> z <= (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   523
by (blast_tac (claset() addEs [zless_asym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   524
qed "zless_imp_zle";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   525
691c70898518 new files in Integ
paulson
parents:
diff changeset
   526
Addsimps [zle_refl, zless_imp_zle];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   527
691c70898518 new files in Integ
paulson
parents:
diff changeset
   528
(* Axiom 'linorder_linear' of class 'linorder': *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   529
Goal "(z::int) <= w | w <= z";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   530
by (simp_tac (simpset() addsimps [zle_eq_zless_or_eq]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   531
by (cut_facts_tac [zless_linear] 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   532
by (Blast_tac 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   533
qed "zle_linear";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   534
691c70898518 new files in Integ
paulson
parents:
diff changeset
   535
Goal "[| i <= j; j < k |] ==> i < (k::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   536
by (dtac zle_imp_zless_or_eq 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   537
by (blast_tac (claset() addIs [zless_trans]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   538
qed "zle_zless_trans";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   539
691c70898518 new files in Integ
paulson
parents:
diff changeset
   540
Goal "[| i < j; j <= k |] ==> i < (k::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   541
by (dtac zle_imp_zless_or_eq 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   542
by (blast_tac (claset() addIs [zless_trans]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   543
qed "zless_zle_trans";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   544
691c70898518 new files in Integ
paulson
parents:
diff changeset
   545
Goal "[| i <= j; j <= k |] ==> i <= (k::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   546
by (EVERY1 [dtac zle_imp_zless_or_eq, dtac zle_imp_zless_or_eq,
691c70898518 new files in Integ
paulson
parents:
diff changeset
   547
            rtac zless_or_eq_imp_zle, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   548
	    blast_tac (claset() addIs [zless_trans])]);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   549
qed "zle_trans";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   550
691c70898518 new files in Integ
paulson
parents:
diff changeset
   551
Goal "[| z <= w; w <= z |] ==> z = (w::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   552
by (EVERY1 [dtac zle_imp_zless_or_eq, dtac zle_imp_zless_or_eq,
691c70898518 new files in Integ
paulson
parents:
diff changeset
   553
            blast_tac (claset() addEs [zless_asym])]);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   554
qed "zle_anti_sym";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   555
691c70898518 new files in Integ
paulson
parents:
diff changeset
   556
(* Axiom 'order_less_le' of class 'order': *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   557
Goal "(w::int) < z = (w <= z & w ~= z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   558
by (simp_tac (simpset() addsimps [zle_def, int_neq_iff]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   559
by (blast_tac (claset() addSEs [zless_asym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   560
qed "int_less_le";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   561
691c70898518 new files in Integ
paulson
parents:
diff changeset
   562
(* [| w <= z; w ~= z |] ==> w < z *)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   563
bind_thm ("zle_neq_implies_zless", [int_less_le, conjI] MRS iffD2);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   564
691c70898518 new files in Integ
paulson
parents:
diff changeset
   565
691c70898518 new files in Integ
paulson
parents:
diff changeset
   566
691c70898518 new files in Integ
paulson
parents:
diff changeset
   567
(*** Subtraction laws ***)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   568
691c70898518 new files in Integ
paulson
parents:
diff changeset
   569
Goal "x + (y - z) = (x + y) - (z::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   570
by (simp_tac (simpset() addsimps (zdiff_def::zadd_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   571
qed "zadd_zdiff_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   572
691c70898518 new files in Integ
paulson
parents:
diff changeset
   573
Goal "(x - y) + z = (x + z) - (y::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   574
by (simp_tac (simpset() addsimps (zdiff_def::zadd_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   575
qed "zdiff_zadd_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   576
691c70898518 new files in Integ
paulson
parents:
diff changeset
   577
Goal "(x - y) - z = x - (y + (z::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   578
by (simp_tac (simpset() addsimps (zdiff_def::zadd_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   579
qed "zdiff_zdiff_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   580
691c70898518 new files in Integ
paulson
parents:
diff changeset
   581
Goal "x - (y - z) = (x + z) - (y::int)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   582
by (simp_tac (simpset() addsimps (zdiff_def::zadd_ac)) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   583
qed "zdiff_zdiff_eq2";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   584
691c70898518 new files in Integ
paulson
parents:
diff changeset
   585
Goalw [zless_def, zdiff_def] "(x-y < z) = (x < z + (y::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   586
by (simp_tac (simpset() addsimps zadd_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   587
qed "zdiff_zless_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   588
691c70898518 new files in Integ
paulson
parents:
diff changeset
   589
Goalw [zless_def, zdiff_def] "(x < z-y) = (x + (y::int) < z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   590
by (simp_tac (simpset() addsimps zadd_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   591
qed "zless_zdiff_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   592
691c70898518 new files in Integ
paulson
parents:
diff changeset
   593
Goalw [zle_def] "(x-y <= z) = (x <= z + (y::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   594
by (simp_tac (simpset() addsimps [zless_zdiff_eq]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   595
qed "zdiff_zle_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   596
691c70898518 new files in Integ
paulson
parents:
diff changeset
   597
Goalw [zle_def] "(x <= z-y) = (x + (y::int) <= z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   598
by (simp_tac (simpset() addsimps [zdiff_zless_eq]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   599
qed "zle_zdiff_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   600
691c70898518 new files in Integ
paulson
parents:
diff changeset
   601
Goalw [zdiff_def] "(x-y = z) = (x = z + (y::int))";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   602
by (auto_tac (claset(), simpset() addsimps [zadd_assoc]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   603
qed "zdiff_eq_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   604
691c70898518 new files in Integ
paulson
parents:
diff changeset
   605
Goalw [zdiff_def] "(x = z-y) = (x + (y::int) = z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   606
by (auto_tac (claset(), simpset() addsimps [zadd_assoc]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   607
qed "eq_zdiff_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   608
691c70898518 new files in Integ
paulson
parents:
diff changeset
   609
(*This list of rewrites simplifies (in)equalities by bringing subtractions
691c70898518 new files in Integ
paulson
parents:
diff changeset
   610
  to the top and then moving negative terms to the other side.  
691c70898518 new files in Integ
paulson
parents:
diff changeset
   611
  Use with zadd_ac*)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   612
val zcompare_rls = 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   613
    [symmetric zdiff_def,
691c70898518 new files in Integ
paulson
parents:
diff changeset
   614
     zadd_zdiff_eq, zdiff_zadd_eq, zdiff_zdiff_eq, zdiff_zdiff_eq2, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   615
     zdiff_zless_eq, zless_zdiff_eq, zdiff_zle_eq, zle_zdiff_eq, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   616
     zdiff_eq_eq, eq_zdiff_eq];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   617
691c70898518 new files in Integ
paulson
parents:
diff changeset
   618
691c70898518 new files in Integ
paulson
parents:
diff changeset
   619
(** Cancellation laws **)
691c70898518 new files in Integ
paulson
parents:
diff changeset
   620
691c70898518 new files in Integ
paulson
parents:
diff changeset
   621
Goal "!!w::int. (z + w' = z + w) = (w' = w)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   622
by Safe_tac;
691c70898518 new files in Integ
paulson
parents:
diff changeset
   623
by (dres_inst_tac [("f", "%x. x + -z")] arg_cong 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   624
by (asm_full_simp_tac (simpset() addsimps zadd_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   625
qed "zadd_left_cancel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   626
691c70898518 new files in Integ
paulson
parents:
diff changeset
   627
Addsimps [zadd_left_cancel];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   628
691c70898518 new files in Integ
paulson
parents:
diff changeset
   629
Goal "!!z::int. (w' + z = w + z) = (w' = w)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   630
by (asm_full_simp_tac (simpset() addsimps zadd_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   631
qed "zadd_right_cancel";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   632
691c70898518 new files in Integ
paulson
parents:
diff changeset
   633
Addsimps [zadd_right_cancel];
691c70898518 new files in Integ
paulson
parents:
diff changeset
   634
691c70898518 new files in Integ
paulson
parents:
diff changeset
   635
691c70898518 new files in Integ
paulson
parents:
diff changeset
   636
Goal "(w < z + $# 1) = (w<z | w=z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   637
by (auto_tac (claset(),
691c70898518 new files in Integ
paulson
parents:
diff changeset
   638
	      simpset() addsimps [zless_iff_Suc_zadd, zadd_assoc, 
691c70898518 new files in Integ
paulson
parents:
diff changeset
   639
				  add_znat]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   640
by (cut_inst_tac [("m","n")] znat_Suc 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   641
by (exhaust_tac "n" 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   642
auto();
691c70898518 new files in Integ
paulson
parents:
diff changeset
   643
by (full_simp_tac (simpset() addsimps zadd_ac) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   644
by (asm_full_simp_tac (simpset() addsimps [zadd_assoc RS sym]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   645
qed "zless_add_nat1_eq";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   646
691c70898518 new files in Integ
paulson
parents:
diff changeset
   647
691c70898518 new files in Integ
paulson
parents:
diff changeset
   648
Goal "(w + $# 1 <= z) = (w<z)";
691c70898518 new files in Integ
paulson
parents:
diff changeset
   649
by (simp_tac (simpset() addsimps [zle_def, zless_add_nat1_eq]) 1);
691c70898518 new files in Integ
paulson
parents:
diff changeset
   650
by (auto_tac (claset() addIs [zle_anti_sym] addEs [zless_asym],
691c70898518 new files in Integ
paulson
parents:
diff changeset
   651
	      simpset() addsimps [symmetric zle_def]));
691c70898518 new files in Integ
paulson
parents:
diff changeset
   652
qed "add_nat1_zle_eq";