src/ZF/ex/Primrec.ML
author paulson
Wed, 13 Jan 1999 11:57:09 +0100
changeset 6112 5e4871c5136b
parent 6071 1b2392ac5752
child 6153 bff90585cce5
permissions -rw-r--r--
datatype package improvements
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
     1
(*  Title:      ZF/ex/Primrec
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     2
    ID:         $Id$
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     4
    Copyright   1994  University of Cambridge
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     5
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     6
Primitive Recursive Functions
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     7
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     8
Proof adopted from
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
     9
Nora Szasz, 
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    10
A Machine Checked Proof that Ackermann's Function is not Primitive Recursive,
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    11
In: Huet & Plotkin, eds., Logical Environments (CUP, 1993), 317-338.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    12
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    13
See also E. Mendelson, Introduction to Mathematical Logic.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    14
(Van Nostrand, 1964), page 250, exercise 11.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    15
*)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    16
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    17
(*** Inductive definition of the PR functions ***)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    18
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    19
(* c: prim_rec ==> c: list(nat) -> nat *)
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    20
val prim_rec_into_fun = prim_rec.dom_subset RS subsetD;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    21
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    22
simpset_ref() := simpset() setSolver (type_auto_tac ([prim_rec_into_fun] @ 
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    23
					      pr_typechecks @ prim_rec.intrs));
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    24
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    25
Goal "i:nat ==> ACK(i): prim_rec";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
    26
by (induct_tac "i" 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
    27
by (ALLGOALS Asm_simp_tac);
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    28
qed "ACK_in_prim_rec";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    29
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    30
val ack_typechecks =
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    31
    [ACK_in_prim_rec, prim_rec_into_fun RS apply_type,
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    32
     add_type, list_add_type, nat_into_Ord] @ 
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
    33
    nat_typechecks @ list.intrs @ prim_rec.intrs;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    34
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    35
simpset_ref() := simpset() setSolver (type_auto_tac ack_typechecks);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    36
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
    37
Goal "[| i:nat;  j:nat |] ==>  ack(i,j): nat";
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    38
by Auto_tac;
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
    39
qed "ack_type";
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    40
Addsimps [ack_type];
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    41
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    42
(** Ackermann's function cases **)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    43
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    44
(*PROPERTY A 1*)
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    45
Goal "j:nat ==> ack(0,j) = succ(j)";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
    46
by (asm_simp_tac (simpset() addsimps [SC]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    47
qed "ack_0";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    48
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    49
(*PROPERTY A 2*)
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    50
Goal "ack(succ(i), 0) = ack(i,1)";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
    51
by (asm_simp_tac (simpset() addsimps [CONST,PREC_0]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    52
qed "ack_succ_0";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    53
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    54
(*PROPERTY A 3*)
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    55
Goal "[| i:nat;  j:nat |]  \
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    56
\     ==> ack(succ(i), succ(j)) = ack(i, ack(succ(i), j))";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
    57
by (asm_simp_tac (simpset() addsimps [CONST,PREC_succ,COMP_1,PROJ_0]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    58
qed "ack_succ_succ";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    59
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
    60
Addsimps [ack_0, ack_succ_0, ack_succ_succ, ack_type, nat_into_Ord];
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    61
Delsimps [ACK_0, ACK_succ];
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    62
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    63
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    64
(*PROPERTY A 4*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
    65
Goal "i:nat ==> ALL j:nat. j < ack(i,j)";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
    66
by (induct_tac "i" 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
    67
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    68
by (rtac ballI 1);
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
    69
by (induct_tac "j" 1);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    70
by (etac (succ_leI RS lt_trans1) 2);
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    71
by (rtac (nat_0I RS nat_0_le RS lt_trans) 1);
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
    72
by Auto_tac;
6112
5e4871c5136b datatype package improvements
paulson
parents: 6071
diff changeset
    73
qed_spec_mp "lt_ack2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    74
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    75
(*PROPERTY A 5-, the single-step lemma*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
    76
Goal "[| i:nat; j:nat |] ==> ack(i,j) < ack(i, succ(j))";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
    77
by (induct_tac "i" 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
    78
by (ALLGOALS (asm_simp_tac (simpset() addsimps [lt_ack2])));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    79
qed "ack_lt_ack_succ2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    80
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    81
(*PROPERTY A 5, monotonicity for < *)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
    82
Goal "[| j<k; i:nat; k:nat |] ==> ack(i,j) < ack(i,k)";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    83
by (forward_tac [lt_nat_in_nat] 1 THEN assume_tac 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    84
by (etac succ_lt_induct 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    85
by (assume_tac 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    86
by (rtac lt_trans 2);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    87
by (REPEAT (ares_tac ([ack_lt_ack_succ2, ack_type] @ pr_typechecks) 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
    88
qed "ack_lt_mono2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    89
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    90
(*PROPERTY A 5', monotonicity for le *)
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
    91
Goal "[| j le k;  i: nat;  k:nat |] ==> ack(i,j) le ack(i,k)";
3840
e0baea4d485a fixed dots;
wenzelm
parents: 3328
diff changeset
    92
by (res_inst_tac [("f", "%j. ack(i,j)")] Ord_lt_mono_imp_le_mono 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    93
by (REPEAT (ares_tac [ack_lt_mono2, ack_type RS nat_into_Ord] 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    94
qed "ack_le_mono2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    95
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
    96
(*PROPERTY A 6*)
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
    97
Goal "[| i:nat;  j:nat |] ==> ack(i, succ(j)) le ack(succ(i), j)";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
    98
by (induct_tac "j" 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
    99
by (ALLGOALS Asm_simp_tac);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   100
by (rtac ack_le_mono2 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   101
by (rtac (lt_ack2 RS succ_leI RS le_trans) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   102
by (REPEAT (ares_tac (ack_typechecks) 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   103
qed "ack2_le_ack1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   104
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   105
(*PROPERTY A 7-, the single-step lemma*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
   106
Goal "[| i:nat; j:nat |] ==> ack(i,j) < ack(succ(i),j)";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   107
by (rtac (ack_lt_mono2 RS lt_trans2) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   108
by (rtac ack2_le_ack1 4);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   109
by (REPEAT (ares_tac ([nat_le_refl, ack_type] @ pr_typechecks) 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   110
qed "ack_lt_ack_succ1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   111
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   112
(*PROPERTY A 7, monotonicity for < *)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
   113
Goal "[| i<j; j:nat; k:nat |] ==> ack(i,k) < ack(j,k)";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   114
by (forward_tac [lt_nat_in_nat] 1 THEN assume_tac 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   115
by (etac succ_lt_induct 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   116
by (assume_tac 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   117
by (rtac lt_trans 2);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   118
by (REPEAT (ares_tac ([ack_lt_ack_succ1, ack_type] @ pr_typechecks) 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   119
qed "ack_lt_mono1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   120
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   121
(*PROPERTY A 7', monotonicity for le *)
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   122
Goal "[| i le j; j:nat; k:nat |] ==> ack(i,k) le ack(j,k)";
3840
e0baea4d485a fixed dots;
wenzelm
parents: 3328
diff changeset
   123
by (res_inst_tac [("f", "%j. ack(j,k)")] Ord_lt_mono_imp_le_mono 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   124
by (REPEAT (ares_tac [ack_lt_mono1, ack_type RS nat_into_Ord] 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   125
qed "ack_le_mono1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   126
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   127
(*PROPERTY A 8*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
   128
Goal "j:nat ==> ack(1,j) = succ(succ(j))";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
   129
by (induct_tac "j" 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   130
by (ALLGOALS Asm_simp_tac);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   131
qed "ack_1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   132
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   133
(*PROPERTY A 9*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
   134
Goal "j:nat ==> ack(succ(1),j) = succ(succ(succ(j#+j)))";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
   135
by (induct_tac "j" 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   136
by (ALLGOALS (asm_simp_tac (simpset() addsimps [ack_1, add_succ_right])));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   137
qed "ack_2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   138
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   139
(*PROPERTY A 10*)
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   140
Goal "[| i1:nat; i2:nat; j:nat |] ==> \
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   141
\               ack(i1, ack(i2,j)) < ack(succ(succ(i1#+i2)), j)";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   142
by (rtac (ack2_le_ack1 RSN (2,lt_trans2)) 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   143
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   144
by (rtac (add_le_self RS ack_le_mono1 RS lt_trans1) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   145
by (rtac (add_le_self2 RS ack_lt_mono1 RS ack_lt_mono2) 5);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   146
by Auto_tac;
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   147
qed "ack_nest_bound";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   148
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   149
(*PROPERTY A 11*)
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   150
Goal "[| i1:nat; i2:nat; j:nat |] ==> \
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   151
\          ack(i1,j) #+ ack(i2,j) < ack(succ(succ(succ(succ(i1#+i2)))), j)";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   152
by (res_inst_tac [("j", "ack(succ(1), ack(i1 #+ i2, j))")] lt_trans 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   153
by (asm_simp_tac (simpset() addsimps [ack_2]) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   154
by (rtac (ack_nest_bound RS lt_trans2) 2);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   155
by (Asm_simp_tac 5);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   156
by (rtac (add_le_mono RS leI RS leI) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   157
by (REPEAT (ares_tac ([add_le_self, add_le_self2, ack_le_mono1] @
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   158
                      ack_typechecks) 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   159
qed "ack_add_bound";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   160
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   161
(*PROPERTY A 12.  Article uses existential quantifier but the ALF proof
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   162
  used k#+4.  Quantified version must be nested EX k'. ALL i,j... *)
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   163
Goal "[| i < ack(k,j);  j:nat;  k:nat |] ==> \
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   164
\             i#+j < ack(succ(succ(succ(succ(k)))), j)";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   165
by (res_inst_tac [("j", "ack(k,j) #+ ack(0,j)")] lt_trans 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   166
by (rtac (ack_add_bound RS lt_trans2) 2);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   167
by (asm_simp_tac (simpset() addsimps [add_0_right]) 5);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   168
by (REPEAT (ares_tac ([add_lt_mono, lt_ack2] @ ack_typechecks) 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   169
qed "ack_add_bound2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   170
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   171
(*** MAIN RESULT ***)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   172
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   173
Addsimps [list_add_type, nat_into_Ord];
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   174
6065
3b4a29166f26 induct_tac and exhaust_tac
paulson
parents: 6044
diff changeset
   175
Goalw [SC_def] "l: list(nat) ==> SC ` l < ack(1, list_add(l))";
3b4a29166f26 induct_tac and exhaust_tac
paulson
parents: 6044
diff changeset
   176
by (exhaust_tac "l" 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   177
by (asm_simp_tac (simpset() addsimps [succ_iff]) 1);
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   178
by (asm_simp_tac (simpset() addsimps [ack_1, add_le_self]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   179
qed "SC_case";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   180
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   181
(*PROPERTY A 4'? Extra lemma needed for CONST case, constant functions*)
5137
60205b0de9b9 Huge tidy-up: removal of leading \!\!
paulson
parents: 5068
diff changeset
   182
Goal "[| i:nat; j:nat |] ==> i < ack(i,j)";
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
   183
by (induct_tac "i" 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   184
by (asm_simp_tac (simpset() addsimps [nat_0_le]) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   185
by (etac ([succ_leI, ack_lt_ack_succ1] MRS lt_trans1) 1);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   186
by Auto_tac;
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   187
qed "lt_ack1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   188
5068
fb28eaa07e01 isatool fixgoal;
wenzelm
parents: 4152
diff changeset
   189
Goalw [CONST_def]
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   190
    "[| l: list(nat);  k: nat |] ==> CONST(k) ` l < ack(k, list_add(l))";
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   191
by (asm_simp_tac (simpset() addsimps [lt_ack1]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   192
qed "CONST_case";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   193
5068
fb28eaa07e01 isatool fixgoal;
wenzelm
parents: 4152
diff changeset
   194
Goalw [PROJ_def]
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   195
    "l: list(nat) ==> ALL i:nat. PROJ(i) ` l < ack(0, list_add(l))";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   196
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   197
by (etac list.induct 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   198
by (asm_simp_tac (simpset() addsimps [nat_0_le]) 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   199
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   200
by (rtac ballI 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   201
by (eres_inst_tac [("n","x")] natE 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   202
by (asm_simp_tac (simpset() addsimps [add_le_self]) 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   203
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   204
by (etac (bspec RS lt_trans2) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   205
by (rtac (add_le_self2 RS succ_leI) 2);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   206
by Auto_tac;
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   207
qed "PROJ_case_lemma";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   208
val PROJ_case = PROJ_case_lemma RS bspec;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   209
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   210
(** COMP case **)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   211
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   212
Goal "fs : list({f: prim_rec .                                 \
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   213
\                  EX kf:nat. ALL l:list(nat).                  \
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   214
\                             f`l < ack(kf, list_add(l))})      \
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   215
\      ==> EX k:nat. ALL l: list(nat).                          \
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   216
\                list_add(map(%f. f ` l, fs)) < ack(k, list_add(l))";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   217
by (etac list.induct 1);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   218
by (res_inst_tac [("x","0")] bexI 1);
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   219
by (asm_simp_tac (simpset() addsimps [lt_ack1, nat_0_le]) 1);
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   220
by Auto_tac;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   221
by (rtac (ballI RS bexI) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   222
by (rtac (add_lt_mono RS lt_trans) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   223
by (REPEAT (FIRSTGOAL (etac bspec)));
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   224
by (rtac ack_add_bound 5);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   225
by Auto_tac;
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   226
qed "COMP_map_lemma";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   227
5068
fb28eaa07e01 isatool fixgoal;
wenzelm
parents: 4152
diff changeset
   228
Goalw [COMP_def]
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   229
 "[| kg: nat;                                 \
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   230
\         ALL l:list(nat). g`l < ack(kg, list_add(l));          \
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   231
\         fs : list({f: prim_rec .                               \
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   232
\                    EX kf:nat. ALL l:list(nat).                \
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   233
\                       f`l < ack(kf, list_add(l))})            \
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   234
\      |] ==> EX k:nat. ALL l: list(nat). COMP(g,fs)`l < ack(k, list_add(l))";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   235
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   236
by (forward_tac [list_CollectD] 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   237
by (etac (COMP_map_lemma RS bexE) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   238
by (rtac (ballI RS bexI) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   239
by (etac (bspec RS lt_trans) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   240
by (rtac lt_trans 2);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   241
by (rtac ack_nest_bound 3);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   242
by (etac (bspec RS ack_lt_mono2) 2);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   243
by Auto_tac;
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   244
qed "COMP_case";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   245
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   246
(** PREC case **)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   247
5068
fb28eaa07e01 isatool fixgoal;
wenzelm
parents: 4152
diff changeset
   248
Goalw [PREC_def]
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   249
 "[| ALL l:list(nat). f`l #+ list_add(l) < ack(kf, list_add(l)); \
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   250
\           ALL l:list(nat). g`l #+ list_add(l) < ack(kg, list_add(l)); \
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   251
\           f: prim_rec;  kf: nat;                                       \
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   252
\           g: prim_rec;  kg: nat;                                       \
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   253
\           l: list(nat)                                                \
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   254
\        |] ==> PREC(f,g)`l #+ list_add(l) < ack(succ(kf#+kg), list_add(l))";
6065
3b4a29166f26 induct_tac and exhaust_tac
paulson
parents: 6044
diff changeset
   255
by (exhaust_tac "l" 1);
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   256
by (asm_simp_tac (simpset() addsimps [[nat_le_refl, lt_ack2] MRS lt_trans]) 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   257
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   258
by (etac ssubst 1);  (*get rid of the needless assumption*)
6070
032babd0120b ZF: the natural numbers as a datatype
paulson
parents: 6065
diff changeset
   259
by (induct_tac "a" 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   260
(*base case*)
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   261
by (EVERY1 [Asm_simp_tac, rtac lt_trans, etac bspec,
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   262
             assume_tac, rtac (add_le_self RS ack_lt_mono1),
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   263
             REPEAT o ares_tac (ack_typechecks)]);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   264
(*ind step*)
3328
480ad4e72662 Slight simplifications
paulson
parents: 2637
diff changeset
   265
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   266
by (rtac (succ_leI RS lt_trans1) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   267
by (res_inst_tac [("j", "g ` ?ll #+ ?mm")] lt_trans1 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   268
by (etac bspec 2);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   269
by (rtac (nat_le_refl RS add_le_mono) 1);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   270
	(*Auto_tac is a little slow*)
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   271
by (TRYALL (type_auto_tac ack_typechecks []));
4091
771b1f6422a8 isatool fixclasimp;
wenzelm
parents: 3840
diff changeset
   272
by (asm_simp_tac (simpset() addsimps [add_le_self2]) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   273
(*final part of the simplification*)
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   274
by (Asm_simp_tac 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   275
by (rtac (add_le_self2 RS ack_le_mono1 RS lt_trans1) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   276
by (etac ack_lt_mono2 5);
6071
1b2392ac5752 removal of DO_GOAL
paulson
parents: 6070
diff changeset
   277
by Auto_tac;
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   278
qed "PREC_case_lemma";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   279
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   280
Goal "[| f: prim_rec;  kf: nat;                               \
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   281
\        g: prim_rec;  kg: nat;                               \
5147
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   282
\        ALL l:list(nat). f`l < ack(kf, list_add(l));        \
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   283
\        ALL l:list(nat). g`l < ack(kg, list_add(l))         \
825877190618 More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5137
diff changeset
   284
\     |] ==> EX k:nat. ALL l: list(nat). PREC(f,g)`l< ack(k, list_add(l))";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   285
by (rtac (ballI RS bexI) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   286
by (rtac ([add_le_self, PREC_case_lemma] MRS lt_trans1) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   287
by (REPEAT
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   288
    (SOMEGOAL
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   289
     (FIRST' [test_assume_tac,
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   290
              match_tac (ack_typechecks),
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   291
              rtac (ack_add_bound2 RS ballI) THEN' etac bspec])));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   292
qed "PREC_case";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   293
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   294
Goal "f:prim_rec ==> EX k:nat. ALL l:list(nat). f`l < ack(k, list_add(l))";
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   295
by (etac prim_rec.induct 1);
4152
451104c223e2 Ran expandshort, especially to introduce Safe_tac
paulson
parents: 4091
diff changeset
   296
by Safe_tac;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   297
by (DEPTH_SOLVE
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   298
    (ares_tac ([SC_case, CONST_case, PROJ_case, COMP_case, PREC_case,
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   299
                       bexI, ballI] @ nat_typechecks) 1));
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   300
qed "ack_bounds_prim_rec";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   301
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   302
Goal "~ (lam l:list(nat). list_case(0, %x xs. ack(x,x), l)) : prim_rec";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   303
by (rtac notI 1);
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   304
by (etac (ack_bounds_prim_rec RS bexE) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   305
by (rtac lt_irrefl 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   306
by (dres_inst_tac [("x", "[x]")] bspec 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1461
diff changeset
   307
by (Asm_simp_tac 1);
6044
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   308
by (Asm_full_simp_tac 1);
e0f9d930e956 Needs separate theory Primrec_defs due to new inductive defs package
paulson
parents: 5268
diff changeset
   309
qed "ack_not_prim_rec";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents:
diff changeset
   310