src/HOL/Integ/IntDiv.ML
author paulson
Mon, 22 Oct 2001 11:54:22 +0200
changeset 11868 56db9f3a6b3e
parent 11704 3c50a2cd6f00
permissions -rw-r--r--
Numerals now work for the integers: the binary numerals for 0 and 1 rewrite
to their abstract counterparts, while other binary numerals work correctly.
     1 (*  Title:      HOL/IntDiv.ML
     2     ID:         $Id$
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1999  University of Cambridge
     5 
     6 The division operators div, mod and the divides relation "dvd"
     7 
     8 Here is the division algorithm in ML:
     9 
    10     fun posDivAlg (a,b) =
    11       if a<b then (0,a)
    12       else let val (q,r) = posDivAlg(a, 2*b)
    13 	       in  if 0<=r-b then (2*q+1, r-b) else (2*q, r)
    14 	   end;
    15 
    16     fun negDivAlg (a,b) =
    17       if 0<=a+b then (~1,a+b)
    18       else let val (q,r) = negDivAlg(a, 2*b)
    19 	       in  if 0<=r-b then (2*q+1, r-b) else (2*q, r)
    20 	   end;
    21 
    22     fun negateSnd (q,r:int) = (q,~r);
    23 
    24     fun divAlg (a,b) = if 0<=a then 
    25 			  if b>0 then posDivAlg (a,b) 
    26 			   else if a=0 then (0,0)
    27 				else negateSnd (negDivAlg (~a,~b))
    28 		       else 
    29 			  if 0<b then negDivAlg (a,b)
    30 			  else        negateSnd (posDivAlg (~a,~b));
    31 *)
    32 
    33 Addsimps [zless_nat_conj];
    34 
    35 (*** Uniqueness and monotonicity of quotients and remainders ***)
    36 
    37 Goal "[| b*q' + r'  <= b*q + r;  0 <= r';  0 < b;  r < b |] \
    38 \     ==> q' <= (q::int)";
    39 by (subgoal_tac "r' + b * (q'-q) <= r" 1);
    40 by (simp_tac (simpset() addsimps [zdiff_zmult_distrib2]) 2);
    41 by (subgoal_tac "0 < b * (1 + q - q')" 1);
    42 by (etac order_le_less_trans 2);
    43 by (full_simp_tac (simpset() addsimps [zdiff_zmult_distrib2,
    44 				       zadd_zmult_distrib2]) 2);
    45 by (subgoal_tac "b * q' < b * (1 + q)" 1);
    46 by (full_simp_tac (simpset() addsimps [zdiff_zmult_distrib2,
    47 				       zadd_zmult_distrib2]) 2);
    48 by (asm_full_simp_tac (simpset() addsimps [zmult_zless_cancel1]) 1); 
    49 qed "unique_quotient_lemma";
    50 
    51 Goal "[| b*q' + r' <= b*q + r;  r <= 0;  b < 0;  b < r' |] \
    52 \     ==> q <= (q'::int)";
    53 by (res_inst_tac [("b", "-b"), ("r", "-r'"), ("r'", "-r")] 
    54     unique_quotient_lemma 1);
    55 by (auto_tac (claset(), 
    56 	      simpset() addsimps [zmult_zminus, zmult_zminus_right])); 
    57 qed "unique_quotient_lemma_neg";
    58 
    59 
    60 Goal "[| quorem ((a,b), (q,r));  quorem ((a,b), (q',r'));  b ~= 0 |] \
    61 \     ==> q = q'";
    62 by (asm_full_simp_tac 
    63     (simpset() addsimps split_ifs@
    64                         [quorem_def, linorder_neq_iff]) 1);
    65 by Safe_tac; 
    66 by (ALLGOALS Asm_full_simp_tac);
    67 by (REPEAT 
    68     (blast_tac (claset() addIs [order_antisym]
    69 			 addDs [order_eq_refl RS unique_quotient_lemma, 
    70 				order_eq_refl RS unique_quotient_lemma_neg,
    71 				sym]) 1));
    72 qed "unique_quotient";
    73 
    74 
    75 Goal "[| quorem ((a,b), (q,r));  quorem ((a,b), (q',r'));  b ~= 0 |] \
    76 \     ==> r = r'";
    77 by (subgoal_tac "q = q'" 1);
    78 by (blast_tac (claset() addIs [unique_quotient]) 2);
    79 by (asm_full_simp_tac (simpset() addsimps [quorem_def]) 1);
    80 qed "unique_remainder";
    81 
    82 
    83 (*** Correctness of posDivAlg, the division algorithm for a>=0 and b>0 ***)
    84 
    85 
    86 Goal "adjust b (q,r) = (let diff = r-b in \
    87 \                         if 0 <= diff then (2*q + 1, diff)  \
    88 \                                      else (2*q, r))";
    89 by (simp_tac (simpset() addsimps [Let_def,adjust_def]) 1);
    90 qed "adjust_eq";
    91 Addsimps [adjust_eq];
    92 
    93 (*Proving posDivAlg's termination condition*)
    94 val [tc] = posDivAlg.tcs;
    95 goalw_cterm [] (cterm_of (sign_of (the_context ())) (HOLogic.mk_Trueprop tc));
    96 by Auto_tac;
    97 val lemma = result();
    98 
    99 (* removing the termination condition from the generated theorems *)
   100 
   101 bind_thm ("posDivAlg_raw_eqn", lemma RS hd posDivAlg.simps);
   102 
   103 (**use with simproc to avoid re-proving the premise*)
   104 Goal "0 < b ==> \
   105 \     posDivAlg (a,b) =      \
   106 \      (if a<b then (0,a) else adjust b (posDivAlg(a, 2*b)))";
   107 by (rtac (posDivAlg_raw_eqn RS trans) 1);
   108 by (Asm_simp_tac 1);
   109 qed "posDivAlg_eqn";
   110 
   111 bind_thm ("posDivAlg_induct", lemma RS posDivAlg.induct);
   112 
   113 
   114 (*Correctness of posDivAlg: it computes quotients correctly*)
   115 Goal "0 <= a --> 0 < b --> quorem ((a, b), posDivAlg (a, b))";
   116 by (induct_thm_tac posDivAlg_induct "a b" 1);
   117 by Auto_tac;
   118 by (ALLGOALS (asm_full_simp_tac (simpset() addsimps [quorem_def])));
   119 (*base case: a<b*)
   120 by (asm_full_simp_tac (simpset() addsimps [posDivAlg_eqn]) 1);
   121 (*main argument*)
   122 by (stac posDivAlg_eqn 1);
   123 by (ALLGOALS Asm_simp_tac);
   124 by (etac splitE 1);
   125 by (auto_tac (claset(), simpset() addsimps [zadd_zmult_distrib2, Let_def]));
   126 qed_spec_mp "posDivAlg_correct";
   127 
   128 
   129 (*** Correctness of negDivAlg, the division algorithm for a<0 and b>0 ***)
   130 
   131 (*Proving negDivAlg's termination condition*)
   132 val [tc] = negDivAlg.tcs;
   133 goalw_cterm [] (cterm_of (sign_of (the_context ())) (HOLogic.mk_Trueprop tc));
   134 by Auto_tac;
   135 val lemma = result();
   136 
   137 (* removing the termination condition from the generated theorems *)
   138 
   139 bind_thm ("negDivAlg_raw_eqn", lemma RS hd negDivAlg.simps);
   140 
   141 (**use with simproc to avoid re-proving the premise*)
   142 Goal "0 < b ==> \
   143 \     negDivAlg (a,b) =      \
   144 \      (if 0<=a+b then (-1,a+b) else adjust b (negDivAlg(a, 2*b)))";
   145 by (rtac (negDivAlg_raw_eqn RS trans) 1);
   146 by (Asm_simp_tac 1);
   147 qed "negDivAlg_eqn";
   148 
   149 bind_thm ("negDivAlg_induct", lemma RS negDivAlg.induct);
   150 
   151 
   152 (*Correctness of negDivAlg: it computes quotients correctly
   153   It doesn't work if a=0 because the 0/b=0 rather than -1*)
   154 Goal "a < 0 --> 0 < b --> quorem ((a, b), negDivAlg (a, b))";
   155 by (induct_thm_tac negDivAlg_induct "a b" 1);
   156 by Auto_tac;
   157 by (ALLGOALS (asm_full_simp_tac (simpset() addsimps [quorem_def])));
   158 (*base case: 0<=a+b*)
   159 by (asm_full_simp_tac (simpset() addsimps [negDivAlg_eqn]) 1);
   160 (*main argument*)
   161 by (stac negDivAlg_eqn 1);
   162 by (ALLGOALS Asm_simp_tac);
   163 by (etac splitE 1);
   164 by (auto_tac (claset(), simpset() addsimps [zadd_zmult_distrib2, Let_def]));
   165 qed_spec_mp "negDivAlg_correct";
   166 
   167 
   168 (*** Existence shown by proving the division algorithm to be correct ***)
   169 
   170 (*the case a=0*)
   171 Goal "b ~= 0 ==> quorem ((0,b), (0,0))";
   172 by (auto_tac (claset(), 
   173 	      simpset() addsimps [quorem_def, linorder_neq_iff]));
   174 qed "quorem_0";
   175 
   176 Goal "posDivAlg (0, b) = (0, 0)";
   177 by (stac posDivAlg_raw_eqn 1);
   178 by Auto_tac;
   179 qed "posDivAlg_0";
   180 Addsimps [posDivAlg_0];
   181 
   182 Goal "negDivAlg (-1, b) = (-1, b - 1)";
   183 by (stac negDivAlg_raw_eqn 1);
   184 by Auto_tac;
   185 qed "negDivAlg_minus1";
   186 Addsimps [negDivAlg_minus1];
   187 
   188 Goalw [negateSnd_def] "negateSnd(q,r) = (q,-r)";
   189 by Auto_tac;
   190 qed "negateSnd_eq";
   191 Addsimps [negateSnd_eq];
   192 
   193 Goal "quorem ((-a,-b), qr) ==> quorem ((a,b), negateSnd qr)";
   194 by (auto_tac (claset(), simpset() addsimps split_ifs@[quorem_def]));
   195 qed "quorem_neg";
   196 
   197 Goal "b ~= 0 ==> quorem ((a,b), divAlg(a,b))";
   198 by (auto_tac (claset(), 
   199 	      simpset() addsimps [quorem_0, divAlg_def]));
   200 by (REPEAT_FIRST (resolve_tac [quorem_neg, posDivAlg_correct,
   201 			       negDivAlg_correct]));
   202 by (auto_tac (claset(), 
   203 	      simpset() addsimps [quorem_def, linorder_neq_iff]));
   204 qed "divAlg_correct";
   205 
   206 (** Arbitrary definitions for division by zero.  Useful to simplify 
   207     certain equations **)
   208 
   209 Goal "a div (0::int) = 0";
   210 by (simp_tac (simpset() addsimps [div_def, divAlg_def, posDivAlg_raw_eqn]) 1);
   211 qed "DIVISION_BY_ZERO_ZDIV";  (*NOT for adding to default simpset*)
   212 
   213 Goal "a mod (0::int) = a";
   214 by (simp_tac (simpset() addsimps [mod_def, divAlg_def, posDivAlg_raw_eqn]) 1);
   215 qed "DIVISION_BY_ZERO_ZMOD";  (*NOT for adding to default simpset*)
   216 
   217 fun zdiv_undefined_case_tac s i =
   218   case_tac s i THEN 
   219   asm_simp_tac (simpset() addsimps [DIVISION_BY_ZERO_ZDIV, 
   220 				    DIVISION_BY_ZERO_ZMOD]) i;
   221 
   222 (** Basic laws about division and remainder **)
   223 
   224 Goal "(a::int) = b * (a div b) + (a mod b)";
   225 by (zdiv_undefined_case_tac "b = 0" 1);
   226 by (cut_inst_tac [("a","a"),("b","b")] divAlg_correct 1);
   227 by (auto_tac (claset(), 
   228 	      simpset() addsimps [quorem_def, div_def, mod_def]));
   229 qed "zmod_zdiv_equality";  
   230 
   231 Goal "(0::int) < b ==> 0 <= a mod b & a mod b < b";
   232 by (cut_inst_tac [("a","a"),("b","b")] divAlg_correct 1);
   233 by (auto_tac (claset(), 
   234 	      simpset() addsimps [quorem_def, mod_def]));
   235 bind_thm ("pos_mod_sign", result() RS conjunct1);
   236 bind_thm ("pos_mod_bound", result() RS conjunct2);
   237 
   238 Goal "b < (0::int) ==> a mod b <= 0 & b < a mod b";
   239 by (cut_inst_tac [("a","a"),("b","b")] divAlg_correct 1);
   240 by (auto_tac (claset(), 
   241 	      simpset() addsimps [quorem_def, div_def, mod_def]));
   242 bind_thm ("neg_mod_sign", result() RS conjunct1);
   243 bind_thm ("neg_mod_bound", result() RS conjunct2);
   244 
   245 
   246 (** proving general properties of div and mod **)
   247 
   248 Goal "b ~= 0 ==> quorem ((a, b), (a div b, a mod b))";
   249 by (cut_inst_tac [("a","a"),("b","b")] zmod_zdiv_equality 1);
   250 by (auto_tac
   251     (claset(),
   252      simpset() addsimps [quorem_def, linorder_neq_iff, 
   253 			 pos_mod_sign,pos_mod_bound,
   254 			 neg_mod_sign, neg_mod_bound]));
   255 qed "quorem_div_mod";
   256 
   257 Goal "[| quorem((a,b),(q,r));  b ~= 0 |] ==> a div b = q";
   258 by (asm_simp_tac (simpset() addsimps [quorem_div_mod RS unique_quotient]) 1);
   259 qed "quorem_div";
   260 
   261 Goal "[| quorem((a,b),(q,r));  b ~= 0 |] ==> a mod b = r";
   262 by (asm_simp_tac (simpset() addsimps [quorem_div_mod RS unique_remainder]) 1);
   263 qed "quorem_mod";
   264 
   265 Goal "[| (0::int) <= a;  a < b |] ==> a div b = 0";
   266 by (rtac quorem_div 1);
   267 by (auto_tac (claset(), simpset() addsimps [quorem_def]));
   268 qed "div_pos_pos_trivial";
   269 
   270 Goal "[| a <= (0::int);  b < a |] ==> a div b = 0";
   271 by (rtac quorem_div 1);
   272 by (auto_tac (claset(), simpset() addsimps [quorem_def]));
   273 qed "div_neg_neg_trivial";
   274 
   275 Goal "[| (0::int) < a;  a+b <= 0 |] ==> a div b = -1";
   276 by (rtac quorem_div 1);
   277 by (auto_tac (claset(), simpset() addsimps [quorem_def]));
   278 qed "div_pos_neg_trivial";
   279 
   280 (*There is no div_neg_pos_trivial because  0 div b = 0 would supersede it*)
   281 
   282 Goal "[| (0::int) <= a;  a < b |] ==> a mod b = a";
   283 by (res_inst_tac [("q","0")] quorem_mod 1);
   284 by (auto_tac (claset(), simpset() addsimps [quorem_def]));
   285 qed "mod_pos_pos_trivial";
   286 
   287 Goal "[| a <= (0::int);  b < a |] ==> a mod b = a";
   288 by (res_inst_tac [("q","0")] quorem_mod 1);
   289 by (auto_tac (claset(), simpset() addsimps [quorem_def]));
   290 qed "mod_neg_neg_trivial";
   291 
   292 Goal "[| (0::int) < a;  a+b <= 0 |] ==> a mod b = a+b";
   293 by (res_inst_tac [("q","-1")] quorem_mod 1);
   294 by (auto_tac (claset(), simpset() addsimps [quorem_def]));
   295 qed "mod_pos_neg_trivial";
   296 
   297 (*There is no mod_neg_pos_trivial...*)
   298 
   299 
   300 (*Simpler laws such as -a div b = -(a div b) FAIL, but see just below*)
   301 Goal "(-a) div (-b) = a div (b::int)";
   302 by (zdiv_undefined_case_tac "b = 0" 1);
   303 by (stac ((simplify(simpset()) (quorem_div_mod RS quorem_neg)) 
   304 	  RS quorem_div) 1);
   305 by Auto_tac;
   306 qed "zdiv_zminus_zminus";
   307 Addsimps [zdiv_zminus_zminus];
   308 
   309 (*Simpler laws such as -a mod b = -(a mod b) FAIL, but see just below*)
   310 Goal "(-a) mod (-b) = - (a mod (b::int))";
   311 by (zdiv_undefined_case_tac "b = 0" 1);
   312 by (stac ((simplify(simpset()) (quorem_div_mod RS quorem_neg)) 
   313 	  RS quorem_mod) 1);
   314 by Auto_tac;
   315 qed "zmod_zminus_zminus";
   316 Addsimps [zmod_zminus_zminus];
   317 
   318 
   319 (*** div, mod and unary minus ***)
   320 
   321 Goal "quorem((a,b),(q,r)) \
   322 \     ==> quorem ((-a,b), (if r=0 then -q else -q - 1), \
   323 \                         (if r=0 then 0 else b-r))";
   324 by (auto_tac
   325     (claset(),
   326      simpset() addsimps split_ifs@
   327                         [quorem_def, linorder_neq_iff, 
   328 			 zdiff_zmult_distrib2]));
   329 val lemma = result();
   330 
   331 Goal "b ~= (0::int) \
   332 \     ==> (-a) div b = \
   333 \         (if a mod b = 0 then - (a div b) else  - (a div b) - 1)";
   334 by (blast_tac (claset() addIs [quorem_div_mod RS lemma RS quorem_div]) 1);
   335 qed "zdiv_zminus1_eq_if";
   336 
   337 Goal "(-a::int) mod b = (if a mod b = 0 then 0 else  b - (a mod b))";
   338 by (zdiv_undefined_case_tac "b = 0" 1);
   339 by (blast_tac (claset() addIs [quorem_div_mod RS lemma RS quorem_mod]) 1);
   340 qed "zmod_zminus1_eq_if";
   341 
   342 Goal "a div (-b) = (-a::int) div b";
   343 by (cut_inst_tac [("a","-a")] zdiv_zminus_zminus 1);
   344 by Auto_tac;  
   345 qed "zdiv_zminus2";
   346 
   347 Goal "a mod (-b) = - ((-a::int) mod b)";
   348 by (cut_inst_tac [("a","-a"),("b","b")] zmod_zminus_zminus 1);
   349 by Auto_tac;  
   350 qed "zmod_zminus2";
   351 
   352 Goal "b ~= (0::int) \
   353 \     ==> a div (-b) = \
   354 \         (if a mod b = 0 then - (a div b) else  - (a div b) - 1)";
   355 by (asm_simp_tac (simpset() addsimps [zdiv_zminus1_eq_if, zdiv_zminus2]) 1); 
   356 qed "zdiv_zminus2_eq_if";
   357 
   358 Goal "a mod (-b::int) = (if a mod b = 0 then 0 else  (a mod b) - b)";
   359 by (asm_simp_tac (simpset() addsimps [zmod_zminus1_eq_if, zmod_zminus2]) 1); 
   360 qed "zmod_zminus2_eq_if";
   361 
   362 
   363 (*** division of a number by itself ***)
   364 
   365 Goal "[| (0::int) < a; a = r + a*q; r < a |] ==> 1 <= q";
   366 by (subgoal_tac "0 < a*q" 1);
   367 by (arith_tac 2);
   368 by (asm_full_simp_tac (simpset() addsimps [int_0_less_mult_iff]) 1);
   369 val lemma1 = result();
   370 
   371 Goal "[| (0::int) < a; a = r + a*q; 0 <= r |] ==> q <= 1";
   372 by (subgoal_tac "0 <= a*(1-q)" 1);
   373 by (asm_simp_tac (simpset() addsimps [zdiff_zmult_distrib2]) 2);
   374 by (asm_full_simp_tac (simpset() addsimps [int_0_le_mult_iff]) 1);
   375 val lemma2 = result();
   376 
   377 Goal "[| quorem((a,a),(q,r));  a ~= (0::int) |] ==> q = 1";
   378 by (asm_full_simp_tac 
   379     (simpset() addsimps split_ifs@[quorem_def, linorder_neq_iff]) 1);
   380 by (rtac order_antisym 1);
   381 by Safe_tac;
   382 by Auto_tac;
   383 by (res_inst_tac [("a", "-a"),("r", "-r")] lemma1 3);
   384 by (res_inst_tac [("a", "-a"),("r", "-r")] lemma2 1);
   385 by (REPEAT (force_tac  (claset() addIs [lemma1,lemma2], 
   386 	      simpset() addsimps [zadd_commute, zmult_zminus]) 1));
   387 qed "self_quotient";
   388 
   389 Goal "[| quorem((a,a),(q,r));  a ~= (0::int) |] ==> r = 0";
   390 by (ftac self_quotient 1);
   391 by (assume_tac 1);
   392 by (asm_full_simp_tac (simpset() addsimps [quorem_def]) 1);
   393 qed "self_remainder";
   394 
   395 Goal "a ~= 0 ==> a div a = (1::int)";
   396 by (asm_simp_tac (simpset() addsimps [quorem_div_mod RS self_quotient]) 1);
   397 qed "zdiv_self";
   398 Addsimps [zdiv_self];
   399 
   400 (*Here we have 0 mod 0 = 0, also assumed by Knuth (who puts m mod 0 = 0) *)
   401 Goal "a mod a = (0::int)";
   402 by (zdiv_undefined_case_tac "a = 0" 1);
   403 by (asm_simp_tac (simpset() addsimps [quorem_div_mod RS self_remainder]) 1);
   404 qed "zmod_self";
   405 Addsimps [zmod_self];
   406 
   407 
   408 (*** Computation of division and remainder ***)
   409 
   410 Goal "(0::int) div b = 0";
   411 by (simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   412 qed "zdiv_zero";
   413 
   414 Goal "(0::int) < b ==> -1 div b = -1";
   415 by (asm_simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   416 qed "div_eq_minus1";
   417 
   418 Goal "(0::int) mod b = 0";
   419 by (simp_tac (simpset() addsimps [mod_def, divAlg_def]) 1);
   420 qed "zmod_zero";
   421 
   422 Addsimps [zdiv_zero, zmod_zero];
   423 
   424 Goal "(0::int) < b ==> -1 div b = -1";
   425 by (asm_simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   426 qed "zdiv_minus1";
   427 
   428 Goal "(0::int) < b ==> -1 mod b = b - 1";
   429 by (asm_simp_tac (simpset() addsimps [mod_def, divAlg_def]) 1);
   430 qed "zmod_minus1";
   431 
   432 (** a positive, b positive **)
   433 
   434 Goal "[| 0 < a;  0 <= b |] ==> a div b = fst (posDivAlg(a,b))";
   435 by (asm_simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   436 qed "div_pos_pos";
   437 
   438 Goal "[| 0 < a;  0 <= b |] ==> a mod b = snd (posDivAlg(a,b))";
   439 by (asm_simp_tac (simpset() addsimps [mod_def, divAlg_def]) 1);
   440 qed "mod_pos_pos";
   441 
   442 (** a negative, b positive **)
   443 
   444 Goal "[| a < 0;  0 < b |] ==> a div b = fst (negDivAlg(a,b))";
   445 by (asm_simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   446 qed "div_neg_pos";
   447 
   448 Goal "[| a < 0;  0 < b |] ==> a mod b = snd (negDivAlg(a,b))";
   449 by (asm_simp_tac (simpset() addsimps [mod_def, divAlg_def]) 1);
   450 qed "mod_neg_pos";
   451 
   452 (** a positive, b negative **)
   453 
   454 Goal "[| 0 < a;  b < 0 |] ==> a div b = fst (negateSnd(negDivAlg(-a,-b)))";
   455 by (asm_simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   456 qed "div_pos_neg";
   457 
   458 Goal "[| 0 < a;  b < 0 |] ==> a mod b = snd (negateSnd(negDivAlg(-a,-b)))";
   459 by (asm_simp_tac (simpset() addsimps [mod_def, divAlg_def]) 1);
   460 qed "mod_pos_neg";
   461 
   462 (** a negative, b negative **)
   463 
   464 Goal "[| a < 0;  b <= 0 |] ==> a div b = fst (negateSnd(posDivAlg(-a,-b)))";
   465 by (asm_simp_tac (simpset() addsimps [div_def, divAlg_def]) 1);
   466 qed "div_neg_neg";
   467 
   468 Goal "[| a < 0;  b <= 0 |] ==> a mod b = snd (negateSnd(posDivAlg(-a,-b)))";
   469 by (asm_simp_tac (simpset() addsimps [mod_def, divAlg_def]) 1);
   470 qed "mod_neg_neg";
   471 
   472 Addsimps (map (read_instantiate_sg (sign_of (the_context ()))
   473 	       [("a", "number_of ?v"), ("b", "number_of ?w")])
   474 	  [div_pos_pos, div_neg_pos, div_pos_neg, div_neg_neg,
   475 	   mod_pos_pos, mod_neg_pos, mod_pos_neg, mod_neg_neg,
   476 	   posDivAlg_eqn, negDivAlg_eqn]);
   477 
   478 
   479 (** Special-case simplification **)
   480 
   481 Goal "a mod (1::int) = 0";
   482 by (cut_inst_tac [("a","a"),("b","1")] pos_mod_sign 1);
   483 by (cut_inst_tac [("a","a"),("b","1")] pos_mod_bound 2);
   484 by Auto_tac;
   485 qed "zmod_1";
   486 Addsimps [zmod_1];
   487 
   488 Goal "a div (1::int) = a";
   489 by (cut_inst_tac [("a","a"),("b","1")] zmod_zdiv_equality 1);
   490 by Auto_tac;
   491 qed "zdiv_1";
   492 Addsimps [zdiv_1];
   493 
   494 Goal "a mod (-1::int) = 0";
   495 by (cut_inst_tac [("a","a"),("b","-1")] neg_mod_sign 1);
   496 by (cut_inst_tac [("a","a"),("b","-1")] neg_mod_bound 2);
   497 by Auto_tac;
   498 qed "zmod_minus1_right";
   499 Addsimps [zmod_minus1_right];
   500 
   501 Goal "a div (-1::int) = -a";
   502 by (cut_inst_tac [("a","a"),("b","-1")] zmod_zdiv_equality 1);
   503 by Auto_tac;
   504 qed "zdiv_minus1_right";
   505 Addsimps [zdiv_minus1_right];
   506 
   507 (** The last remaining cases: 1 div z and 1 mod z **)
   508 
   509 Addsimps (map (fn th => int_0_less_1 RS inst "b" "number_of ?w" th) 
   510               [div_pos_pos, div_pos_neg, mod_pos_pos, mod_pos_neg]);
   511 
   512 Addsimps (map (read_instantiate_sg (sign_of (the_context ()))
   513 	       [("a", "1"), ("b", "number_of ?w")])
   514 	  [posDivAlg_eqn, negDivAlg_eqn]);
   515 
   516 
   517 (*** Monotonicity in the first argument (divisor) ***)
   518 
   519 Goal "[| a <= a';  0 < (b::int) |] ==> a div b <= a' div b";
   520 by (cut_inst_tac [("a","a"),("b","b")] zmod_zdiv_equality 1);
   521 by (cut_inst_tac [("a","a'"),("b","b")] zmod_zdiv_equality 1);
   522 by (rtac unique_quotient_lemma 1);
   523 by (etac subst 1);
   524 by (etac subst 1);
   525 by (ALLGOALS (asm_simp_tac (simpset() addsimps [pos_mod_sign,pos_mod_bound])));
   526 qed "zdiv_mono1";
   527 
   528 Goal "[| a <= a';  (b::int) < 0 |] ==> a' div b <= a div b";
   529 by (cut_inst_tac [("a","a"),("b","b")] zmod_zdiv_equality 1);
   530 by (cut_inst_tac [("a","a'"),("b","b")] zmod_zdiv_equality 1);
   531 by (rtac unique_quotient_lemma_neg 1);
   532 by (etac subst 1);
   533 by (etac subst 1);
   534 by (ALLGOALS (asm_simp_tac (simpset() addsimps [neg_mod_sign,neg_mod_bound])));
   535 qed "zdiv_mono1_neg";
   536 
   537 
   538 (*** Monotonicity in the second argument (dividend) ***)
   539 
   540 Goal "[| b*q + r = b'*q' + r';  0 <= b'*q' + r';  \
   541 \        r' < b';  0 <= r;  0 < b';  b' <= b |]  \
   542 \     ==> q <= (q'::int)";
   543 by (subgoal_tac "0 <= q'" 1);
   544  by (subgoal_tac "0 < b'*(q' + 1)" 2);
   545   by (asm_simp_tac (simpset() addsimps [zadd_zmult_distrib2]) 3);
   546  by (asm_full_simp_tac (simpset() addsimps [int_0_less_mult_iff]) 2);
   547 by (subgoal_tac "b*q < b*(q' + 1)" 1);
   548  by (asm_full_simp_tac (simpset() addsimps [zmult_zless_cancel1]) 1); 
   549 by (subgoal_tac "b*q = r' - r + b'*q'" 1);
   550  by (Simp_tac 2);
   551 by (asm_simp_tac (simpset() addsimps [zadd_zmult_distrib2]) 1);
   552 by (stac zadd_commute 1 THEN rtac zadd_zless_mono 1 THEN arith_tac 1);
   553 by (rtac zmult_zle_mono1 1);
   554 by Auto_tac;
   555 qed "zdiv_mono2_lemma";
   556 
   557 Goal "[| (0::int) <= a;  0 < b';  b' <= b |]  \
   558 \     ==> a div b <= a div b'";
   559 by (subgoal_tac "b ~= 0" 1);
   560 by (arith_tac 2);
   561 by (cut_inst_tac [("a","a"),("b","b")] zmod_zdiv_equality 1);
   562 by (cut_inst_tac [("a","a"),("b","b'")] zmod_zdiv_equality 1);
   563 by (rtac zdiv_mono2_lemma 1);
   564 by (etac subst 1);
   565 by (etac subst 1);
   566 by (ALLGOALS (asm_simp_tac (simpset() addsimps [pos_mod_sign,pos_mod_bound])));
   567 qed "zdiv_mono2";
   568 
   569 Goal "[| b*q + r = b'*q' + r';  b'*q' + r' < 0;  \
   570 \        r < b;  0 <= r';  0 < b';  b' <= b |]  \
   571 \     ==> q' <= (q::int)";
   572 by (subgoal_tac "q' < 0" 1);
   573  by (subgoal_tac "b'*q' < 0" 2);
   574   by (arith_tac 3);
   575  by (asm_full_simp_tac (simpset() addsimps [zmult_less_0_iff]) 2);
   576 by (subgoal_tac "b*q' < b*(q + 1)" 1);
   577  by (asm_full_simp_tac (simpset() addsimps [zmult_zless_cancel1]) 1); 
   578 by (asm_simp_tac (simpset() addsimps [zadd_zmult_distrib2]) 1);
   579 by (subgoal_tac "b*q' <= b'*q'" 1);
   580  by (asm_simp_tac (simpset() addsimps [zmult_zle_mono1_neg]) 2);
   581 by (subgoal_tac "b'*q' < b + b*q" 1);
   582  by (Asm_simp_tac 2);
   583 by (arith_tac 1);
   584 qed "zdiv_mono2_neg_lemma";
   585 
   586 Goal "[| a < (0::int);  0 < b';  b' <= b |]  \
   587 \     ==> a div b' <= a div b";
   588 by (cut_inst_tac [("a","a"),("b","b")] zmod_zdiv_equality 1);
   589 by (cut_inst_tac [("a","a"),("b","b'")] zmod_zdiv_equality 1);
   590 by (rtac zdiv_mono2_neg_lemma 1);
   591 by (etac subst 1);
   592 by (etac subst 1);
   593 by (ALLGOALS (asm_simp_tac (simpset() addsimps [pos_mod_sign,pos_mod_bound])));
   594 qed "zdiv_mono2_neg";
   595 
   596 
   597 (*** More algebraic laws for div and mod ***)
   598 
   599 (** proving (a*b) div c = a * (b div c) + a * (b mod c) **)
   600 
   601 Goal "[| quorem((b,c),(q,r));  c ~= 0 |] \
   602 \     ==> quorem ((a*b, c), (a*q + a*r div c, a*r mod c))";
   603 by (auto_tac
   604     (claset(),
   605      simpset() addsimps split_ifs@
   606                         [quorem_def, linorder_neq_iff, 
   607 			 zadd_zmult_distrib2,
   608 			 pos_mod_sign,pos_mod_bound,
   609 			 neg_mod_sign, neg_mod_bound]));
   610 by (ALLGOALS(rtac zmod_zdiv_equality));
   611 val lemma = result();
   612 
   613 Goal "(a*b) div c = a*(b div c) + a*(b mod c) div (c::int)";
   614 by (zdiv_undefined_case_tac "c = 0" 1);
   615 by (blast_tac (claset() addIs [quorem_div_mod RS lemma RS quorem_div]) 1);
   616 qed "zdiv_zmult1_eq";
   617 
   618 Goal "(a*b) mod c = a*(b mod c) mod (c::int)";
   619 by (zdiv_undefined_case_tac "c = 0" 1);
   620 by (blast_tac (claset() addIs [quorem_div_mod RS lemma RS quorem_mod]) 1);
   621 qed "zmod_zmult1_eq";
   622 
   623 Goal "(a*b) mod (c::int) = ((a mod c) * b) mod c";
   624 by (rtac trans 1);
   625 by (res_inst_tac [("s","b*a mod c")] trans 1);
   626 by (rtac zmod_zmult1_eq 2);
   627 by (ALLGOALS (simp_tac (simpset() addsimps [zmult_commute])));
   628 qed "zmod_zmult1_eq'";
   629 
   630 Goal "(a*b) mod (c::int) = ((a mod c) * (b mod c)) mod c";
   631 by (rtac (zmod_zmult1_eq' RS trans) 1);
   632 by (rtac zmod_zmult1_eq 1);
   633 qed "zmod_zmult_distrib";
   634 
   635 Goal "b ~= (0::int) ==> (a*b) div b = a";
   636 by (asm_simp_tac (simpset() addsimps [zdiv_zmult1_eq]) 1);
   637 qed "zdiv_zmult_self1";
   638 
   639 Goal "b ~= (0::int) ==> (b*a) div b = a";
   640 by (stac zmult_commute 1 THEN etac zdiv_zmult_self1 1);
   641 qed "zdiv_zmult_self2";
   642 
   643 Addsimps [zdiv_zmult_self1, zdiv_zmult_self2];
   644 
   645 Goal "(a*b) mod b = (0::int)";
   646 by (simp_tac (simpset() addsimps [zmod_zmult1_eq]) 1);
   647 qed "zmod_zmult_self1";
   648 
   649 Goal "(b*a) mod b = (0::int)";
   650 by (simp_tac (simpset() addsimps [zmult_commute, zmod_zmult1_eq]) 1);
   651 qed "zmod_zmult_self2";
   652 
   653 Addsimps [zmod_zmult_self1, zmod_zmult_self2];
   654 
   655 Goal "(m mod d = 0) = (EX q::int. m = d*q)";
   656 by (cut_inst_tac [("a","m"),("b","d")] zmod_zdiv_equality 1);
   657 by Auto_tac;  
   658 qed "zmod_eq_0_iff";
   659 AddSDs [zmod_eq_0_iff RS iffD1];
   660 
   661 
   662 (** proving (a+b) div c = a div c + b div c + ((a mod c + b mod c) div c) **)
   663 
   664 Goal "[| quorem((a,c),(aq,ar));  quorem((b,c),(bq,br));  c ~= 0 |] \
   665 \     ==> quorem ((a+b, c), (aq + bq + (ar+br) div c, (ar+br) mod c))";
   666 by (auto_tac
   667     (claset(),
   668      simpset() addsimps split_ifs@
   669                         [quorem_def, linorder_neq_iff, 
   670 			 zadd_zmult_distrib2,
   671 			 pos_mod_sign,pos_mod_bound,
   672 			 neg_mod_sign, neg_mod_bound]));
   673 by (ALLGOALS(rtac zmod_zdiv_equality));
   674 val lemma = result();
   675 
   676 (*NOT suitable for rewriting: the RHS has an instance of the LHS*)
   677 Goal "(a+b) div (c::int) = a div c + b div c + ((a mod c + b mod c) div c)";
   678 by (zdiv_undefined_case_tac "c = 0" 1);
   679 by (blast_tac (claset() addIs [[quorem_div_mod,quorem_div_mod]
   680 			       MRS lemma RS quorem_div]) 1);
   681 qed "zdiv_zadd1_eq";
   682 
   683 Goal "(a+b) mod (c::int) = (a mod c + b mod c) mod c";
   684 by (zdiv_undefined_case_tac "c = 0" 1);
   685 by (blast_tac (claset() addIs [[quorem_div_mod,quorem_div_mod]
   686 			       MRS lemma RS quorem_mod]) 1);
   687 qed "zmod_zadd1_eq";
   688 
   689 Goal "(a mod b) div b = (0::int)";
   690 by (zdiv_undefined_case_tac "b = 0" 1);
   691 by (auto_tac (claset(), 
   692        simpset() addsimps [linorder_neq_iff, 
   693 			   pos_mod_sign, pos_mod_bound, div_pos_pos_trivial, 
   694 			   neg_mod_sign, neg_mod_bound, div_neg_neg_trivial]));
   695 qed "mod_div_trivial";
   696 Addsimps [mod_div_trivial];
   697 
   698 Goal "(a mod b) mod b = a mod (b::int)";
   699 by (zdiv_undefined_case_tac "b = 0" 1);
   700 by (auto_tac (claset(), 
   701        simpset() addsimps [linorder_neq_iff, 
   702 			   pos_mod_sign, pos_mod_bound, mod_pos_pos_trivial, 
   703 			   neg_mod_sign, neg_mod_bound, mod_neg_neg_trivial]));
   704 qed "mod_mod_trivial";
   705 Addsimps [mod_mod_trivial];
   706 
   707 Goal "(a+b) mod (c::int) = ((a mod c) + b) mod c";
   708 by (rtac (trans RS sym) 1);
   709 by (rtac zmod_zadd1_eq 1);
   710 by (Simp_tac 1);
   711 by (rtac (zmod_zadd1_eq RS sym) 1);
   712 qed "zmod_zadd_left_eq";
   713 
   714 Goal "(a+b) mod (c::int) = (a + (b mod c)) mod c";
   715 by (rtac (trans RS sym) 1);
   716 by (rtac zmod_zadd1_eq 1);
   717 by (Simp_tac 1);
   718 by (rtac (zmod_zadd1_eq RS sym) 1);
   719 qed "zmod_zadd_right_eq";
   720 
   721 
   722 Goal "a ~= (0::int) ==> (a+b) div a = b div a + 1";
   723 by (asm_simp_tac (simpset() addsimps [zdiv_zadd1_eq]) 1);
   724 qed "zdiv_zadd_self1";
   725 
   726 Goal "a ~= (0::int) ==> (b+a) div a = b div a + 1";
   727 by (asm_simp_tac (simpset() addsimps [zdiv_zadd1_eq]) 1);
   728 qed "zdiv_zadd_self2";
   729 Addsimps [zdiv_zadd_self1, zdiv_zadd_self2];
   730 
   731 Goal "(a+b) mod a = b mod (a::int)";
   732 by (zdiv_undefined_case_tac "a = 0" 1);
   733 by (asm_simp_tac (simpset() addsimps [zmod_zadd1_eq]) 1);
   734 qed "zmod_zadd_self1";
   735 
   736 Goal "(b+a) mod a = b mod (a::int)";
   737 by (zdiv_undefined_case_tac "a = 0" 1);
   738 by (asm_simp_tac (simpset() addsimps [zmod_zadd1_eq]) 1);
   739 qed "zmod_zadd_self2";
   740 Addsimps [zmod_zadd_self1, zmod_zadd_self2];
   741 
   742 
   743 (*** proving  a div (b*c) = (a div b) div c ***)
   744 
   745 (*The condition c>0 seems necessary.  Consider that 7 div ~6 = ~2 but
   746   7 div 2 div ~3 = 3 div ~3 = ~1.  The subcase (a div b) mod c = 0 seems
   747   to cause particular problems.*)
   748 
   749 (** first, four lemmas to bound the remainder for the cases b<0 and b>0 **)
   750 
   751 Goal "[| (0::int) < c;  b < r;  r <= 0 |] ==> b*c < b*(q mod c) + r";
   752 by (subgoal_tac "b * (c - q mod c) < r * 1" 1);
   753 by (asm_full_simp_tac (simpset() addsimps [zdiff_zmult_distrib2]) 1);
   754 by (rtac order_le_less_trans 1);
   755 by (etac zmult_zless_mono1 2);
   756 by (rtac zmult_zle_mono2_neg 1);
   757 by (auto_tac
   758     (claset(),
   759      simpset() addsimps zcompare_rls@
   760                         [inst "z" "1" zadd_commute, add1_zle_eq, 
   761                          pos_mod_bound]));
   762 val lemma1 = result();
   763 
   764 Goal "[| (0::int) < c;   b < r;  r <= 0 |] ==> b * (q mod c) + r <= 0";
   765 by (subgoal_tac "b * (q mod c) <= 0" 1);
   766 by (arith_tac 1);
   767 by (asm_simp_tac (simpset() addsimps [zmult_le_0_iff, pos_mod_sign]) 1);
   768 val lemma2 = result();
   769 
   770 Goal "[| (0::int) < c;  0 <= r;  r < b |] ==> 0 <= b * (q mod c) + r";
   771 by (subgoal_tac "0 <= b * (q mod c)" 1);
   772 by (arith_tac 1);
   773 by (asm_simp_tac (simpset() addsimps [int_0_le_mult_iff, pos_mod_sign]) 1);
   774 val lemma3 = result();
   775 
   776 Goal "[| (0::int) < c; 0 <= r; r < b |] ==> b * (q mod c) + r < b * c";
   777 by (subgoal_tac "r * 1 < b * (c - q mod c)" 1);
   778 by (asm_full_simp_tac (simpset() addsimps [zdiff_zmult_distrib2]) 1);
   779 by (rtac order_less_le_trans 1);
   780 by (etac zmult_zless_mono1 1);
   781 by (rtac zmult_zle_mono2 2);
   782 by (auto_tac
   783     (claset(),
   784      simpset() addsimps zcompare_rls@
   785                         [inst "z" "1" zadd_commute, add1_zle_eq,
   786                          pos_mod_bound]));
   787 val lemma4 = result();
   788 
   789 Goal "[| quorem ((a,b), (q,r));  b ~= 0;  0 < c |] \
   790 \     ==> quorem ((a, b*c), (q div c, b*(q mod c) + r))";
   791 by (auto_tac  
   792     (claset(),
   793      simpset() addsimps zmult_ac@
   794                         [zmod_zdiv_equality, quorem_def, linorder_neq_iff,
   795 			 int_0_less_mult_iff,
   796 			 zadd_zmult_distrib2 RS sym,
   797 			 lemma1, lemma2, lemma3, lemma4]));
   798 val lemma = result();
   799 
   800 Goal "(0::int) < c ==> a div (b*c) = (a div b) div c";
   801 by (zdiv_undefined_case_tac "b = 0" 1);
   802 by (force_tac (claset(),
   803 	       simpset() addsimps [quorem_div_mod RS lemma RS quorem_div, 
   804 				   zmult_eq_0_iff]) 1);
   805 qed "zdiv_zmult2_eq";
   806 
   807 Goal "(0::int) < c ==> a mod (b*c) = b*(a div b mod c) + a mod b";
   808 by (zdiv_undefined_case_tac "b = 0" 1);
   809 by (force_tac (claset(),
   810 	       simpset() addsimps [quorem_div_mod RS lemma RS quorem_mod, 
   811 				   zmult_eq_0_iff]) 1);
   812 qed "zmod_zmult2_eq";
   813 
   814 
   815 (*** Cancellation of common factors in "div" ***)
   816 
   817 Goal "[| (0::int) < b;  c ~= 0 |] ==> (c*a) div (c*b) = a div b";
   818 by (stac zdiv_zmult2_eq 1);
   819 by Auto_tac;
   820 val lemma1 = result();
   821 
   822 Goal "[| b < (0::int);  c ~= 0 |] ==> (c*a) div (c*b) = a div b";
   823 by (subgoal_tac "(c * (-a)) div (c * (-b)) = (-a) div (-b)" 1);
   824 by (rtac lemma1 2);
   825 by Auto_tac;
   826 val lemma2 = result();
   827 
   828 Goal "c ~= (0::int) ==> (c*a) div (c*b) = a div b";
   829 by (zdiv_undefined_case_tac "b = 0" 1);
   830 by (auto_tac
   831     (claset(), 
   832      simpset() addsimps [read_instantiate [("x", "b")] linorder_neq_iff, 
   833 			 lemma1, lemma2]));
   834 qed "zdiv_zmult_zmult1";
   835 
   836 Goal "c ~= (0::int) ==> (a*c) div (b*c) = a div b";
   837 by (dtac zdiv_zmult_zmult1 1);
   838 by (auto_tac (claset(), simpset() addsimps [zmult_commute]));
   839 qed "zdiv_zmult_zmult2";
   840 
   841 
   842 
   843 (*** Distribution of factors over "mod" ***)
   844 
   845 Goal "[| (0::int) < b;  c ~= 0 |] ==> (c*a) mod (c*b) = c * (a mod b)";
   846 by (stac zmod_zmult2_eq 1);
   847 by Auto_tac;
   848 val lemma1 = result();
   849 
   850 Goal "[| b < (0::int);  c ~= 0 |] ==> (c*a) mod (c*b) = c * (a mod b)";
   851 by (subgoal_tac "(c * (-a)) mod (c * (-b)) = c * ((-a) mod (-b))" 1);
   852 by (rtac lemma1 2);
   853 by Auto_tac;
   854 val lemma2 = result();
   855 
   856 Goal "(c*a) mod (c*b) = (c::int) * (a mod b)";
   857 by (zdiv_undefined_case_tac "b = 0" 1);
   858 by (zdiv_undefined_case_tac "c = 0" 1);
   859 by (auto_tac
   860     (claset(), 
   861      simpset() addsimps [read_instantiate [("x", "b")] linorder_neq_iff, 
   862 			 lemma1, lemma2]));
   863 qed "zmod_zmult_zmult1";
   864 
   865 Goal "(a*c) mod (b*c) = (a mod b) * (c::int)";
   866 by (cut_inst_tac [("c","c")] zmod_zmult_zmult1 1);
   867 by (auto_tac (claset(), simpset() addsimps [zmult_commute]));
   868 qed "zmod_zmult_zmult2";
   869 
   870 
   871 (*** Speeding up the division algorithm with shifting ***)
   872 
   873 (** computing "div" by shifting **)
   874 
   875 Goal "(0::int) <= a ==> (1 + 2*b) div (2*a) = b div a";
   876 by (zdiv_undefined_case_tac "a = 0" 1);
   877 by (subgoal_tac "1 <= a" 1);
   878  by (arith_tac 2);
   879 by (subgoal_tac "1 < a * 2" 1);
   880  by (arith_tac 2);
   881 by (subgoal_tac "2*(1 + b mod a) <= 2*a" 1);
   882  by (rtac zmult_zle_mono2 2);
   883 by (auto_tac (claset(),
   884 	      simpset() addsimps [inst "z" "1" zadd_commute, zmult_commute, 
   885 				  add1_zle_eq, pos_mod_bound]));
   886 by (stac zdiv_zadd1_eq 1);
   887 by (asm_simp_tac (simpset() addsimps [zdiv_zmult_zmult2, zmod_zmult_zmult2, 
   888 				      div_pos_pos_trivial]) 1);
   889 by (stac div_pos_pos_trivial 1);
   890 by (asm_simp_tac (simpset() 
   891            addsimps [mod_pos_pos_trivial,
   892                     pos_mod_sign RS zadd_zle_mono1 RSN (2,order_trans)]) 1);
   893 by (auto_tac (claset(),
   894 	      simpset() addsimps [mod_pos_pos_trivial]));
   895 by (subgoal_tac "0 <= b mod a" 1);
   896  by (asm_simp_tac (simpset() addsimps [pos_mod_sign]) 2);
   897 by (arith_tac 1);
   898 qed "pos_zdiv_mult_2";
   899 
   900 
   901 Goal "a <= (0::int) ==> (1 + 2*b) div (2*a) = (b+1) div a";
   902 by (subgoal_tac "(1 + 2*(-b - 1)) div (2 * (-a)) = (-b - 1) div (-a)" 1);
   903 by (rtac pos_zdiv_mult_2 2);
   904 by (auto_tac (claset(),
   905 	      simpset() addsimps [zmult_zminus_right]));
   906 by (subgoal_tac "(-1 - (2 * b)) = - (1 + (2 * b))" 1);
   907 by (Simp_tac 2);
   908 by (asm_full_simp_tac (HOL_ss
   909 		       addsimps [zdiv_zminus_zminus, zdiff_def,
   910 				 zminus_zadd_distrib RS sym]) 1);
   911 qed "neg_zdiv_mult_2";
   912 
   913 
   914 (*Not clear why this must be proved separately; probably number_of causes
   915   simplification problems*)
   916 Goal "~ 0 <= x ==> x <= (0::int)";
   917 by Auto_tac;
   918 val lemma = result();
   919 
   920 Goal "number_of (v BIT b) div number_of (w BIT False) = \
   921 \         (if ~b | (0::int) <= number_of w                   \
   922 \          then number_of v div (number_of w)    \
   923 \          else (number_of v + (1::int)) div (number_of w))";
   924 by (simp_tac (simpset_of Int.thy addsimps [zadd_assoc, number_of_BIT]) 1);
   925 by (subgoal_tac "2 ~= (0::int)" 1);
   926  by (Simp_tac 2);  (*we do this because the next step can't simplify numerals*)
   927 by (asm_simp_tac (simpset()
   928            delsimps bin_arith_extra_simps
   929  	   addsimps [zdiv_zmult_zmult1, pos_zdiv_mult_2, lemma, 
   930                      neg_zdiv_mult_2]) 1);
   931 qed "zdiv_number_of_BIT";
   932 Addsimps [zdiv_number_of_BIT];
   933 
   934 
   935 (** computing "mod" by shifting (proofs resemble those for "div") **)
   936 
   937 Goal "(0::int) <= a ==> (1 + 2*b) mod (2*a) = 1 + 2 * (b mod a)";
   938 by (zdiv_undefined_case_tac "a = 0" 1);
   939 by (subgoal_tac "1 <= a" 1);
   940  by (arith_tac 2);
   941 by (subgoal_tac "1 < a * 2" 1);
   942  by (arith_tac 2);
   943 by (subgoal_tac "2*(1 + b mod a) <= 2*a" 1);
   944  by (rtac zmult_zle_mono2 2);
   945 by (auto_tac (claset(),
   946 	      simpset() addsimps [inst "z" "1" zadd_commute, zmult_commute, 
   947 				  add1_zle_eq, pos_mod_bound]));
   948 by (stac zmod_zadd1_eq 1);
   949 by (asm_simp_tac (simpset() addsimps [zmod_zmult_zmult2, 
   950 				      mod_pos_pos_trivial]) 1);
   951 by (rtac mod_pos_pos_trivial 1);
   952 by (asm_simp_tac (simpset() 
   953                   addsimps [mod_pos_pos_trivial,
   954                     pos_mod_sign RS zadd_zle_mono1 RSN (2,order_trans)]) 1);
   955 by (auto_tac (claset(),
   956 	      simpset() addsimps [mod_pos_pos_trivial]));
   957 by (subgoal_tac "0 <= b mod a" 1);
   958  by (asm_simp_tac (simpset() addsimps [pos_mod_sign]) 2);
   959 by (arith_tac 1);
   960 qed "pos_zmod_mult_2";
   961 
   962 
   963 Goal "a <= (0::int) ==> (1 + 2*b) mod (2*a) = 2 * ((b+1) mod a) - 1";
   964 by (subgoal_tac 
   965     "(1 + 2*(-b - 1)) mod (2*(-a)) = 1 + 2*((-b - 1) mod (-a))" 1);
   966 by (rtac pos_zmod_mult_2 2);
   967 by (auto_tac (claset(), simpset() addsimps [zmult_zminus_right]));
   968 by (subgoal_tac "(-1 - (2 * b)) = - (1 + (2 * b))" 1);
   969 by (Simp_tac 2);
   970 by (asm_full_simp_tac (HOL_ss
   971 		       addsimps [zmod_zminus_zminus, zdiff_def,
   972 				 zminus_zadd_distrib RS sym]) 1);
   973 by (dtac (zminus_equation RS iffD1 RS sym) 1);
   974 by Auto_tac;
   975 qed "neg_zmod_mult_2";
   976 
   977 Goal "number_of (v BIT b) mod number_of (w BIT False) = \
   978 \         (if b then \
   979 \               if (0::int) <= number_of w \
   980 \               then 2 * (number_of v mod number_of w) + 1    \
   981 \               else 2 * ((number_of v + (1::int)) mod number_of w) - 1  \
   982 \          else 2 * (number_of v mod number_of w))";
   983 by (simp_tac (simpset_of Int.thy addsimps [zadd_assoc, number_of_BIT]) 1);
   984 by (asm_simp_tac (simpset()
   985 		  delsimps bin_arith_extra_simps@bin_rel_simps
   986 		  addsimps [zmod_zmult_zmult1,
   987 			    pos_zmod_mult_2, lemma, neg_zmod_mult_2]) 1);
   988 by (Simp_tac 1); 
   989 qed "zmod_number_of_BIT";
   990 
   991 Addsimps [zmod_number_of_BIT];
   992 
   993 
   994 (** Quotients of signs **)
   995 
   996 Goal "[| a < (0::int);  0 < b |] ==> a div b < 0";
   997 by (subgoal_tac "a div b <= -1" 1);
   998 by (Force_tac 1);
   999 by (rtac order_trans 1);
  1000 by (res_inst_tac [("a'","-1")]  zdiv_mono1 1);
  1001 by (auto_tac (claset(), simpset() addsimps [zdiv_minus1]));
  1002 qed "div_neg_pos_less0";
  1003 
  1004 Goal "[| (0::int) <= a;  b < 0 |] ==> a div b <= 0";
  1005 by (dtac zdiv_mono1_neg 1);
  1006 by Auto_tac;
  1007 qed "div_nonneg_neg_le0";
  1008 
  1009 Goal "(0::int) < b ==> (0 <= a div b) = (0 <= a)";
  1010 by Auto_tac;
  1011 by (dtac zdiv_mono1 2);
  1012 by (auto_tac (claset(), simpset() addsimps [linorder_neq_iff]));
  1013 by (full_simp_tac (simpset() addsimps [linorder_not_less RS sym]) 1);
  1014 by (blast_tac (claset() addIs [div_neg_pos_less0]) 1);
  1015 qed "pos_imp_zdiv_nonneg_iff";
  1016 
  1017 Goal "b < (0::int) ==> (0 <= a div b) = (a <= (0::int))";
  1018 by (stac (zdiv_zminus_zminus RS sym) 1);
  1019 by (stac pos_imp_zdiv_nonneg_iff 1);
  1020 by Auto_tac;
  1021 qed "neg_imp_zdiv_nonneg_iff";
  1022 
  1023 (*But not (a div b <= 0 iff a<=0); consider a=1, b=2 when a div b = 0.*)
  1024 Goal "(0::int) < b ==> (a div b < 0) = (a < 0)";
  1025 by (asm_simp_tac (simpset() addsimps [linorder_not_le RS sym,
  1026 				      pos_imp_zdiv_nonneg_iff]) 1);
  1027 qed "pos_imp_zdiv_neg_iff";
  1028 
  1029 (*Again the law fails for <=: consider a = -1, b = -2 when a div b = 0*)
  1030 Goal "b < (0::int) ==> (a div b < 0) = (0 < a)";
  1031 by (asm_simp_tac (simpset() addsimps [linorder_not_le RS sym,
  1032 				      neg_imp_zdiv_nonneg_iff]) 1);
  1033 qed "neg_imp_zdiv_neg_iff";