src/HOL/Integ/Integ.ML
author clasohm
Fri, 24 Mar 1995 12:30:35 +0100
changeset 972 e61b058d58d2
parent 925 15539deb6863
child 1266 3ae9fe3c0f68
permissions -rw-r--r--
changed syntax of tuples from <..., ...> to (..., ...)
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     1
(*  Title: 	Integ.ML
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     2
    ID:         $Id$
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     3
    Authors: 	Riccardo Mattolini, Dip. Sistemi e Informatica
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     4
        	Lawrence C Paulson, Cambridge University Computer Laboratory
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     5
    Copyright   1994 Universita' di Firenze
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     6
    Copyright   1993  University of Cambridge
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
The integers as equivalence classes over nat*nat.
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
     9
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    10
Could also prove...
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    11
"znegative(z) ==> $# zmagnitude(z) = $~ z"
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    12
"~ znegative(z) ==> $# zmagnitude(z) = z"
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    13
< is a linear ordering
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    14
+ and * are monotonic wrt <
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    15
*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    16
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    17
open Integ;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    18
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";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    25
by (res_inst_tac [("k2","x2")] (add_left_cancel RS iffD1) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    26
by (rtac (add_left_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    27
by (rtac (eqb RS ssubst) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    28
by (rtac (add_left_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    29
by (rtac (eqa RS ssubst) 1);
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";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    38
by (fast_tac (rel_cs addIs prems) 1);
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)";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    45
by (fast_tac rel_cs 1);
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
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    56
val intrel_cs = rel_cs addSIs [intrelI] addSEs [intrelE];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    57
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    58
goal Integ.thy "((x1,y1),(x2,y2)): intrel = (x1+y2 = x2+y1)";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    59
by (fast_tac intrel_cs 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    60
qed "intrel_iff";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    61
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    62
goal Integ.thy "(x,x): intrel";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    63
by (rtac (surjective_pairing RS ssubst) 1 THEN rtac (refl RS intrelI) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    64
qed "intrel_refl";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    65
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    66
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
    67
    "equiv {x::(nat*nat).True} intrel";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    68
by (fast_tac (intrel_cs addSIs [intrel_refl] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    69
                        addSEs [sym, integ_trans_lemma]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    70
qed "equiv_intrel";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    71
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    72
val equiv_intrel_iff =
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    73
    [TrueI, TrueI] MRS 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    74
    ([CollectI, CollectI] MRS 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    75
    (equiv_intrel RS eq_equiv_class_iff));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    76
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
    77
goalw Integ.thy  [Integ_def,intrel_def,quotient_def] "intrel^^{(x,y)}:Integ";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    78
by (fast_tac set_cs 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    79
qed "intrel_in_integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    80
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    81
goal Integ.thy "inj_onto Abs_Integ Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    82
by (rtac inj_onto_inverseI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    83
by (etac Abs_Integ_inverse 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    84
qed "inj_onto_Abs_Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    85
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    86
val intrel_ss = 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    87
    arith_ss addsimps [equiv_intrel_iff, inj_onto_Abs_Integ RS inj_onto_iff,
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
    88
		       intrel_iff, intrel_in_integ, Abs_Integ_inverse];
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);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   107
by (fast_tac set_cs 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   108
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   109
by (asm_full_simp_tac arith_ss 1);
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)";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   117
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   118
by (asm_simp_tac (intrel_ss addsimps add_ac) 1);
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);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   128
by (simp_tac (set_ss addsimps 
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
by (rewtac split_def);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   131
by (simp_tac prod_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   132
qed "zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   133
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   134
(*by lcp*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   135
val [prem] = goal Integ.thy
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   136
    "(!!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
   137
by (res_inst_tac [("x1","z")] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   138
    (rewrite_rule [Integ_def] Rep_Integ RS quotientE) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   139
by (dres_inst_tac [("f","Abs_Integ")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   140
by (res_inst_tac [("p","x")] PairE 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   141
by (rtac prem 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   142
by (asm_full_simp_tac (HOL_ss addsimps [Rep_Integ_inverse]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   143
qed "eq_Abs_Integ";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   144
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   145
goal Integ.thy "$~ ($~ z) = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   146
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   147
by (asm_simp_tac (HOL_ss addsimps [zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   148
qed "zminus_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   149
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   150
goal Integ.thy "inj(zminus)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   151
by (rtac injI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   152
by (dres_inst_tac [("f","zminus")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   153
by (asm_full_simp_tac (HOL_ss addsimps [zminus_zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   154
qed "inj_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   155
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   156
goalw Integ.thy [znat_def] "$~ ($#0) = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   157
by (simp_tac (arith_ss addsimps [zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   158
qed "zminus_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   159
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
(**** znegative: the test for negative integers ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   162
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   163
goal Arith.thy "!!m x n::nat. n+m=x ==> m<=x";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   164
by (dtac (disjI2 RS less_or_eq_imp_le) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   165
by (asm_full_simp_tac (arith_ss addsimps add_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   166
by (dtac add_leD1 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   167
by (assume_tac 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   168
qed "not_znegative_znat_lemma";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   169
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   170
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   171
goalw Integ.thy [znegative_def, znat_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   172
    "~ znegative($# n)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   173
by (simp_tac intrel_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   174
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   175
by (rtac ccontr 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   176
by (etac notE 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   177
by (asm_full_simp_tac arith_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   178
by (dtac not_znegative_znat_lemma 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   179
by (fast_tac (HOL_cs addDs [leD]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   180
qed "not_znegative_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   181
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   182
goalw Integ.thy [znegative_def, znat_def] "znegative($~ $# Suc(n))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   183
by (simp_tac (intrel_ss addsimps [zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   184
by (REPEAT (ares_tac [exI, conjI] 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   185
by (rtac (intrelI RS ImageI) 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   186
by (rtac singletonI 3);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   187
by (simp_tac arith_ss 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   188
by (rtac less_add_Suc1 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   189
qed "znegative_zminus_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   190
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   191
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   192
(**** zmagnitude: magnitide of an integer, as a natural number ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   193
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   194
goal Arith.thy "!!n::nat. n - Suc(n+m)=0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   195
by (nat_ind_tac "n" 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   196
by (ALLGOALS(asm_simp_tac arith_ss));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   197
qed "diff_Suc_add_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   198
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   199
goal Arith.thy "Suc((n::nat)+m)-n=Suc(m)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   200
by (nat_ind_tac "n" 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   201
by (ALLGOALS(asm_simp_tac arith_ss));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   202
qed "diff_Suc_add_inverse";
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 [congruent_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   205
    "congruent intrel (split (%x y. intrel^^{((y-x) + (x-(y::nat)),0)}))";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   206
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   207
by (asm_simp_tac intrel_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   208
by (etac rev_mp 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   209
by (res_inst_tac [("m","x1"),("n","y1")] diff_induct 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   210
by (asm_simp_tac (arith_ss addsimps [inj_Suc RS inj_eq]) 3);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   211
by (asm_simp_tac (arith_ss addsimps [diff_add_inverse,diff_add_0]) 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   212
by (asm_simp_tac arith_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   213
by (rtac impI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   214
by (etac subst 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   215
by (res_inst_tac [("m1","x")] (add_commute RS ssubst) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   216
by (asm_simp_tac (arith_ss addsimps [diff_add_inverse,diff_add_0]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   217
by (rtac impI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   218
by (asm_simp_tac (arith_ss addsimps
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   219
		  [diff_add_inverse, diff_add_0, diff_Suc_add_0,
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   220
		   diff_Suc_add_inverse]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   221
qed "zmagnitude_congruent";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   222
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   223
(*Resolve th against the corresponding facts for zmagnitude*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   224
val zmagnitude_ize = RSLIST [equiv_intrel, zmagnitude_congruent];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   225
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   226
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   227
goalw Integ.thy [zmagnitude_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   228
    "zmagnitude (Abs_Integ(intrel^^{(x,y)})) = \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   229
\    Abs_Integ(intrel^^{((y - x) + (x - y),0)})";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   230
by (res_inst_tac [("f","Abs_Integ")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   231
by (asm_simp_tac (intrel_ss addsimps [zmagnitude_ize UN_equiv_class]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   232
qed "zmagnitude";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   233
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   234
goalw Integ.thy [znat_def] "zmagnitude($# n) = $#n";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   235
by (asm_simp_tac (intrel_ss addsimps [zmagnitude]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   236
qed "zmagnitude_znat";
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 [znat_def] "zmagnitude($~ $# n) = $#n";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   239
by (asm_simp_tac (intrel_ss addsimps [zmagnitude, zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   240
qed "zmagnitude_zminus_znat";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   241
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   242
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   243
(**** zadd: addition on Integ ****)
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
(** Congruence property for addition **)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   246
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   247
goalw Integ.thy [congruent2_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   248
    "congruent2 intrel (%p1 p2.                  \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   249
\         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
   250
(*Proof via congruent2_commuteI seems longer*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   251
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   252
by (asm_simp_tac (intrel_ss addsimps [add_assoc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   253
(*The rest should be trivial, but rearranging terms is hard*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   254
by (res_inst_tac [("x1","x1a")] (add_left_commute RS ssubst) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   255
by (asm_simp_tac (arith_ss addsimps [add_assoc RS sym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   256
by (asm_simp_tac (arith_ss addsimps add_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   257
qed "zadd_congruent2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   258
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   259
(*Resolve th against the corresponding facts for zadd*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   260
val zadd_ize = RSLIST [equiv_intrel, zadd_congruent2];
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
goalw Integ.thy [zadd_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   263
  "Abs_Integ(intrel^^{(x1,y1)}) + Abs_Integ(intrel^^{(x2,y2)}) = \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   264
\  Abs_Integ(intrel^^{(x1+x2, y1+y2)})";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   265
by (asm_simp_tac
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   266
    (intrel_ss addsimps [zadd_ize UN_equiv_class2]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   267
qed "zadd";
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
goalw Integ.thy [znat_def] "$#0 + z = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   270
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   271
by (asm_simp_tac (arith_ss addsimps [zadd]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   272
qed "zadd_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   273
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   274
goal Integ.thy "$~ (z + w) = $~ z + $~ w";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   275
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   276
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   277
by (asm_simp_tac (arith_ss addsimps [zminus,zadd]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   278
qed "zminus_zadd_distrib";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   279
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   280
goal Integ.thy "(z::int) + w = w + z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   281
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   282
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   283
by (asm_simp_tac (intrel_ss addsimps (add_ac @ [zadd])) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   284
qed "zadd_commute";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   285
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   286
goal Integ.thy "((z1::int) + z2) + z3 = z1 + (z2 + z3)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   287
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   288
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   289
by (res_inst_tac [("z","z3")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   290
by (asm_simp_tac (arith_ss addsimps [zadd, add_assoc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   291
qed "zadd_assoc";
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
(*For AC rewriting*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   294
goal Integ.thy "(x::int)+(y+z)=y+(x+z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   295
by (rtac (zadd_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   296
by (rtac (zadd_assoc RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   297
by (rtac (zadd_commute RS arg_cong) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   298
qed "zadd_left_commute";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   299
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   300
(*Integer addition is an AC operator*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   301
val zadd_ac = [zadd_assoc,zadd_commute,zadd_left_commute];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   302
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   303
goalw Integ.thy [znat_def] "$# (m + n) = ($#m) + ($#n)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   304
by (asm_simp_tac (arith_ss addsimps [zadd]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   305
qed "znat_add";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   306
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   307
goalw Integ.thy [znat_def] "z + ($~ z) = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   308
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   309
by (asm_simp_tac (intrel_ss addsimps [zminus, zadd, add_commute]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   310
qed "zadd_zminus_inverse";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   311
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   312
goal Integ.thy "($~ z) + z = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   313
by (rtac (zadd_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   314
by (rtac zadd_zminus_inverse 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   315
qed "zadd_zminus_inverse2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   316
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   317
goal Integ.thy "z + $#0 = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   318
by (rtac (zadd_commute RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   319
by (rtac zadd_0 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   320
qed "zadd_0_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   321
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   322
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   323
(*Need properties of subtraction?  Or use $- just as an abbreviation!*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   324
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   325
(**** zmult: multiplication on Integ ****)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   326
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   327
(** Congruence property for multiplication **)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   328
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   329
goal Integ.thy "((k::nat) + l) + (m + n) = (k + m) + (n + l)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   330
by (simp_tac (arith_ss addsimps add_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   331
qed "zmult_congruent_lemma";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   332
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   333
goal Integ.thy 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   334
    "congruent2 intrel (%p1 p2.  		\
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   335
\               split (%x1 y1. split (%x2 y2. 	\
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   336
\                   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
   337
by (rtac (equiv_intrel RS congruent2_commuteI) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   338
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   339
by (rewtac split_def);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   340
by (simp_tac (arith_ss addsimps add_ac@mult_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   341
by (asm_simp_tac (arith_ss addsimps add_ac@mult_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   342
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
   343
by (rtac (zmult_congruent_lemma RS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   344
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   345
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   346
by (rtac (zmult_congruent_lemma RS trans RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   347
by (asm_simp_tac (HOL_ss addsimps [add_mult_distrib RS sym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   348
by (asm_simp_tac (arith_ss addsimps add_ac@mult_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   349
qed "zmult_congruent2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   350
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   351
(*Resolve th against the corresponding facts for zmult*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   352
val zmult_ize = RSLIST [equiv_intrel, zmult_congruent2];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   353
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   354
goalw Integ.thy [zmult_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   355
   "Abs_Integ((intrel^^{(x1,y1)})) * Abs_Integ((intrel^^{(x2,y2)})) = 	\
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 925
diff changeset
   356
\   Abs_Integ(intrel ^^ {(x1*x2 + y1*y2, x1*y2 + y1*x2)})";
925
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   357
by (simp_tac (intrel_ss addsimps [zmult_ize UN_equiv_class2]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   358
qed "zmult";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   359
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   360
goalw Integ.thy [znat_def] "$#0 * z = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   361
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   362
by (asm_simp_tac (arith_ss addsimps [zmult]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   363
qed "zmult_0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   364
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   365
goalw Integ.thy [znat_def] "$#Suc(0) * z = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   366
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   367
by (asm_simp_tac (arith_ss addsimps [zmult, add_0_right]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   368
qed "zmult_1";
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) * w = $~ (z * w)";
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);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   373
by (asm_simp_tac (intrel_ss addsimps ([zminus, zmult] @ add_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   374
qed "zmult_zminus";
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
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   377
goal Integ.thy "($~ z) * ($~ w) = (z * w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   378
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   379
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   380
by (asm_simp_tac (intrel_ss addsimps ([zminus, zmult] @ add_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   381
qed "zmult_zminus_zminus";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   382
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   383
goal Integ.thy "(z::int) * w = w * z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   384
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   385
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   386
by (asm_simp_tac (intrel_ss addsimps ([zmult] @ add_ac @ mult_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   387
qed "zmult_commute";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   388
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   389
goal Integ.thy "z * $# 0 = $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   390
by (rtac ([zmult_commute, zmult_0] MRS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   391
qed "zmult_0_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   392
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   393
goal Integ.thy "z * $#Suc(0) = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   394
by (rtac ([zmult_commute, zmult_1] MRS trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   395
qed "zmult_1_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   396
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   397
goal Integ.thy "((z1::int) * z2) * z3 = z1 * (z2 * z3)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   398
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   399
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   400
by (res_inst_tac [("z","z3")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   401
by (asm_simp_tac (intrel_ss addsimps ([zmult] @ add_ac @ mult_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   402
qed "zmult_assoc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   403
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   404
(*For AC rewriting*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   405
qed_goal "zmult_left_commute" Integ.thy
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   406
    "(z1::int)*(z2*z3) = z2*(z1*z3)"
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   407
 (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
   408
           rtac (zmult_commute RS arg_cong) 1]);
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
(*Integer multiplication is an AC operator*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   411
val zmult_ac = [zmult_assoc, zmult_commute, zmult_left_commute];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   412
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   413
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
   414
by (res_inst_tac [("z","z1")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   415
by (res_inst_tac [("z","z2")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   416
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   417
by (asm_simp_tac 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   418
    (intrel_ss addsimps ([zadd, zmult, add_mult_distrib] @ 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   419
			 add_ac @ mult_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   420
qed "zadd_zmult_distrib";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   421
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   422
val zmult_commute'= read_instantiate [("z","w")] zmult_commute;
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   423
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   424
goal Integ.thy "w * ($~ z) = $~ (w * z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   425
by (simp_tac (HOL_ss addsimps [zmult_commute', zmult_zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   426
qed "zmult_zminus_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   427
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   428
goal Integ.thy "(w::int) * (z1 + z2) = (w * z1) + (w * z2)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   429
by (simp_tac (HOL_ss addsimps [zmult_commute',zadd_zmult_distrib]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   430
qed "zadd_zmult_distrib2";
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
val zadd_simps = 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   433
    [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
   434
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   435
val zminus_simps = [zminus_zminus, zminus_0, zminus_zadd_distrib];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   436
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   437
val zmult_simps = [zmult_0, zmult_1, zmult_0_right, zmult_1_right, 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   438
		   zmult_zminus, zmult_zminus_right];
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   439
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   440
val integ_ss =
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   441
    arith_ss addsimps (zadd_simps @ zminus_simps @ zmult_simps @ 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   442
		       [zmagnitude_znat, zmagnitude_zminus_znat]);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   443
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   444
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   445
(**** Additional Theorems (by Mattolini; proofs mainly by lcp) ****)
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
(* Some Theorems about zsuc and zpred *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   448
goalw Integ.thy [zsuc_def] "$#(Suc(n)) = zsuc($# n)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   449
by (simp_tac (arith_ss addsimps [znat_add RS sym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   450
qed "znat_Suc";
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 [zpred_def,zsuc_def,zdiff_def] "$~ zsuc(z) = zpred($~ z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   453
by (simp_tac integ_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   454
qed "zminus_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   455
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   456
goalw Integ.thy [zpred_def,zsuc_def,zdiff_def] "$~ zpred(z) = zsuc($~ z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   457
by (simp_tac integ_ss 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   458
qed "zminus_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   459
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   460
goalw Integ.thy [zsuc_def,zpred_def,zdiff_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   461
   "zpred(zsuc(z)) = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   462
by (simp_tac (integ_ss addsimps [zadd_assoc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   463
qed "zpred_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   464
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   465
goalw Integ.thy [zsuc_def,zpred_def,zdiff_def]
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   466
   "zsuc(zpred(z)) = z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   467
by (simp_tac (integ_ss addsimps [zadd_assoc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   468
qed "zsuc_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   469
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   470
goal Integ.thy "(zpred(z)=w) = (z=zsuc(w))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   471
by (safe_tac HOL_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   472
by (rtac (zsuc_zpred RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   473
by (rtac zpred_zsuc 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   474
qed "zpred_to_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   475
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   476
goal Integ.thy "(zsuc(z)=w)=(z=zpred(w))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   477
by (safe_tac HOL_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   478
by (rtac (zpred_zsuc RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   479
by (rtac zsuc_zpred 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   480
qed "zsuc_to_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   481
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   482
goal Integ.thy "($~ z = w) = (z = $~ w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   483
by (safe_tac HOL_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   484
by (rtac (zminus_zminus RS sym) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   485
by (rtac zminus_zminus 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   486
qed "zminus_exchange";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   487
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   488
goal Integ.thy"(zsuc(z)=zsuc(w)) = (z=w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   489
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   490
by (dres_inst_tac [("f","zpred")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   491
by (asm_full_simp_tac (HOL_ss addsimps [zpred_zsuc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   492
qed "bijective_zsuc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   493
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   494
goal Integ.thy"(zpred(z)=zpred(w)) = (z=w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   495
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   496
by (dres_inst_tac [("f","zsuc")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   497
by (asm_full_simp_tac (HOL_ss addsimps [zsuc_zpred]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   498
qed "bijective_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   499
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   500
(* Additional Theorems about zadd *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   501
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   502
goalw Integ.thy [zsuc_def] "zsuc(z) + w = zsuc(z+w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   503
by (simp_tac (arith_ss addsimps zadd_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   504
qed "zadd_zsuc";
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
goalw Integ.thy [zsuc_def] "w + zsuc(z) = zsuc(w+z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   507
by (simp_tac (arith_ss addsimps zadd_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   508
qed "zadd_zsuc_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   509
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   510
goalw Integ.thy [zpred_def,zdiff_def] "zpred(z) + w = zpred(z+w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   511
by (simp_tac (arith_ss addsimps zadd_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   512
qed "zadd_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   513
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   514
goalw Integ.thy [zpred_def,zdiff_def] "w + zpred(z) = zpred(w+z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   515
by (simp_tac (arith_ss addsimps zadd_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   516
qed "zadd_zpred_right";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   517
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   518
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   519
(* Additional Theorems about zmult *)
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 [zsuc_def] "zsuc(w) * z = z + w * z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   522
by (simp_tac (integ_ss addsimps [zadd_zmult_distrib, zadd_commute]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   523
qed "zmult_zsuc";
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
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
   526
by (simp_tac 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   527
    (integ_ss addsimps [zadd_zmult_distrib2, zadd_commute, zmult_commute]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   528
qed "zmult_zsuc_right";
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
goalw Integ.thy [zpred_def, zdiff_def] "zpred(w) * z = w * z - z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   531
by (simp_tac (integ_ss addsimps [zadd_zmult_distrib]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   532
qed "zmult_zpred";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   533
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   534
goalw Integ.thy [zpred_def, zdiff_def] "z * zpred(w) = w * z - z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   535
by (simp_tac (integ_ss addsimps [zadd_zmult_distrib2, zmult_commute]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   536
qed "zmult_zpred_right";
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
(* Further Theorems about zsuc and zpred *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   539
goal Integ.thy "$#Suc(m) ~= $#0";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   540
by (simp_tac (integ_ss addsimps [inj_znat RS inj_eq]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   541
qed "znat_Suc_not_znat_Zero";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   542
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   543
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
   544
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
goalw Integ.thy [zsuc_def,znat_def] "w ~= zsuc(w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   547
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   548
by (asm_full_simp_tac (intrel_ss addsimps [zadd]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   549
qed "n_not_zsuc_n";
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
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
   552
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   553
goal Integ.thy "w ~= zpred(w)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   554
by (safe_tac HOL_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   555
by (dres_inst_tac [("x","w"),("f","zsuc")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   556
by (asm_full_simp_tac (HOL_ss addsimps [zsuc_zpred,zsuc_n_not_n]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   557
qed "n_not_zpred_n";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   558
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   559
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
   560
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
(* Theorems about less and less_equal *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   563
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   564
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
   565
    "!!w. w<z ==> ? n. z = w + $#(Suc(n))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   566
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   567
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   568
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   569
by (asm_full_simp_tac (intrel_ss addsimps [zadd, zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   570
by (safe_tac (intrel_cs addSDs [less_eq_Suc_add]));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   571
by (res_inst_tac [("x","k")] exI 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   572
by (asm_full_simp_tac (HOL_ss addsimps ([add_Suc RS sym] @ add_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   573
(*To cancel x2, rename it to be first!*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   574
by (rename_tac "a b c" 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   575
by (asm_full_simp_tac (HOL_ss addsimps (add_left_cancel::add_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   576
qed "zless_eq_zadd_Suc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   577
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   578
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
   579
    "z < z + $#(Suc(n))";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   580
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   581
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   582
by (simp_tac (intrel_ss addsimps [zadd, zminus]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   583
by (REPEAT_SOME (ares_tac [refl, exI, singletonI, ImageI, conjI, intrelI]));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   584
by (rtac le_less_trans 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   585
by (rtac lessI 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   586
by (asm_simp_tac (arith_ss addsimps ([le_add1,add_left_cancel_le]@add_ac)) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   587
qed "zless_zadd_Suc";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   588
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   589
goal Integ.thy "!!z1 z2 z3. [| z1<z2; z2<z3 |] ==> z1 < (z3::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   590
by (safe_tac (HOL_cs addSDs [zless_eq_zadd_Suc]));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   591
by (simp_tac 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   592
    (arith_ss addsimps [zadd_assoc, zless_zadd_Suc, znat_add RS sym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   593
qed "zless_trans";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   594
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   595
goalw Integ.thy [zsuc_def] "z<zsuc(z)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   596
by (rtac zless_zadd_Suc 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   597
qed "zlessI";
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
val zless_zsucI = zlessI RSN (2,zless_trans);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   600
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   601
goal Integ.thy "!!z w::int. z<w ==> ~w<z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   602
by (safe_tac (HOL_cs addSDs [zless_eq_zadd_Suc]));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   603
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   604
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   605
by (asm_full_simp_tac (intrel_ss addsimps ([znat_def, zadd])) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   606
by (asm_full_simp_tac
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   607
 (HOL_ss addsimps [add_left_cancel, add_assoc, add_Suc_right RS sym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   608
by (resolve_tac [less_not_refl2 RS notE] 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   609
by (etac sym 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   610
by (REPEAT (resolve_tac [lessI, trans_less_add2, less_SucI] 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   611
qed "zless_not_sym";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   612
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   613
(* [| n<m; m<n |] ==> R *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   614
bind_thm ("zless_asym", (zless_not_sym RS notE));
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
goal Integ.thy "!!z::int. ~ z<z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   617
by (resolve_tac [zless_asym RS notI] 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   618
by (REPEAT (assume_tac 1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   619
qed "zless_not_refl";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   620
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   621
(* z<z ==> R *)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   622
bind_thm ("zless_anti_refl", (zless_not_refl RS notE));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   623
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   624
goal Integ.thy "!!w. z<w ==> w ~= (z::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   625
by(fast_tac (HOL_cs addEs [zless_anti_refl]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   626
qed "zless_not_refl2";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   627
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   628
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   629
(*"Less than" is a linear ordering*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   630
goalw Integ.thy [zless_def, znegative_def, zdiff_def] 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   631
    "z<w | z=w | w<(z::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   632
by (res_inst_tac [("z","z")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   633
by (res_inst_tac [("z","w")] eq_Abs_Integ 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   634
by (safe_tac intrel_cs);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   635
by (asm_full_simp_tac
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   636
    (intrel_ss addsimps [zadd, zminus, Image_iff, Bex_def]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   637
by (res_inst_tac [("m1", "x+ya"), ("n1", "xa+y")] (less_linear RS disjE) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   638
by (etac disjE 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   639
by (assume_tac 2);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   640
by (DEPTH_SOLVE
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   641
    (swap_res_tac [exI] 1 THEN 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   642
     swap_res_tac [exI] 1 THEN 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   643
     etac conjI 1 THEN 
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   644
     simp_tac (arith_ss addsimps add_ac)  1));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   645
qed "zless_linear";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   646
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
(*** Properties of <= ***)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   649
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   650
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
   651
    "($#m < $#n) = (m<n)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   652
by (simp_tac
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   653
    (intrel_ss addsimps [zadd, zminus, Image_iff, Bex_def]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   654
by (fast_tac (HOL_cs addIs [add_commute] addSEs [less_add_eq_less]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   655
qed "zless_eq_less";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   656
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   657
goalw Integ.thy [zle_def, le_def] "($#m <= $#n) = (m<=n)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   658
by (simp_tac (HOL_ss addsimps [zless_eq_less]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   659
qed "zle_eq_le";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   660
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   661
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
   662
by (assume_tac 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   663
qed "zleI";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   664
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   665
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
   666
by (assume_tac 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   667
qed "zleD";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   668
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   669
val zleE = make_elim zleD;
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
goalw Integ.thy [zle_def] "!!z. ~ z <= w ==> w<(z::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   672
by (fast_tac HOL_cs 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   673
qed "not_zleE";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   674
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   675
goalw Integ.thy [zle_def] "!!z. z < w ==> z <= (w::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   676
by (fast_tac (HOL_cs addEs [zless_asym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   677
qed "zless_imp_zle";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   678
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   679
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
   680
by (cut_facts_tac [zless_linear] 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   681
by (fast_tac (HOL_cs addEs [zless_anti_refl,zless_asym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   682
qed "zle_imp_zless_or_eq";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   683
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   684
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
   685
by (cut_facts_tac [zless_linear] 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   686
by (fast_tac (HOL_cs addEs [zless_anti_refl,zless_asym]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   687
qed "zless_or_eq_imp_zle";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   688
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   689
goal Integ.thy "(x <= (y::int)) = (x < y | x=y)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   690
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
   691
qed "zle_eq_zless_or_eq";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   692
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   693
goal Integ.thy "w <= (w::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   694
by (simp_tac (HOL_ss addsimps [zle_eq_zless_or_eq]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   695
qed "zle_refl";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   696
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   697
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
   698
by (dtac zle_imp_zless_or_eq 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   699
by (fast_tac (HOL_cs addIs [zless_trans]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   700
qed "zle_zless_trans";
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 "!!i. [| i <= j; j <= k |] ==> i <= (k::int)";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   703
by (EVERY1 [dtac zle_imp_zless_or_eq, dtac zle_imp_zless_or_eq,
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   704
	    rtac zless_or_eq_imp_zle, fast_tac (HOL_cs addIs [zless_trans])]);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   705
qed "zle_trans";
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
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
   708
by (EVERY1 [dtac zle_imp_zless_or_eq, dtac zle_imp_zless_or_eq,
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   709
	    fast_tac (HOL_cs addEs [zless_anti_refl,zless_asym])]);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   710
qed "zle_anti_sym";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   711
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   712
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   713
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
   714
by (dres_inst_tac [("f", "%x. x + $~z")] arg_cong 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   715
by (asm_full_simp_tac (integ_ss addsimps zadd_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   716
qed "zadd_left_cancel";
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
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   719
(*** Monotonicity results ***)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   720
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   721
goal Integ.thy "!!v w z::int. v < w ==> v + z < w + z";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   722
by (safe_tac (HOL_cs addSDs [zless_eq_zadd_Suc]));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   723
by (simp_tac (HOL_ss addsimps zadd_ac) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   724
by (simp_tac (HOL_ss addsimps [zadd_assoc RS sym, zless_zadd_Suc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   725
qed "zadd_zless_mono1";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   726
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   727
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
   728
by (safe_tac (HOL_cs addSEs [zadd_zless_mono1]));
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   729
by (dres_inst_tac [("z", "$~z")] zadd_zless_mono1 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   730
by (asm_full_simp_tac (integ_ss addsimps [zadd_assoc]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   731
qed "zadd_left_cancel_zless";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   732
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   733
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
   734
by (asm_full_simp_tac
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   735
    (integ_ss addsimps [zle_def, zadd_left_cancel_zless]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   736
qed "zadd_left_cancel_zle";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   737
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   738
(*"v<=w ==> v+z <= w+z"*)
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   739
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
   740
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   741
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   742
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
   743
by (etac (zadd_zle_mono1 RS zle_trans) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   744
by (simp_tac (HOL_ss addsimps [zadd_commute]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   745
(*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
   746
by (etac zadd_zle_mono1 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   747
qed "zadd_zle_mono";
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   748
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   749
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
   750
by (dres_inst_tac [("z", "w")] zadd_zle_mono1 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   751
by (asm_full_simp_tac (integ_ss addsimps [zadd_commute]) 1);
15539deb6863 new version of HOL/Integ with curried function application
clasohm
parents:
diff changeset
   752
qed "zadd_zle_self";