src/HOL/Divides.ML
author wenzelm
Mon, 22 Jun 1998 17:26:46 +0200
changeset 5069 3ea049f7979d
parent 4811 7a98aa1f9a9d
child 5143 b94cd208f073
permissions -rw-r--r--
isatool fixgoal;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     1
(*  Title:      HOL/Divides.ML
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     2
    ID:         $Id$
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     5
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     6
The division operators div, mod and the divides relation "dvd"
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     7
*)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     8
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
     9
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    10
(** Less-then properties **)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    11
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    12
(*In ordinary notation: if 0<n and n<=m then m-n < m *)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    13
goal Arith.thy "!!m. [| 0<n; ~ m<n |] ==> m - n < m";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    14
by (subgoal_tac "0<n --> ~ m<n --> m - n < m" 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    15
by (Blast_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    16
by (res_inst_tac [("m","m"),("n","n")] diff_induct 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    17
by (ALLGOALS(asm_simp_tac(simpset() addsimps [diff_less_Suc])));
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    18
qed "diff_less";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    19
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    20
val wf_less_trans = [eq_reflection, wf_pred_nat RS wf_trancl] MRS 
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    21
                    def_wfrec RS trans;
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    22
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    23
(*** Remainder ***)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    24
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    25
Goal "(%m. m mod n) = wfrec (trancl pred_nat) \
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    26
             \                      (%f j. if j<n then j else f (j-n))";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    27
by (simp_tac (simpset() addsimps [mod_def]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    28
qed "mod_eq";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    29
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    30
Goal "!!m. m<n ==> m mod n = m";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    31
by (rtac (mod_eq RS wf_less_trans) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    32
by (Asm_simp_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    33
qed "mod_less";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    34
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    35
Goal "!!m. [| 0<n;  ~m<n |] ==> m mod n = (m-n) mod n";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    36
by (rtac (mod_eq RS wf_less_trans) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    37
by (asm_simp_tac (simpset() addsimps [diff_less, cut_apply, less_eq]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    38
qed "mod_geq";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    39
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    40
(*NOT suitable for rewriting: loops*)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    41
Goal "!!m. 0<n ==> m mod n = (if m<n then m else (m-n) mod n)";
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    42
by (asm_simp_tac (simpset() addsimps [mod_less, mod_geq]) 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    43
qed "mod_if";
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    44
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    45
Goal "m mod 1 = 0";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    46
by (induct_tac "m" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    47
by (ALLGOALS (asm_simp_tac (simpset() addsimps [mod_less, mod_geq])));
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    48
qed "mod_1";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    49
Addsimps [mod_1];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    50
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    51
Goal "!!n. 0<n ==> n mod n = 0";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    52
by (asm_simp_tac (simpset() addsimps [mod_less, mod_geq]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    53
qed "mod_self";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    54
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    55
Goal "!!n. 0<n ==> (m+n) mod n = m mod n";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    56
by (subgoal_tac "(n + m) mod n = (n+m-n) mod n" 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    57
by (stac (mod_geq RS sym) 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    58
by (ALLGOALS (asm_full_simp_tac (simpset() addsimps [add_commute])));
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    59
qed "mod_add_self2";
4810
d55e2fee2084 New laws for mod
paulson
parents: 4774
diff changeset
    60
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    61
Goal "!!k. 0<n ==> (n+m) mod n = m mod n";
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    62
by (asm_simp_tac (simpset() addsimps [add_commute, mod_add_self2]) 1);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    63
qed "mod_add_self1";
4810
d55e2fee2084 New laws for mod
paulson
parents: 4774
diff changeset
    64
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    65
Goal "!!n. 0<n ==> (m + k*n) mod n = m mod n";
4810
d55e2fee2084 New laws for mod
paulson
parents: 4774
diff changeset
    66
by (induct_tac "k" 1);
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    67
by (ALLGOALS (asm_simp_tac (simpset() addsimps (add_ac @ [mod_add_self1]))));
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    68
qed "mod_mult_self1";
4810
d55e2fee2084 New laws for mod
paulson
parents: 4774
diff changeset
    69
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    70
Goal "!!m. 0<n ==> (m + n*k) mod n = m mod n";
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    71
by (asm_simp_tac (simpset() addsimps [mult_commute, mod_mult_self1]) 1);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    72
qed "mod_mult_self2";
4810
d55e2fee2084 New laws for mod
paulson
parents: 4774
diff changeset
    73
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    74
Addsimps [mod_mult_self1, mod_mult_self2];
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    75
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    76
Goal "!!k. [| 0<k; 0<n |] ==> (m mod n)*k = (m*k) mod (n*k)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    77
by (res_inst_tac [("n","m")] less_induct 1);
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    78
by (stac mod_if 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    79
by (Asm_simp_tac 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    80
by (asm_simp_tac (simpset() addsimps [mod_less, mod_geq, 
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    81
				      diff_less, diff_mult_distrib]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    82
qed "mod_mult_distrib";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    83
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    84
Goal "!!k. [| 0<k; 0<n |] ==> k*(m mod n) = (k*m) mod (k*n)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    85
by (res_inst_tac [("n","m")] less_induct 1);
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    86
by (stac mod_if 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    87
by (Asm_simp_tac 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    88
by (asm_simp_tac (simpset() addsimps [mod_less, mod_geq, 
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
    89
				      diff_less, diff_mult_distrib2]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    90
qed "mod_mult_distrib2";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    91
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
    92
Goal "!!n. 0<n ==> m*n mod n = 0";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    93
by (induct_tac "m" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    94
by (asm_simp_tac (simpset() addsimps [mod_less]) 1);
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
    95
by (dres_inst_tac [("m","m*n")] mod_add_self2 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
    96
by (asm_full_simp_tac (simpset() addsimps [add_commute]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    97
qed "mod_mult_self_is_0";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    98
Addsimps [mod_mult_self_is_0];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
    99
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   100
(*** Quotient ***)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   101
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   102
Goal "(%m. m div n) = wfrec (trancl pred_nat) \
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   103
                        \            (%f j. if j<n then 0 else Suc (f (j-n)))";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   104
by (simp_tac (simpset() addsimps [div_def]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   105
qed "div_eq";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   106
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   107
Goal "!!m. m<n ==> m div n = 0";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   108
by (rtac (div_eq RS wf_less_trans) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   109
by (Asm_simp_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   110
qed "div_less";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   111
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   112
Goal "!!M. [| 0<n;  ~m<n |] ==> m div n = Suc((m-n) div n)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   113
by (rtac (div_eq RS wf_less_trans) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   114
by (asm_simp_tac (simpset() addsimps [diff_less, cut_apply, less_eq]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   115
qed "div_geq";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   116
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   117
(*NOT suitable for rewriting: loops*)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   118
Goal "!!m. 0<n ==> m div n = (if m<n then 0 else Suc((m-n) div n))";
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   119
by (asm_simp_tac (simpset() addsimps [div_less, div_geq]) 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   120
qed "div_if";
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   121
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   122
(*Main Result about quotient and remainder.*)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   123
Goal "!!m. 0<n ==> (m div n)*n + m mod n = m";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   124
by (res_inst_tac [("n","m")] less_induct 1);
4774
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   125
by (stac mod_if 1);
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   126
by (ALLGOALS (asm_simp_tac 
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   127
	      (simpset() addsimps ([add_assoc] @
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   128
				   [div_less, div_geq,
b4760a833480 Tidied proofs by getting rid of case_tac
paulson
parents: 4686
diff changeset
   129
				    add_diff_inverse, diff_less]))));
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   130
qed "mod_div_equality";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   131
4358
aa22fcb46a5d Added thm mult_div_cancel
nipkow
parents: 4356
diff changeset
   132
(* a simple rearrangement of mod_div_equality: *)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   133
Goal "!!k. 0<k ==> k*(m div k) = m - (m mod k)";
4423
a129b817b58a expandshort;
wenzelm
parents: 4385
diff changeset
   134
by (dres_inst_tac [("m","m")] mod_div_equality 1);
4358
aa22fcb46a5d Added thm mult_div_cancel
nipkow
parents: 4356
diff changeset
   135
by (EVERY1[etac subst, simp_tac (simpset() addsimps mult_ac),
aa22fcb46a5d Added thm mult_div_cancel
nipkow
parents: 4356
diff changeset
   136
           K(IF_UNSOLVED no_tac)]);
aa22fcb46a5d Added thm mult_div_cancel
nipkow
parents: 4356
diff changeset
   137
qed "mult_div_cancel";
aa22fcb46a5d Added thm mult_div_cancel
nipkow
parents: 4356
diff changeset
   138
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   139
Goal "m div 1 = m";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   140
by (induct_tac "m" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   141
by (ALLGOALS (asm_simp_tac (simpset() addsimps [div_less, div_geq])));
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   142
qed "div_1";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   143
Addsimps [div_1];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   144
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   145
Goal "!!n. 0<n ==> n div n = 1";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   146
by (asm_simp_tac (simpset() addsimps [div_less, div_geq]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   147
qed "div_self";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   148
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   149
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   150
Goal "!!n. 0<n ==> (m+n) div n = Suc (m div n)";
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   151
by (subgoal_tac "(n + m) div n = Suc ((n+m-n) div n)" 1);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   152
by (stac (div_geq RS sym) 2);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   153
by (ALLGOALS (asm_full_simp_tac (simpset() addsimps [add_commute])));
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   154
qed "div_add_self2";
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   155
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   156
Goal "!!k. 0<n ==> (n+m) div n = Suc (m div n)";
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   157
by (asm_simp_tac (simpset() addsimps [add_commute, div_add_self2]) 1);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   158
qed "div_add_self1";
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   159
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   160
Goal "!!n. 0<n ==> (m + k*n) div n = k + m div n";
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   161
by (induct_tac "k" 1);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   162
by (ALLGOALS (asm_simp_tac (simpset() addsimps (add_ac @ [div_add_self1]))));
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   163
qed "div_mult_self1";
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   164
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   165
Goal "!!m. 0<n ==> (m + n*k) div n = k + m div n";
4811
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   166
by (asm_simp_tac (simpset() addsimps [mult_commute, div_mult_self1]) 1);
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   167
qed "div_mult_self2";
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   168
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   169
Addsimps [div_mult_self1, div_mult_self2];
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   170
7a98aa1f9a9d Renamed mod_XXX_cancel to mod_XXX_self
paulson
parents: 4810
diff changeset
   171
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   172
(* Monotonicity of div in first argument *)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   173
Goal "!!n. 0<k ==> ALL m. m <= n --> (m div k) <= (n div k)";
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   174
by (res_inst_tac [("n","n")] less_induct 1);
3718
d78cf498a88c Minor tidying to use Clarify_tac, etc.
paulson
parents: 3496
diff changeset
   175
by (Clarify_tac 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   176
by (case_tac "na<k" 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   177
(* 1  case n<k *)
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   178
by (subgoal_tac "m<k" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   179
by (asm_simp_tac (simpset() addsimps [div_less]) 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   180
by (trans_tac 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   181
(* 2  case n >= k *)
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   182
by (case_tac "m<k" 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   183
(* 2.1  case m<k *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   184
by (asm_simp_tac (simpset() addsimps [div_less]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   185
(* 2.2  case m>=k *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   186
by (asm_simp_tac (simpset() addsimps [div_geq, diff_less, diff_le_mono]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   187
qed_spec_mp "div_le_mono";
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   188
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   189
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   190
(* Antimonotonicity of div in second argument *)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   191
Goal "!!k m n. [| 0<m; m<=n |] ==> (k div n) <= (k div m)";
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   192
by (subgoal_tac "0<n" 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   193
 by (trans_tac 2);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   194
by (res_inst_tac [("n","k")] less_induct 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   195
by (Simp_tac 1);
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   196
by (rename_tac "k" 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   197
by (case_tac "k<n" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   198
 by (asm_simp_tac (simpset() addsimps [div_less]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   199
by (subgoal_tac "~(k<m)" 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   200
 by (trans_tac 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   201
by (asm_simp_tac (simpset() addsimps [div_geq]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   202
by (subgoal_tac "(k-n) div n <= (k-m) div n" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   203
 by (best_tac (claset() addIs [le_trans] 
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   204
                       addss (simpset() addsimps [diff_less])) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   205
by (REPEAT (eresolve_tac [div_le_mono,diff_le_mono2] 1));
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   206
qed "div_le_mono2";
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   207
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   208
Goal "!!m n. 0<n ==> m div n <= m";
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   209
by (subgoal_tac "m div n <= m div 1" 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   210
by (Asm_full_simp_tac 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   211
by (rtac div_le_mono2 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   212
by (ALLGOALS trans_tac);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   213
qed "div_le_dividend";
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   214
Addsimps [div_le_dividend];
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   215
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   216
(* Similar for "less than" *)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   217
Goal "!!m n. 1<n ==> (0 < m) --> (m div n < m)";
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   218
by (res_inst_tac [("n","m")] less_induct 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   219
by (Simp_tac 1);
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   220
by (rename_tac "m" 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   221
by (case_tac "m<n" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   222
 by (asm_full_simp_tac (simpset() addsimps [div_less]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   223
by (subgoal_tac "0<n" 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   224
 by (trans_tac 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   225
by (asm_full_simp_tac (simpset() addsimps [div_geq]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   226
by (case_tac "n<m" 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   227
 by (subgoal_tac "(m-n) div n < (m-n)" 1);
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   228
  by (REPEAT (ares_tac [impI,less_trans_Suc] 1));
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   229
  by (asm_full_simp_tac (simpset() addsimps [diff_less]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   230
 by (dres_inst_tac [("m","n")] less_imp_diff_positive 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   231
 by (asm_full_simp_tac (simpset() addsimps [diff_less]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   232
(* case n=m *)
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   233
by (subgoal_tac "m=n" 1);
3496
32e7edc609fd Simplified the new proofs about division
paulson
parents: 3484
diff changeset
   234
 by (trans_tac 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   235
by (asm_simp_tac (simpset() addsimps [div_less]) 1);
3484
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   236
qed_spec_mp "div_less_dividend";
1e93eb09ebb9 Added the following lemmas tp Divides and a few others to Arith and NatDef:
nipkow
parents: 3457
diff changeset
   237
Addsimps [div_less_dividend];
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   238
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   239
(*** Further facts about mod (mainly for the mutilated chess board ***)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   240
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   241
Goal
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   242
    "!!m n. 0<n ==> \
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   243
\           Suc(m) mod n = (if Suc(m mod n) = n then 0 else Suc(m mod n))";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   244
by (res_inst_tac [("n","m")] less_induct 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   245
by (excluded_middle_tac "Suc(na)<n" 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   246
(* case Suc(na) < n *)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   247
by (forward_tac [lessI RS less_trans] 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   248
by (asm_simp_tac (simpset() addsimps [mod_less, less_not_refl2 RS not_sym]) 2);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   249
(* case n <= Suc(na) *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   250
by (asm_full_simp_tac (simpset() addsimps [not_less_iff_le, mod_geq]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   251
by (etac (le_imp_less_or_eq RS disjE) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   252
by (asm_simp_tac (simpset() addsimps [Suc_diff_n]) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   253
by (asm_full_simp_tac (simpset() addsimps [not_less_eq RS sym, 
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   254
                                          diff_less, mod_geq]) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   255
by (asm_simp_tac (simpset() addsimps [mod_less]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   256
qed "mod_Suc";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   257
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   258
Goal "!!m n. 0<n ==> m mod n < n";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   259
by (res_inst_tac [("n","m")] less_induct 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   260
by (excluded_middle_tac "na<n" 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   261
(*case na<n*)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   262
by (asm_simp_tac (simpset() addsimps [mod_less]) 2);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   263
(*case n le na*)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   264
by (asm_full_simp_tac (simpset() addsimps [mod_geq, diff_less]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   265
qed "mod_less_divisor";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   266
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   267
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   268
(** Evens and Odds **)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   269
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   270
(*With less_zeroE, causes case analysis on b<2*)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   271
AddSEs [less_SucE];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   272
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   273
Goal "!!k b. b<2 ==> k mod 2 = b | k mod 2 = (if b=1 then 0 else 1)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   274
by (subgoal_tac "k mod 2 < 2" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   275
by (asm_simp_tac (simpset() addsimps [mod_less_divisor]) 2);
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4477
diff changeset
   276
by (Asm_simp_tac 1);
4356
0dfd34f0d33d Replaced n ~= 0 by 0 < n
nipkow
parents: 4089
diff changeset
   277
by Safe_tac;
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   278
qed "mod2_cases";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   279
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   280
Goal "Suc(Suc(m)) mod 2 = m mod 2";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   281
by (subgoal_tac "m mod 2 < 2" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   282
by (asm_simp_tac (simpset() addsimps [mod_less_divisor]) 2);
3724
f33e301a89f5 Step_tac -> Safe_tac
paulson
parents: 3718
diff changeset
   283
by Safe_tac;
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   284
by (ALLGOALS (asm_simp_tac (simpset() addsimps [mod_Suc])));
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   285
qed "mod2_Suc_Suc";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   286
Addsimps [mod2_Suc_Suc];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   287
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   288
Goal "(0 < m mod 2) = (m mod 2 = 1)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   289
by (subgoal_tac "m mod 2 < 2" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   290
by (asm_simp_tac (simpset() addsimps [mod_less_divisor]) 2);
4477
b3e5857d8d99 New Auto_tac (by Oheimb), and new syntax (without parens), and expandshort
paulson
parents: 4423
diff changeset
   291
by Auto_tac;
4356
0dfd34f0d33d Replaced n ~= 0 by 0 < n
nipkow
parents: 4089
diff changeset
   292
qed "mod2_gr_0";
0dfd34f0d33d Replaced n ~= 0 by 0 < n
nipkow
parents: 4089
diff changeset
   293
Addsimps [mod2_gr_0];
0dfd34f0d33d Replaced n ~= 0 by 0 < n
nipkow
parents: 4089
diff changeset
   294
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   295
Goal "(m+m) mod 2 = 0";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   296
by (induct_tac "m" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   297
by (simp_tac (simpset() addsimps [mod_less]) 1);
3427
e7cef2081106 Removed a few redundant additions of simprules or classical rules
paulson
parents: 3366
diff changeset
   298
by (Asm_simp_tac 1);
4385
f6d019eefa1e Got rid of mod2_neq_0
paulson
parents: 4358
diff changeset
   299
qed "mod2_add_self_eq_0";
f6d019eefa1e Got rid of mod2_neq_0
paulson
parents: 4358
diff changeset
   300
Addsimps [mod2_add_self_eq_0];
f6d019eefa1e Got rid of mod2_neq_0
paulson
parents: 4358
diff changeset
   301
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   302
Goal "((m+m)+n) mod 2 = n mod 2";
4385
f6d019eefa1e Got rid of mod2_neq_0
paulson
parents: 4358
diff changeset
   303
by (induct_tac "m" 1);
f6d019eefa1e Got rid of mod2_neq_0
paulson
parents: 4358
diff changeset
   304
by (simp_tac (simpset() addsimps [mod_less]) 1);
f6d019eefa1e Got rid of mod2_neq_0
paulson
parents: 4358
diff changeset
   305
by (Asm_simp_tac 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   306
qed "mod2_add_self";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   307
Addsimps [mod2_add_self];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   308
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   309
Delrules [less_SucE];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   310
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   311
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   312
(*** More division laws ***)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   313
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   314
Goal "!!n. 0<n ==> m*n div n = m";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   315
by (cut_inst_tac [("m", "m*n")] mod_div_equality 1);
3457
a8ab7c64817c Ran expandshort
paulson
parents: 3427
diff changeset
   316
by (assume_tac 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   317
by (asm_full_simp_tac (simpset() addsimps [mod_mult_self_is_0]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   318
qed "div_mult_self_is_m";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   319
Addsimps [div_mult_self_is_m];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   320
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   321
(*Cancellation law for division*)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   322
Goal "!!k. [| 0<n; 0<k |] ==> (k*m) div (k*n) = m div n";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   323
by (res_inst_tac [("n","m")] less_induct 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   324
by (case_tac "na<n" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   325
by (asm_simp_tac (simpset() addsimps [div_less, zero_less_mult_iff, 
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   326
                                     mult_less_mono2]) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   327
by (subgoal_tac "~ k*na < k*n" 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   328
by (asm_simp_tac
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   329
     (simpset() addsimps [zero_less_mult_iff, div_geq,
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   330
                         diff_mult_distrib2 RS sym, diff_less]) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   331
by (asm_full_simp_tac (simpset() addsimps [not_less_iff_le, 
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   332
                                          le_refl RS mult_le_mono]) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   333
qed "div_cancel";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   334
Addsimps [div_cancel];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   335
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   336
Goal "!!k. [| 0<n; 0<k |] ==> (k*m) mod (k*n) = k * (m mod n)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   337
by (res_inst_tac [("n","m")] less_induct 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   338
by (case_tac "na<n" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   339
by (asm_simp_tac (simpset() addsimps [mod_less, zero_less_mult_iff, 
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   340
                                     mult_less_mono2]) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   341
by (subgoal_tac "~ k*na < k*n" 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   342
by (asm_simp_tac
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   343
     (simpset() addsimps [zero_less_mult_iff, mod_geq,
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   344
                         diff_mult_distrib2 RS sym, diff_less]) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   345
by (asm_full_simp_tac (simpset() addsimps [not_less_iff_le, 
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   346
                                          le_refl RS mult_le_mono]) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   347
qed "mult_mod_distrib";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   348
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   349
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   350
(************************************************)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   351
(** Divides Relation                           **)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   352
(************************************************)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   353
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   354
Goalw [dvd_def] "m dvd 0";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   355
by (blast_tac (claset() addIs [mult_0_right RS sym]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   356
qed "dvd_0_right";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   357
Addsimps [dvd_0_right];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   358
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   359
Goalw [dvd_def] "!!m. 0 dvd m ==> m = 0";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   360
by (fast_tac (claset() addss simpset()) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   361
qed "dvd_0_left";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   362
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   363
Goalw [dvd_def] "1 dvd k";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   364
by (Simp_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   365
qed "dvd_1_left";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   366
AddIffs [dvd_1_left];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   367
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   368
Goalw [dvd_def] "m dvd m";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   369
by (blast_tac (claset() addIs [mult_1_right RS sym]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   370
qed "dvd_refl";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   371
Addsimps [dvd_refl];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   372
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   373
Goalw [dvd_def] "!!m n p. [| m dvd n; n dvd p |] ==> m dvd p";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   374
by (blast_tac (claset() addIs [mult_assoc] ) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   375
qed "dvd_trans";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   376
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   377
Goalw [dvd_def] "!!m n. [| m dvd n; n dvd m |] ==> m=n";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   378
by (fast_tac (claset() addDs [mult_eq_self_implies_10]
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   379
                     addss (simpset() addsimps [mult_assoc, mult_eq_1_iff])) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   380
qed "dvd_anti_sym";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   381
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   382
Goalw [dvd_def] "!!k. [| k dvd m; k dvd n |] ==> k dvd (m + n)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   383
by (blast_tac (claset() addIs [add_mult_distrib2 RS sym]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   384
qed "dvd_add";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   385
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   386
Goalw [dvd_def] "!!k. [| k dvd m; k dvd n |] ==> k dvd (m-n)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   387
by (blast_tac (claset() addIs [diff_mult_distrib2 RS sym]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   388
qed "dvd_diff";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   389
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   390
Goal "!!k. [| k dvd (m-n); k dvd n; n<=m |] ==> k dvd m";
3457
a8ab7c64817c Ran expandshort
paulson
parents: 3427
diff changeset
   391
by (etac (not_less_iff_le RS iffD2 RS add_diff_inverse RS subst) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   392
by (blast_tac (claset() addIs [dvd_add]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   393
qed "dvd_diffD";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   394
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   395
Goalw [dvd_def] "!!k. k dvd n ==> k dvd (m*n)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   396
by (blast_tac (claset() addIs [mult_left_commute]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   397
qed "dvd_mult";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   398
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   399
Goal "!!k. k dvd m ==> k dvd (m*n)";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   400
by (stac mult_commute 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   401
by (etac dvd_mult 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   402
qed "dvd_mult2";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   403
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   404
(* k dvd (m*k) *)
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   405
AddIffs [dvd_refl RS dvd_mult, dvd_refl RS dvd_mult2];
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   406
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   407
Goalw [dvd_def] "!!m. [| f dvd m; f dvd n; 0<n |] ==> f dvd (m mod n)";
3718
d78cf498a88c Minor tidying to use Clarify_tac, etc.
paulson
parents: 3496
diff changeset
   408
by (Clarify_tac 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   409
by (full_simp_tac (simpset() addsimps [zero_less_mult_iff]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   410
by (res_inst_tac 
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   411
    [("x", "(((k div ka)*ka + k mod ka) - ((f*k) div (f*ka)) * ka)")] 
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   412
    exI 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   413
by (asm_simp_tac (simpset() addsimps [diff_mult_distrib2, 
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   414
                                     mult_mod_distrib, add_mult_distrib2]) 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   415
qed "dvd_mod";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   416
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   417
Goal "!!k. [| k dvd (m mod n); k dvd n; 0<n |] ==> k dvd m";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   418
by (subgoal_tac "k dvd ((m div n)*n + m mod n)" 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   419
by (asm_simp_tac (simpset() addsimps [dvd_add, dvd_mult]) 2);
4356
0dfd34f0d33d Replaced n ~= 0 by 0 < n
nipkow
parents: 4089
diff changeset
   420
by (asm_full_simp_tac (simpset() addsimps [mod_div_equality]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   421
qed "dvd_mod_imp_dvd";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   422
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   423
Goalw [dvd_def]  "!!k m n. [| (k*m) dvd (k*n); 0<k |] ==> m dvd n";
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   424
by (etac exE 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   425
by (asm_full_simp_tac (simpset() addsimps mult_ac) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   426
by (Blast_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   427
qed "dvd_mult_cancel";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   428
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   429
Goalw [dvd_def] "!!i j. [| i dvd m; j dvd n|] ==> (i*j) dvd (m*n)";
3718
d78cf498a88c Minor tidying to use Clarify_tac, etc.
paulson
parents: 3496
diff changeset
   430
by (Clarify_tac 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   431
by (res_inst_tac [("x","k*ka")] exI 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   432
by (asm_simp_tac (simpset() addsimps mult_ac) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   433
qed "mult_dvd_mono";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   434
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   435
Goalw [dvd_def] "!!c. (i*j) dvd k ==> i dvd k";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   436
by (full_simp_tac (simpset() addsimps [mult_assoc]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   437
by (Blast_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   438
qed "dvd_mult_left";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   439
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   440
Goalw [dvd_def] "!!n. [| k dvd n; 0 < n |] ==> k <= n";
3718
d78cf498a88c Minor tidying to use Clarify_tac, etc.
paulson
parents: 3496
diff changeset
   441
by (Clarify_tac 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   442
by (ALLGOALS (full_simp_tac (simpset() addsimps [zero_less_mult_iff])));
3457
a8ab7c64817c Ran expandshort
paulson
parents: 3427
diff changeset
   443
by (etac conjE 1);
a8ab7c64817c Ran expandshort
paulson
parents: 3427
diff changeset
   444
by (rtac le_trans 1);
a8ab7c64817c Ran expandshort
paulson
parents: 3427
diff changeset
   445
by (rtac (le_refl RS mult_le_mono) 2);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   446
by (etac Suc_leI 2);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   447
by (Simp_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   448
qed "dvd_imp_le";
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   449
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4811
diff changeset
   450
Goalw [dvd_def] "!!k. 0<k ==> (k dvd n) = (n mod k = 0)";
3724
f33e301a89f5 Step_tac -> Safe_tac
paulson
parents: 3718
diff changeset
   451
by Safe_tac;
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   452
by (stac mult_commute 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   453
by (Asm_simp_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   454
by (eres_inst_tac [("t","n")] (mod_div_equality RS subst) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4059
diff changeset
   455
by (asm_simp_tac (simpset() addsimps [mult_commute]) 1);
3366
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   456
by (Blast_tac 1);
2402c6ab1561 Moving div and mod from Arith to Divides
paulson
parents:
diff changeset
   457
qed "dvd_eq_mod_eq_0";