src/HOL/Integ/Integ.ML
author paulson
Tue, 03 Mar 1998 15:15:04 +0100
changeset 4676 335dfafb1816
parent 4477 b3e5857d8d99
child 4772 8c7e7eaffbdf
permissions -rw-r--r--
Better simplification allows deletion of parts of proofs
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
     1
(*  Title:      Integ.ML
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     2
    ID:         $Id$
2215
ebf910e7ec87 Tidied up some proofs, ...
paulson
parents: 2083
diff changeset
     3
    Authors:    Lawrence C Paulson, Cambridge University Computer Laboratory
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     5
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     6
The integers as equivalence classes over nat*nat.
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     7
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     8
Could also prove...
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     9
"znegative(z) ==> $# zmagnitude(z) = $~ z"
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    10
"~ znegative(z) ==> $# zmagnitude(z) = z"
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    11
< is a linear ordering
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    12
+ and * are monotonic wrt <
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    13
*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    14
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    15
open Integ;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    16
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    17
Delrules [equalityI];
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    18
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    19
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    20
(*** Proving that intrel is an equivalence relation ***)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    21
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    22
val eqa::eqb::prems = goal Arith.thy 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    23
    "[| (x1::nat) + y2 = x2 + y1; x2 + y3 = x3 + y2 |] ==> \
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    24
\       x1 + y3 = x3 + y1";
4473
803d1e302af1 Decremented subscript because of change to iffD1
paulson
parents: 4369
diff changeset
    25
by (res_inst_tac [("k1","x2")] (add_left_cancel RS iffD1) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    26
by (rtac (add_left_commute RS trans) 1);
2036
62ff902eeffc Ran expandshort; used stac instead of ssubst
paulson
parents: 1894
diff changeset
    27
by (stac eqb 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    28
by (rtac (add_left_commute RS trans) 1);
2036
62ff902eeffc Ran expandshort; used stac instead of ssubst
paulson
parents: 1894
diff changeset
    29
by (stac eqa 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    30
by (rtac (add_left_commute) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    31
qed "integ_trans_lemma";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    32
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    33
(** Natural deduction for intrel **)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    34
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    35
val prems = goalw Integ.thy [intrel_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    36
    "[| x1+y2 = x2+y1|] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    37
\    ((x1,y1),(x2,y2)): intrel";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
    38
by (fast_tac (claset() addIs prems) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    39
qed "intrelI";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    40
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    41
(*intrelE is hard to derive because fast_tac tries hyp_subst_tac so soon*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    42
goalw Integ.thy [intrel_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    43
  "p: intrel --> (EX x1 y1 x2 y2. \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    44
\                  p = ((x1,y1),(x2,y2)) & x1+y2 = x2+y1)";
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    45
by (Fast_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    46
qed "intrelE_lemma";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    47
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    48
val [major,minor] = goal Integ.thy
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    49
  "[| p: intrel;  \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    50
\     !!x1 y1 x2 y2. [| p = ((x1,y1),(x2,y2));  x1+y2 = x2+y1|] ==> Q |] \
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    51
\  ==> Q";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    52
by (cut_facts_tac [major RS (intrelE_lemma RS mp)] 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    53
by (REPEAT (eresolve_tac [asm_rl,exE,conjE,minor] 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    54
qed "intrelE";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    55
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    56
AddSIs [intrelI];
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    57
AddSEs [intrelE];
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    58
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    59
goal Integ.thy "((x1,y1),(x2,y2)): intrel = (x1+y2 = x2+y1)";
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    60
by (Fast_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    61
qed "intrel_iff";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    62
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    63
goal Integ.thy "(x,x): intrel";
2036
62ff902eeffc Ran expandshort; used stac instead of ssubst
paulson
parents: 1894
diff changeset
    64
by (stac surjective_pairing 1 THEN rtac (refl RS intrelI) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    65
qed "intrel_refl";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    66
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    67
goalw Integ.thy [equiv_def, refl_def, sym_def, trans_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    68
    "equiv {x::(nat*nat).True} intrel";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
    69
by (fast_tac (claset() addSIs [intrel_refl] 
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    70
                        addSEs [sym, integ_trans_lemma]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    71
qed "equiv_intrel";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    72
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    73
val equiv_intrel_iff =
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    74
    [TrueI, TrueI] MRS 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    75
    ([CollectI, CollectI] MRS 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    76
    (equiv_intrel RS eq_equiv_class_iff));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    77
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    78
goalw Integ.thy  [Integ_def,intrel_def,quotient_def] "intrel^^{(x,y)}:Integ";
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
    79
by (Fast_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    80
qed "intrel_in_integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    81
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    82
goal Integ.thy "inj_onto Abs_Integ Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    83
by (rtac inj_onto_inverseI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    84
by (etac Abs_Integ_inverse 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    85
qed "inj_onto_Abs_Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    86
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
    87
Addsimps [equiv_intrel_iff, inj_onto_Abs_Integ RS inj_onto_iff,
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
    88
          intrel_iff, intrel_in_integ, Abs_Integ_inverse];
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    89
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    90
goal Integ.thy "inj(Rep_Integ)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    91
by (rtac inj_inverseI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    92
by (rtac Rep_Integ_inverse 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    93
qed "inj_Rep_Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    94
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    95
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    96
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    97
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    98
(** znat: the injection from nat to Integ **)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    99
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   100
goal Integ.thy "inj(znat)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   101
by (rtac injI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   102
by (rewtac znat_def);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   103
by (dtac (inj_onto_Abs_Integ RS inj_ontoD) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   104
by (REPEAT (rtac intrel_in_integ 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   105
by (dtac eq_equiv_class 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   106
by (rtac equiv_intrel 1);
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
   107
by (Fast_tac 1);
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   108
by Safe_tac;
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   109
by (Asm_full_simp_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   110
qed "inj_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   111
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   112
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   113
(**** zminus: unary negation on Integ ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   114
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   115
goalw Integ.thy [congruent_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   116
  "congruent intrel (%p. split (%x y. intrel^^{(y,x)}) p)";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   117
by Safe_tac;
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   118
by (asm_simp_tac (simpset() addsimps add_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   119
qed "zminus_congruent";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   120
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   121
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   122
(*Resolve th against the corresponding facts for zminus*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   123
val zminus_ize = RSLIST [equiv_intrel, zminus_congruent];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   124
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   125
goalw Integ.thy [zminus_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   126
      "$~ Abs_Integ(intrel^^{(x,y)}) = Abs_Integ(intrel ^^ {(y,x)})";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   127
by (res_inst_tac [("f","Abs_Integ")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   128
by (simp_tac (simpset() addsimps 
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   129
   [intrel_in_integ RS Abs_Integ_inverse,zminus_ize UN_equiv_class]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   130
qed "zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   131
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   132
(*by lcp*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   133
val [prem] = goal Integ.thy
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   134
    "(!!x y. z = Abs_Integ(intrel^^{(x,y)}) ==> P) ==> P";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   135
by (res_inst_tac [("x1","z")] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   136
    (rewrite_rule [Integ_def] Rep_Integ RS quotientE) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   137
by (dres_inst_tac [("f","Abs_Integ")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   138
by (res_inst_tac [("p","x")] PairE 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   139
by (rtac prem 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   140
by (asm_full_simp_tac (simpset() addsimps [Rep_Integ_inverse]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   141
qed "eq_Abs_Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   142
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   143
goal Integ.thy "$~ ($~ z) = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   144
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   145
by (asm_simp_tac (simpset() addsimps [zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   146
qed "zminus_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   147
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   148
goal Integ.thy "inj(zminus)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   149
by (rtac injI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   150
by (dres_inst_tac [("f","zminus")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   151
by (asm_full_simp_tac (simpset() addsimps [zminus_zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   152
qed "inj_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   153
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   154
goalw Integ.thy [znat_def] "$~ ($#0) = $#0";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   155
by (simp_tac (simpset() addsimps [zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   156
qed "zminus_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   157
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   158
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   159
(**** znegative: the test for negative integers ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   160
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   161
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   162
goalw Integ.thy [znegative_def, znat_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   163
    "~ znegative($# n)";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   164
by (Simp_tac 1);
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   165
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   166
qed "not_znegative_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   167
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   168
goalw Integ.thy [znegative_def, znat_def] "znegative($~ $# Suc(n))";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   169
by (simp_tac (simpset() addsimps [zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   170
qed "znegative_zminus_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   171
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   172
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   173
(**** zmagnitude: magnitide of an integer, as a natural number ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   174
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   175
goal Arith.thy "!!n::nat. n - Suc(n+m)=0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   176
by (nat_ind_tac "n" 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   177
by (ALLGOALS Asm_simp_tac);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   178
qed "diff_Suc_add_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   179
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   180
goal Arith.thy "Suc((n::nat)+m)-n=Suc(m)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   181
by (nat_ind_tac "n" 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   182
by (ALLGOALS Asm_simp_tac);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   183
qed "diff_Suc_add_inverse";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   184
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   185
goalw Integ.thy [congruent_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   186
    "congruent intrel (split (%x y. intrel^^{((y-x) + (x-(y::nat)),0)}))";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   187
by Safe_tac;
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   188
by (Asm_simp_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   189
by (etac rev_mp 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   190
by (res_inst_tac [("m","x1"),("n","y1")] diff_induct 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   191
by (asm_simp_tac (simpset() addsimps [inj_Suc RS inj_eq]) 3);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   192
by (asm_simp_tac (simpset() addsimps [diff_add_inverse,diff_add_0]) 2);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   193
by (Asm_simp_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   194
by (rtac impI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   195
by (etac subst 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   196
by (res_inst_tac [("m1","x")] (add_commute RS ssubst) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   197
by (asm_simp_tac (simpset() addsimps [diff_add_inverse,diff_add_0]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   198
qed "zmagnitude_congruent";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   199
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   200
(*Resolve th against the corresponding facts for zmagnitude*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   201
val zmagnitude_ize = RSLIST [equiv_intrel, zmagnitude_congruent];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   202
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   203
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   204
goalw Integ.thy [zmagnitude_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   205
    "zmagnitude (Abs_Integ(intrel^^{(x,y)})) = \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   206
\    Abs_Integ(intrel^^{((y - x) + (x - y),0)})";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   207
by (res_inst_tac [("f","Abs_Integ")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   208
by (asm_simp_tac (simpset() addsimps [zmagnitude_ize UN_equiv_class]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   209
qed "zmagnitude";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   210
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   211
goalw Integ.thy [znat_def] "zmagnitude($# n) = $#n";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   212
by (asm_simp_tac (simpset() addsimps [zmagnitude]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   213
qed "zmagnitude_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   214
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   215
goalw Integ.thy [znat_def] "zmagnitude($~ $# n) = $#n";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   216
by (asm_simp_tac (simpset() addsimps [zmagnitude, zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   217
qed "zmagnitude_zminus_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   218
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   219
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   220
(**** zadd: addition on Integ ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   221
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   222
(** Congruence property for addition **)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   223
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   224
goalw Integ.thy [congruent2_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   225
    "congruent2 intrel (%p1 p2.                  \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   226
\         split (%x1 y1. split (%x2 y2. intrel^^{(x1+x2, y1+y2)}) p2) p1)";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   227
(*Proof via congruent2_commuteI seems longer*)
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   228
by Safe_tac;
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   229
by (asm_simp_tac (simpset() addsimps [add_assoc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   230
(*The rest should be trivial, but rearranging terms is hard*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   231
by (res_inst_tac [("x1","x1a")] (add_left_commute RS ssubst) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   232
by (asm_simp_tac (simpset() addsimps [add_assoc RS sym]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   233
qed "zadd_congruent2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   234
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   235
(*Resolve th against the corresponding facts for zadd*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   236
val zadd_ize = RSLIST [equiv_intrel, zadd_congruent2];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   237
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   238
goalw Integ.thy [zadd_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   239
  "Abs_Integ(intrel^^{(x1,y1)}) + Abs_Integ(intrel^^{(x2,y2)}) = \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   240
\  Abs_Integ(intrel^^{(x1+x2, y1+y2)})";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   241
by (asm_simp_tac
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   242
    (simpset() addsimps [zadd_ize UN_equiv_class2]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   243
qed "zadd";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   244
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   245
goalw Integ.thy [znat_def] "$#0 + z = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   246
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   247
by (asm_simp_tac (simpset() addsimps [zadd]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   248
qed "zadd_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   249
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   250
goal Integ.thy "$~ (z + w) = $~ z + $~ w";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   251
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   252
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   253
by (asm_simp_tac (simpset() addsimps [zminus,zadd]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   254
qed "zminus_zadd_distrib";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   255
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   256
goal Integ.thy "(z::int) + w = w + z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   257
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   258
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   259
by (asm_simp_tac (simpset() addsimps (add_ac @ [zadd])) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   260
qed "zadd_commute";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   261
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   262
goal Integ.thy "((z1::int) + z2) + z3 = z1 + (z2 + z3)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   263
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   264
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   265
by (res_inst_tac [("z","z3")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   266
by (asm_simp_tac (simpset() addsimps [zadd, add_assoc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   267
qed "zadd_assoc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   268
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   269
(*For AC rewriting*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   270
goal Integ.thy "(x::int)+(y+z)=y+(x+z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   271
by (rtac (zadd_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   272
by (rtac (zadd_assoc RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   273
by (rtac (zadd_commute RS arg_cong) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   274
qed "zadd_left_commute";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   275
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   276
(*Integer addition is an AC operator*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   277
val zadd_ac = [zadd_assoc,zadd_commute,zadd_left_commute];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   278
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   279
goalw Integ.thy [znat_def] "$# (m + n) = ($#m) + ($#n)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   280
by (asm_simp_tac (simpset() addsimps [zadd]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   281
qed "znat_add";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   282
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   283
goalw Integ.thy [znat_def] "z + ($~ z) = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   284
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   285
by (asm_simp_tac (simpset() addsimps [zminus, zadd, add_commute]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   286
qed "zadd_zminus_inverse";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   287
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   288
goal Integ.thy "($~ z) + z = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   289
by (rtac (zadd_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   290
by (rtac zadd_zminus_inverse 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   291
qed "zadd_zminus_inverse2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   292
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   293
goal Integ.thy "z + $#0 = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   294
by (rtac (zadd_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   295
by (rtac zadd_0 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   296
qed "zadd_0_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   297
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   298
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   299
(** Lemmas **)
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   300
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   301
qed_goal "zadd_assoc_cong" Integ.thy
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   302
    "!!z. (z::int) + v = z' + v' ==> z + (v + w) = z' + (v' + w)"
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   303
 (fn _ => [(asm_simp_tac (simpset() addsimps [zadd_assoc RS sym]) 1)]);
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   304
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   305
qed_goal "zadd_assoc_swap" Integ.thy "(z::int) + (v + w) = v + (z + w)"
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   306
 (fn _ => [(REPEAT (ares_tac [zadd_commute RS zadd_assoc_cong] 1))]);
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   307
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   308
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   309
(*Need properties of subtraction?  Or use $- just as an abbreviation!*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   310
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   311
(**** zmult: multiplication on Integ ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   312
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   313
(** Congruence property for multiplication **)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   314
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   315
goal Integ.thy "((k::nat) + l) + (m + n) = (k + m) + (n + l)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   316
by (simp_tac (simpset() addsimps add_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   317
qed "zmult_congruent_lemma";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   318
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   319
goal Integ.thy 
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
   320
    "congruent2 intrel (%p1 p2.                 \
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
   321
\               split (%x1 y1. split (%x2 y2.   \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   322
\                   intrel^^{(x1*x2 + y1*y2, x1*y2 + y1*x2)}) p2) p1)";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   323
by (rtac (equiv_intrel RS congruent2_commuteI) 1);
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   324
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   325
by (rewtac split_def);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   326
by (simp_tac (simpset() addsimps add_ac@mult_ac) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   327
by (asm_simp_tac (simpset() delsimps [equiv_intrel_iff]
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   328
                           addsimps add_ac@mult_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   329
by (rtac (intrelI RS(equiv_intrel RS equiv_class_eq)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   330
by (rtac (zmult_congruent_lemma RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   331
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   332
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   333
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   334
by (asm_simp_tac (simpset() addsimps [add_mult_distrib RS sym]) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   335
by (asm_simp_tac (simpset() addsimps add_ac@mult_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   336
qed "zmult_congruent2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   337
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   338
(*Resolve th against the corresponding facts for zmult*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   339
val zmult_ize = RSLIST [equiv_intrel, zmult_congruent2];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   340
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   341
goalw Integ.thy [zmult_def]
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
   342
   "Abs_Integ((intrel^^{(x1,y1)})) * Abs_Integ((intrel^^{(x2,y2)})) =   \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   343
\   Abs_Integ(intrel ^^ {(x1*x2 + y1*y2, x1*y2 + y1*x2)})";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   344
by (simp_tac (simpset() addsimps [zmult_ize UN_equiv_class2]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   345
qed "zmult";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   346
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   347
goalw Integ.thy [znat_def] "$#0 * z = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   348
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   349
by (asm_simp_tac (simpset() addsimps [zmult]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   350
qed "zmult_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   351
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   352
goalw Integ.thy [znat_def] "$#Suc(0) * z = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   353
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   354
by (asm_simp_tac (simpset() addsimps [zmult]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   355
qed "zmult_1";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   356
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   357
goal Integ.thy "($~ z) * w = $~ (z * w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   358
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   359
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   360
by (asm_simp_tac (simpset() addsimps ([zminus, zmult] @ add_ac)) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   361
qed "zmult_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   362
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   363
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   364
goal Integ.thy "($~ z) * ($~ w) = (z * w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   365
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   366
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   367
by (asm_simp_tac (simpset() addsimps ([zminus, zmult] @ add_ac)) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   368
qed "zmult_zminus_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   369
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   370
goal Integ.thy "(z::int) * w = w * z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   371
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   372
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   373
by (asm_simp_tac (simpset() addsimps ([zmult] @ add_ac @ mult_ac)) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   374
qed "zmult_commute";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   375
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   376
goal Integ.thy "z * $# 0 = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   377
by (rtac ([zmult_commute, zmult_0] MRS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   378
qed "zmult_0_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   379
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   380
goal Integ.thy "z * $#Suc(0) = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   381
by (rtac ([zmult_commute, zmult_1] MRS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   382
qed "zmult_1_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   383
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   384
goal Integ.thy "((z1::int) * z2) * z3 = z1 * (z2 * z3)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   385
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   386
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   387
by (res_inst_tac [("z","z3")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   388
by (asm_simp_tac (simpset() addsimps ([add_mult_distrib2,zmult] @ 
2036
62ff902eeffc Ran expandshort; used stac instead of ssubst
paulson
parents: 1894
diff changeset
   389
                                     add_ac @ mult_ac)) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   390
qed "zmult_assoc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   391
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   392
(*For AC rewriting*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   393
qed_goal "zmult_left_commute" Integ.thy
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   394
    "(z1::int)*(z2*z3) = z2*(z1*z3)"
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   395
 (fn _ => [rtac (zmult_commute RS trans) 1, rtac (zmult_assoc RS trans) 1,
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   396
           rtac (zmult_commute RS arg_cong) 1]);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   397
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   398
(*Integer multiplication is an AC operator*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   399
val zmult_ac = [zmult_assoc, zmult_commute, zmult_left_commute];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   400
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   401
goal Integ.thy "((z1::int) + z2) * w = (z1 * w) + (z2 * w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   402
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   403
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   404
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   405
by (asm_simp_tac 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   406
    (simpset() addsimps ([add_mult_distrib2, zadd, zmult] @ 
2036
62ff902eeffc Ran expandshort; used stac instead of ssubst
paulson
parents: 1894
diff changeset
   407
                        add_ac @ mult_ac)) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   408
qed "zadd_zmult_distrib";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   409
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   410
val zmult_commute'= read_instantiate [("z","w")] zmult_commute;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   411
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   412
goal Integ.thy "w * ($~ z) = $~ (w * z)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   413
by (simp_tac (simpset() addsimps [zmult_commute', zmult_zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   414
qed "zmult_zminus_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   415
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   416
goal Integ.thy "(w::int) * (z1 + z2) = (w * z1) + (w * z2)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   417
by (simp_tac (simpset() addsimps [zmult_commute',zadd_zmult_distrib]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   418
qed "zadd_zmult_distrib2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   419
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   420
val zadd_simps = 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   421
    [zadd_0, zadd_0_right, zadd_zminus_inverse, zadd_zminus_inverse2];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   422
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   423
val zminus_simps = [zminus_zminus, zminus_0, zminus_zadd_distrib];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   424
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   425
val zmult_simps = [zmult_0, zmult_1, zmult_0_right, zmult_1_right, 
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
   426
                   zmult_zminus, zmult_zminus_right];
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   427
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   428
Addsimps (zadd_simps @ zminus_simps @ zmult_simps @ 
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   429
          [zmagnitude_znat, zmagnitude_zminus_znat]);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   430
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   431
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   432
(**** Additional Theorems (by Mattolini; proofs mainly by lcp) ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   433
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   434
(* Some Theorems about zsuc and zpred *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   435
goalw Integ.thy [zsuc_def] "$#(Suc(n)) = zsuc($# n)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   436
by (simp_tac (simpset() addsimps [znat_add RS sym]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   437
qed "znat_Suc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   438
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   439
goalw Integ.thy [zpred_def,zsuc_def,zdiff_def] "$~ zsuc(z) = zpred($~ z)";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   440
by (Simp_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   441
qed "zminus_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   442
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   443
goalw Integ.thy [zpred_def,zsuc_def,zdiff_def] "$~ zpred(z) = zsuc($~ z)";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 972
diff changeset
   444
by (Simp_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   445
qed "zminus_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   446
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   447
goalw Integ.thy [zsuc_def,zpred_def,zdiff_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   448
   "zpred(zsuc(z)) = z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   449
by (simp_tac (simpset() addsimps [zadd_assoc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   450
qed "zpred_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   451
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   452
goalw Integ.thy [zsuc_def,zpred_def,zdiff_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   453
   "zsuc(zpred(z)) = z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   454
by (simp_tac (simpset() addsimps [zadd_assoc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   455
qed "zsuc_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   456
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   457
goal Integ.thy "(zpred(z)=w) = (z=zsuc(w))";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   458
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   459
by (rtac (zsuc_zpred RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   460
by (rtac zpred_zsuc 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   461
qed "zpred_to_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   462
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   463
goal Integ.thy "(zsuc(z)=w)=(z=zpred(w))";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   464
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   465
by (rtac (zpred_zsuc RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   466
by (rtac zsuc_zpred 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   467
qed "zsuc_to_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   468
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   469
goal Integ.thy "($~ z = w) = (z = $~ w)";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   470
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   471
by (rtac (zminus_zminus RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   472
by (rtac zminus_zminus 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   473
qed "zminus_exchange";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   474
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   475
goal Integ.thy"(zsuc(z)=zsuc(w)) = (z=w)";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   476
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   477
by (dres_inst_tac [("f","zpred")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   478
by (asm_full_simp_tac (simpset() addsimps [zpred_zsuc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   479
qed "bijective_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   480
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   481
goal Integ.thy"(zpred(z)=zpred(w)) = (z=w)";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   482
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   483
by (dres_inst_tac [("f","zsuc")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   484
by (asm_full_simp_tac (simpset() addsimps [zsuc_zpred]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   485
qed "bijective_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   486
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   487
(* Additional Theorems about zadd *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   488
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   489
goalw Integ.thy [zsuc_def] "zsuc(z) + w = zsuc(z+w)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   490
by (simp_tac (simpset() addsimps zadd_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   491
qed "zadd_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   492
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   493
goalw Integ.thy [zsuc_def] "w + zsuc(z) = zsuc(w+z)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   494
by (simp_tac (simpset() addsimps zadd_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   495
qed "zadd_zsuc_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   496
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   497
goalw Integ.thy [zpred_def,zdiff_def] "zpred(z) + w = zpred(z+w)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   498
by (simp_tac (simpset() addsimps zadd_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   499
qed "zadd_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   500
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   501
goalw Integ.thy [zpred_def,zdiff_def] "w + zpred(z) = zpred(w+z)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   502
by (simp_tac (simpset() addsimps zadd_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   503
qed "zadd_zpred_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   504
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   505
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   506
(* Additional Theorems about zmult *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   507
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   508
goalw Integ.thy [zsuc_def] "zsuc(w) * z = z + w * z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   509
by (simp_tac (simpset() addsimps [zadd_zmult_distrib, zadd_commute]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   510
qed "zmult_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   511
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   512
goalw Integ.thy [zsuc_def] "z * zsuc(w) = z + w * z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   513
by (simp_tac 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   514
    (simpset() addsimps [zadd_zmult_distrib2, zadd_commute, zmult_commute]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   515
qed "zmult_zsuc_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   516
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   517
goalw Integ.thy [zpred_def, zdiff_def] "zpred(w) * z = w * z - z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   518
by (simp_tac (simpset() addsimps [zadd_zmult_distrib]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   519
qed "zmult_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   520
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   521
goalw Integ.thy [zpred_def, zdiff_def] "z * zpred(w) = w * z - z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   522
by (simp_tac (simpset() addsimps [zadd_zmult_distrib2, zmult_commute]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   523
qed "zmult_zpred_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   524
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   525
(* Further Theorems about zsuc and zpred *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   526
goal Integ.thy "$#Suc(m) ~= $#0";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   527
by (simp_tac (simpset() addsimps [inj_znat RS inj_eq]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   528
qed "znat_Suc_not_znat_Zero";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   529
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   530
bind_thm ("znat_Zero_not_znat_Suc", (znat_Suc_not_znat_Zero RS not_sym));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   531
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   532
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   533
goalw Integ.thy [zsuc_def,znat_def] "w ~= zsuc(w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   534
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   535
by (asm_full_simp_tac (simpset() addsimps [zadd]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   536
qed "n_not_zsuc_n";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   537
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   538
val zsuc_n_not_n = n_not_zsuc_n RS not_sym;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   539
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   540
goal Integ.thy "w ~= zpred(w)";
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   541
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   542
by (dres_inst_tac [("x","w"),("f","zsuc")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   543
by (asm_full_simp_tac (simpset() addsimps [zsuc_zpred,zsuc_n_not_n]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   544
qed "n_not_zpred_n";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   545
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   546
val zpred_n_not_n = n_not_zpred_n RS not_sym;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   547
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   548
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   549
(* Theorems about less and less_equal *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   550
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   551
goalw Integ.thy [zless_def, znegative_def, zdiff_def, znat_def] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   552
    "!!w. w<z ==> ? n. z = w + $#(Suc(n))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   553
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   554
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   555
by Safe_tac;
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   556
by (asm_full_simp_tac (simpset() addsimps [zadd, zminus]) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   557
by (safe_tac (claset() addSDs [less_eq_Suc_add]));
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   558
by (res_inst_tac [("x","k")] exI 1);
4676
335dfafb1816 Better simplification allows deletion of parts of proofs
paulson
parents: 4477
diff changeset
   559
by (asm_full_simp_tac (simpset() addsimps add_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   560
qed "zless_eq_zadd_Suc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   561
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   562
goalw Integ.thy [zless_def, znegative_def, zdiff_def, znat_def] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   563
    "z < z + $#(Suc(n))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   564
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4676
335dfafb1816 Better simplification allows deletion of parts of proofs
paulson
parents: 4477
diff changeset
   565
by (Clarify_tac 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   566
by (simp_tac (simpset() addsimps [zadd, zminus]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   567
qed "zless_zadd_Suc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   568
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   569
goal Integ.thy "!!z1 z2 z3. [| z1<z2; z2<z3 |] ==> z1 < (z3::int)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   570
by (safe_tac (claset() addSDs [zless_eq_zadd_Suc]));
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   571
by (simp_tac 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   572
    (simpset() addsimps [zadd_assoc, zless_zadd_Suc, znat_add RS sym]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   573
qed "zless_trans";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   574
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   575
goalw Integ.thy [zsuc_def] "z<zsuc(z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   576
by (rtac zless_zadd_Suc 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   577
qed "zlessI";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   578
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   579
val zless_zsucI = zlessI RSN (2,zless_trans);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   580
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   581
goal Integ.thy "!!z w::int. z<w ==> ~w<z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   582
by (safe_tac (claset() addSDs [zless_eq_zadd_Suc]));
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   583
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   584
by Safe_tac;
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   585
by (asm_full_simp_tac (simpset() addsimps ([znat_def, zadd])) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   586
qed "zless_not_sym";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   587
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   588
(* [| n<m; m<n |] ==> R *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   589
bind_thm ("zless_asym", (zless_not_sym RS notE));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   590
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   591
goal Integ.thy "!!z::int. ~ z<z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   592
by (resolve_tac [zless_asym RS notI] 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   593
by (REPEAT (assume_tac 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   594
qed "zless_not_refl";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   595
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   596
(* z<z ==> R *)
1619
cb62d89b7adb Now use _irrefl instead of _anti_refl
paulson
parents: 1465
diff changeset
   597
bind_thm ("zless_irrefl", (zless_not_refl RS notE));
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   598
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   599
goal Integ.thy "!!w. z<w ==> w ~= (z::int)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   600
by (fast_tac (claset() addEs [zless_irrefl]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   601
qed "zless_not_refl2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   602
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   603
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   604
(*"Less than" is a linear ordering*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   605
goalw Integ.thy [zless_def, znegative_def, zdiff_def] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   606
    "z<w | z=w | w<(z::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   607
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   608
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
4162
4c2da701b801 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4089
diff changeset
   609
by Safe_tac;
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   610
by (asm_full_simp_tac
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   611
    (simpset() addsimps [zadd, zminus, Image_iff, Bex_def]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   612
by (res_inst_tac [("m1", "x+ya"), ("n1", "xa+y")] (less_linear RS disjE) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   613
by (REPEAT (fast_tac (claset() addss (simpset() addsimps add_ac)) 1));
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   614
qed "zless_linear";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   615
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   616
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   617
(*** Properties of <= ***)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   618
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   619
goalw Integ.thy  [zless_def, znegative_def, zdiff_def, znat_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   620
    "($#m < $#n) = (m<n)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   621
by (simp_tac
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   622
    (simpset() addsimps [zadd, zminus, Image_iff, Bex_def]) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   623
by (fast_tac (claset() addIs [add_commute] addSEs [less_add_eq_less]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   624
qed "zless_eq_less";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   625
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   626
goalw Integ.thy [zle_def, le_def] "($#m <= $#n) = (m<=n)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   627
by (simp_tac (simpset() addsimps [zless_eq_less]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   628
qed "zle_eq_le";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   629
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   630
goalw Integ.thy [zle_def] "!!w. ~(w<z) ==> z<=(w::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   631
by (assume_tac 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   632
qed "zleI";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   633
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   634
goalw Integ.thy [zle_def] "!!w. z<=w ==> ~(w<(z::int))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   635
by (assume_tac 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   636
qed "zleD";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   637
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   638
val zleE = make_elim zleD;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   639
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   640
goalw Integ.thy [zle_def] "!!z. ~ z <= w ==> w<(z::int)";
1894
c2c8279d40f0 Classical tactics now use default claset.
berghofe
parents: 1798
diff changeset
   641
by (Fast_tac 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   642
qed "not_zleE";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   643
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   644
goalw Integ.thy [zle_def] "!!z. z < w ==> z <= (w::int)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   645
by (fast_tac (claset() addEs [zless_asym]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   646
qed "zless_imp_zle";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   647
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   648
goalw Integ.thy [zle_def] "!!z. z <= w ==> z < w | z=(w::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   649
by (cut_facts_tac [zless_linear] 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   650
by (fast_tac (claset() addEs [zless_irrefl,zless_asym]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   651
qed "zle_imp_zless_or_eq";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   652
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   653
goalw Integ.thy [zle_def] "!!z. z<w | z=w ==> z <=(w::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   654
by (cut_facts_tac [zless_linear] 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   655
by (fast_tac (claset() addEs [zless_irrefl,zless_asym]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   656
qed "zless_or_eq_imp_zle";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   657
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   658
goal Integ.thy "(x <= (y::int)) = (x < y | x=y)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   659
by (REPEAT(ares_tac [iffI, zless_or_eq_imp_zle, zle_imp_zless_or_eq] 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   660
qed "zle_eq_zless_or_eq";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   661
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   662
goal Integ.thy "w <= (w::int)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   663
by (simp_tac (simpset() addsimps [zle_eq_zless_or_eq]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   664
qed "zle_refl";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   665
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   666
val prems = goal Integ.thy "!!i. [| i <= j; j < k |] ==> i < (k::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   667
by (dtac zle_imp_zless_or_eq 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   668
by (fast_tac (claset() addIs [zless_trans]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   669
qed "zle_zless_trans";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   670
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   671
goal Integ.thy "!!i. [| i <= j; j <= k |] ==> i <= (k::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   672
by (EVERY1 [dtac zle_imp_zless_or_eq, dtac zle_imp_zless_or_eq,
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   673
            rtac zless_or_eq_imp_zle, fast_tac (claset() addIs [zless_trans])]);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   674
qed "zle_trans";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   675
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   676
goal Integ.thy "!!z. [| z <= w; w <= z |] ==> z = (w::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   677
by (EVERY1 [dtac zle_imp_zless_or_eq, dtac zle_imp_zless_or_eq,
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   678
            fast_tac (claset() addEs [zless_irrefl,zless_asym])]);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   679
qed "zle_anti_sym";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   680
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   681
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   682
goal Integ.thy "!!w w' z::int. z + w' = z + w ==> w' = w";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   683
by (dres_inst_tac [("f", "%x. x + $~z")] arg_cong 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   684
by (asm_full_simp_tac (simpset() addsimps zadd_ac) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   685
qed "zadd_left_cancel";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   686
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   687
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   688
(*** Monotonicity results ***)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   689
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   690
goal Integ.thy "!!v w z::int. v < w ==> v + z < w + z";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   691
by (safe_tac (claset() addSDs [zless_eq_zadd_Suc]));
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   692
by (simp_tac (simpset() addsimps zadd_ac) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   693
by (simp_tac (simpset() addsimps [zadd_assoc RS sym, zless_zadd_Suc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   694
qed "zadd_zless_mono1";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   695
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   696
goal Integ.thy "!!v w z::int. (v+z < w+z) = (v < w)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   697
by (safe_tac (claset() addSEs [zadd_zless_mono1]));
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   698
by (dres_inst_tac [("z", "$~z")] zadd_zless_mono1 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   699
by (asm_full_simp_tac (simpset() addsimps [zadd_assoc]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   700
qed "zadd_left_cancel_zless";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   701
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   702
goal Integ.thy "!!v w z::int. (v+z <= w+z) = (v <= w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   703
by (asm_full_simp_tac
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   704
    (simpset() addsimps [zle_def, zadd_left_cancel_zless]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   705
qed "zadd_left_cancel_zle";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   706
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   707
(*"v<=w ==> v+z <= w+z"*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   708
bind_thm ("zadd_zle_mono1", zadd_left_cancel_zle RS iffD2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   709
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   710
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   711
goal Integ.thy "!!z' z::int. [| w'<=w; z'<=z |] ==> w' + z' <= w + z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   712
by (etac (zadd_zle_mono1 RS zle_trans) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   713
by (simp_tac (simpset() addsimps [zadd_commute]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   714
(*w moves to the end because it is free while z', z are bound*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   715
by (etac zadd_zle_mono1 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   716
qed "zadd_zle_mono";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   717
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   718
goal Integ.thy "!!w z::int. z<=$#0 ==> w+z <= w";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   719
by (dres_inst_tac [("z", "w")] zadd_zle_mono1 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   720
by (asm_full_simp_tac (simpset() addsimps [zadd_commute]) 1);
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   721
qed "zadd_zle_self";
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   722
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   723
4195
7f7bf0bd0f63 ASCII-fied;
wenzelm
parents: 4162
diff changeset
   724
(**** Comparisons: lemmas and proofs by Norbert Voelker ****)
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   725
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   726
(** One auxiliary theorem...**)
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   727
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   728
goal HOL.thy "(x = False) = (~ x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   729
  by (fast_tac HOL_cs 1);
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   730
qed "eq_False_conv";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   731
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   732
(** Additional theorems for Integ.thy **) 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   733
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   734
Addsimps [zless_eq_less, zle_eq_le,
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   735
	  znegative_zminus_znat, not_znegative_znat]; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   736
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   737
goal Integ.thy "!! x. (x::int) = y ==> x <= y"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   738
  by (etac subst 1); by (rtac zle_refl 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   739
qed "zequalD1"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   740
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   741
goal Integ.thy "($~ x < $~ y) = (y < x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   742
  by (rewrite_goals_tac [zless_def,zdiff_def]); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   743
  by (simp_tac (simpset() addsimps zadd_ac ) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   744
qed "zminus_zless_zminus"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   745
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   746
goal Integ.thy "($~ x <= $~ y) = (y <= x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   747
  by (simp_tac (HOL_ss addsimps[zle_def, zminus_zless_zminus]) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   748
qed "zminus_zle_zminus"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   749
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   750
goal Integ.thy "(x < $~ y) = (y < $~ x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   751
  by (rewrite_goals_tac [zless_def,zdiff_def]); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   752
  by (simp_tac (simpset() addsimps zadd_ac ) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   753
qed "zless_zminus"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   754
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   755
goal Integ.thy "($~ x < y) = ($~ y < x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   756
  by (rewrite_goals_tac [zless_def,zdiff_def]); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   757
  by (simp_tac (simpset() addsimps zadd_ac ) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   758
qed "zminus_zless"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   759
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   760
goal Integ.thy "(x <= $~ y) = (y <=  $~ x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   761
  by (simp_tac (HOL_ss addsimps[zle_def, zminus_zless]) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   762
qed "zle_zminus"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   763
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   764
goal Integ.thy "($~ x <= y) = ($~ y <=  x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   765
  by (simp_tac (HOL_ss addsimps[zle_def, zless_zminus]) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   766
qed "zminus_zle"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   767
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   768
goal Integ.thy " $#0 < $# Suc n"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   769
  by (rtac (zero_less_Suc RS (zless_eq_less RS iffD2)) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   770
qed "zero_zless_Suc_pos"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   771
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   772
goal Integ.thy "($# n= $# m) = (n = m)"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   773
  by (fast_tac (HOL_cs addSEs[inj_znat RS injD]) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   774
qed "znat_znat_eq"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   775
AddIffs[znat_znat_eq]; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   776
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   777
goal Integ.thy "$~ $# Suc n < $#0";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   778
  by (stac (zminus_0 RS sym) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   779
  by (rtac (zminus_zless_zminus RS iffD2) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   780
  by (rtac (zero_less_Suc RS (zless_eq_less RS iffD2)) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   781
qed "negative_zless_0"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   782
Addsimps [zero_zless_Suc_pos, negative_zless_0]; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   783
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   784
goal Integ.thy "$~ $#  n <= $#0";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   785
  by (rtac zless_or_eq_imp_zle 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   786
  by (nat_ind_tac "n" 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   787
  by (ALLGOALS Asm_simp_tac); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   788
qed "negative_zle_0"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   789
Addsimps[negative_zle_0]; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   790
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   791
goal Integ.thy "~($#0 <= $~ $# Suc n)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   792
  by (stac zle_zminus 1);
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   793
  by (Simp_tac 1);
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   794
qed "not_zle_0_negative"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   795
Addsimps[not_zle_0_negative]; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   796
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   797
goal Integ.thy "($# n <= $~ $# m) = (n = 0 & m = 0)"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   798
  by (safe_tac HOL_cs); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   799
  by (Simp_tac 3); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   800
  by (dtac (zle_zminus RS iffD1) 2); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   801
  by (ALLGOALS(dtac (negative_zle_0 RSN(2,zle_trans)))); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   802
  by (ALLGOALS Asm_full_simp_tac); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   803
qed "znat_zle_znegative"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   804
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   805
goal Integ.thy "~($# n < $~ $# Suc m)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   806
  by (rtac notI 1); by (forward_tac [zless_imp_zle] 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   807
  by (dtac (znat_zle_znegative RS iffD1) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   808
  by (safe_tac HOL_cs); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   809
  by (dtac (zless_zminus RS iffD1) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   810
  by (Asm_full_simp_tac 1);
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   811
qed "not_znat_zless_negative"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   812
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   813
goal Integ.thy "($~ $# n = $# m) = (n = 0 & m = 0)"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   814
  by (rtac iffI 1);
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   815
  by (rtac  (znat_zle_znegative RS iffD1) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   816
  by (dtac sym 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   817
  by (ALLGOALS Asm_simp_tac); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   818
qed "negative_eq_positive"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   819
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   820
Addsimps [zminus_zless_zminus, zminus_zle_zminus, 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   821
	  negative_eq_positive, not_znat_zless_negative]; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   822
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   823
goalw Integ.thy [zdiff_def,zless_def] "!! x. znegative x = (x < $# 0)";
4477
b3e5857d8d99 New Auto_tac (by Oheimb), and new syntax (without parens), and expandshort
paulson
parents: 4473
diff changeset
   824
  by Auto_tac; 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   825
qed "znegative_less_0"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   826
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   827
goalw Integ.thy [zdiff_def,zless_def] "!! x. (~znegative x) = ($# 0 <= x)";
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   828
  by (stac znegative_less_0 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   829
  by (safe_tac (HOL_cs addSDs[zleD,not_zleE,zleI]) ); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   830
qed "not_znegative_ge_0"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   831
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   832
goal Integ.thy "!! x. znegative x ==> ? n. x = $~ $# Suc n"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   833
  by (dtac (znegative_less_0 RS iffD1 RS zless_eq_zadd_Suc) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   834
  by (etac exE 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   835
  by (rtac exI 1);
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   836
  by (dres_inst_tac [("f","(% z. z + $~ $# Suc n )")] arg_cong 1); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 3725
diff changeset
   837
  by (auto_tac(claset(), simpset() addsimps [zadd_assoc])); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   838
qed "znegativeD"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   839
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   840
goal Integ.thy "!! x. ~znegative x ==> ? n. x = $# n"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   841
  by (dtac (not_znegative_ge_0 RS iffD1) 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   842
  by (dtac zle_imp_zless_or_eq 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   843
  by (etac disjE 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   844
  by (dtac zless_eq_zadd_Suc 1); 
4477
b3e5857d8d99 New Auto_tac (by Oheimb), and new syntax (without parens), and expandshort
paulson
parents: 4473
diff changeset
   845
  by Auto_tac; 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   846
qed "not_znegativeD"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   847
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   848
(* a case theorem distinguishing positive and negative int *)  
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   849
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   850
val prems = goal Integ.thy 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   851
    "[|!! n. P ($# n); !! n. P ($~ $# Suc n) |] ==> P z"; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   852
  by (cut_inst_tac [("P","znegative z")] excluded_middle 1); 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   853
  by (fast_tac (HOL_cs addSDs[znegativeD,not_znegativeD] addSIs prems) 1); 
3725
c7fa890d0d92 result() -> qed
paulson
parents: 2683
diff changeset
   854
qed "int_cases"; 
2224
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   855
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   856
fun int_case_tac x = res_inst_tac [("z",x)] int_cases; 
4fc4b465be5b New material from Norbert Voelker for efficient binary comparisons
paulson
parents: 2215
diff changeset
   857