src/HOL/ex/Primrec.thy
author nipkow
Sun, 13 May 2007 07:11:21 +0200
changeset 22944 1d471b8dec4e
parent 22283 26140713540b
child 23776 2215169c93fa
permissions -rw-r--r--
Got rid of listsp
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
     1
(*  Title:      HOL/ex/Primrec.thy
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
     2
    ID:         $Id$
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
     4
    Copyright   1997  University of Cambridge
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
     5
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
     6
Primitive Recursive Functions.  Demonstrates recursive definitions,
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
     7
the TFL package.
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
     8
*)
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
     9
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    10
header {* Primitive Recursive Functions *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    11
16417
9bc16273c2d4 migrated theory headers to new format
haftmann
parents: 11704
diff changeset
    12
theory Primrec imports Main begin
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    13
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    14
text {*
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    15
  Proof adopted from
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    16
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    17
  Nora Szasz, A Machine Checked Proof that Ackermann's Function is not
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    18
  Primitive Recursive, In: Huet \& Plotkin, eds., Logical Environments
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    19
  (CUP, 1993), 317-338.
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    20
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    21
  See also E. Mendelson, Introduction to Mathematical Logic.  (Van
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    22
  Nostrand, 1964), page 250, exercise 11.
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    23
  \medskip
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    24
*}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    25
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    26
consts ack :: "nat * nat => nat"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    27
recdef ack  "less_than <*lex*> less_than"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    28
  "ack (0, n) =  Suc n"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    29
  "ack (Suc m, 0) = ack (m, 1)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    30
  "ack (Suc m, Suc n) = ack (m, ack (Suc m, n))"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    31
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    32
consts list_add :: "nat list => nat"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    33
primrec
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    34
  "list_add [] = 0"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    35
  "list_add (m # ms) = m + list_add ms"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    36
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    37
consts zeroHd :: "nat list => nat"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    38
primrec
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    39
  "zeroHd [] = 0"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    40
  "zeroHd (m # ms) = m"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    41
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    42
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    43
text {* The set of primitive recursive functions of type @{typ "nat list => nat"}. *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    44
19736
wenzelm
parents: 19676
diff changeset
    45
definition
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    46
  SC :: "nat list => nat" where
19736
wenzelm
parents: 19676
diff changeset
    47
  "SC l = Suc (zeroHd l)"
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
    48
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    49
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    50
  CONSTANT :: "nat => nat list => nat" where
19736
wenzelm
parents: 19676
diff changeset
    51
  "CONSTANT k l = k"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    52
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    53
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    54
  PROJ :: "nat => nat list => nat" where
19736
wenzelm
parents: 19676
diff changeset
    55
  "PROJ i l = zeroHd (drop i l)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    56
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    57
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    58
  COMP :: "(nat list => nat) => (nat list => nat) list => nat list => nat" where
19736
wenzelm
parents: 19676
diff changeset
    59
  "COMP g fs l = g (map (\<lambda>f. f l) fs)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    60
21404
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    61
definition
eb85850d3eb7 more robust syntax for definition/abbreviation/notation;
wenzelm
parents: 19736
diff changeset
    62
  PREC :: "(nat list => nat) => (nat list => nat) => nat list => nat" where
19736
wenzelm
parents: 19676
diff changeset
    63
  "PREC f g l =
wenzelm
parents: 19676
diff changeset
    64
    (case l of
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    65
      [] => 0
19736
wenzelm
parents: 19676
diff changeset
    66
    | x # l' => nat_rec (f l') (\<lambda>y r. g (r # y # l')) x)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    67
  -- {* Note that @{term g} is applied first to @{term "PREC f g y"} and then to @{term y}! *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    68
22283
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
    69
inductive2 PRIMREC :: "(nat list => nat) => bool"
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
    70
  where
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
    71
    SC: "PRIMREC SC"
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
    72
  | CONSTANT: "PRIMREC (CONSTANT k)"
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
    73
  | PROJ: "PRIMREC (PROJ i)"
22944
1d471b8dec4e Got rid of listsp
nipkow
parents: 22283
diff changeset
    74
  | COMP: "PRIMREC g ==> \<forall>f \<in> set fs. PRIMREC f ==> PRIMREC (COMP g fs)"
22283
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
    75
  | PREC: "PRIMREC f ==> PRIMREC g ==> PRIMREC (PREC f g)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    76
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    77
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    78
text {* Useful special cases of evaluation *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    79
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    80
lemma SC [simp]: "SC (x # l) = Suc x"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    81
  apply (simp add: SC_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    82
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    83
19676
187234ec6050 renamed CONST to CONSTANT;
wenzelm
parents: 16731
diff changeset
    84
lemma CONSTANT [simp]: "CONSTANT k l = k"
187234ec6050 renamed CONST to CONSTANT;
wenzelm
parents: 16731
diff changeset
    85
  apply (simp add: CONSTANT_def)
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    86
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    87
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    88
lemma PROJ_0 [simp]: "PROJ 0 (x # l) = x"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    89
  apply (simp add: PROJ_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    90
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    91
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    92
lemma COMP_1 [simp]: "COMP g [f] l = g [f l]"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    93
  apply (simp add: COMP_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    94
  done
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
    95
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    96
lemma PREC_0 [simp]: "PREC f g (0 # l) = f l"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    97
  apply (simp add: PREC_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    98
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
    99
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   100
lemma PREC_Suc [simp]: "PREC f g (Suc x # l) = g (PREC f g (x # l) # x # l)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   101
  apply (simp add: PREC_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   102
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   103
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   104
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   105
text {* PROPERTY A 4 *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   106
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   107
lemma less_ack2 [iff]: "j < ack (i, j)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   108
  apply (induct i j rule: ack.induct)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   109
    apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   110
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   111
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   112
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   113
text {* PROPERTY A 5-, the single-step lemma *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   114
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   115
lemma ack_less_ack_Suc2 [iff]: "ack(i, j) < ack (i, Suc j)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   116
  apply (induct i j rule: ack.induct)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   117
    apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   118
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   119
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   120
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   121
text {* PROPERTY A 5, monotonicity for @{text "<"} *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   122
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   123
lemma ack_less_mono2: "j < k ==> ack (i, j) < ack (i, k)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   124
  apply (induct i k rule: ack.induct)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   125
    apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   126
  apply (blast elim!: less_SucE intro: less_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   127
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   128
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   129
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   130
text {* PROPERTY A 5', monotonicity for @{text \<le>} *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   131
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   132
lemma ack_le_mono2: "j \<le> k ==> ack (i, j) \<le> ack (i, k)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   133
  apply (simp add: order_le_less)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   134
  apply (blast intro: ack_less_mono2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   135
  done
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   136
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   137
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   138
text {* PROPERTY A 6 *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   139
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   140
lemma ack2_le_ack1 [iff]: "ack (i, Suc j) \<le> ack (Suc i, j)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   141
  apply (induct j)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   142
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   143
  apply (blast intro: ack_le_mono2 less_ack2 [THEN Suc_leI] le_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   144
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   145
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   146
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   147
text {* PROPERTY A 7-, the single-step lemma *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   148
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   149
lemma ack_less_ack_Suc1 [iff]: "ack (i, j) < ack (Suc i, j)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   150
  apply (blast intro: ack_less_mono2 less_le_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   151
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   152
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   153
19676
187234ec6050 renamed CONST to CONSTANT;
wenzelm
parents: 16731
diff changeset
   154
text {* PROPERTY A 4'? Extra lemma needed for @{term CONSTANT} case, constant functions *}
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   155
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   156
lemma less_ack1 [iff]: "i < ack (i, j)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   157
  apply (induct i)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   158
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   159
  apply (blast intro: Suc_leI le_less_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   160
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   161
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   162
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   163
text {* PROPERTY A 8 *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   164
11704
3c50a2cd6f00 * sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm
parents: 11701
diff changeset
   165
lemma ack_1 [simp]: "ack (Suc 0, j) = j + 2"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   166
  apply (induct j)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   167
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   168
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   169
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   170
11701
3d51fbf81c17 sane numerals (stage 1): added generic 1, removed 1' and 2 on nat,
wenzelm
parents: 11464
diff changeset
   171
text {* PROPERTY A 9.  The unary @{text 1} and @{text 2} in @{term
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   172
  ack} is essential for the rewriting. *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   173
11704
3c50a2cd6f00 * sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm
parents: 11701
diff changeset
   174
lemma ack_2 [simp]: "ack (Suc (Suc 0), j) = 2 * j + 3"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   175
  apply (induct j)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   176
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   177
  done
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   178
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   179
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   180
text {* PROPERTY A 7, monotonicity for @{text "<"} [not clear why
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   181
  @{thm [source] ack_1} is now needed first!] *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   182
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   183
lemma ack_less_mono1_aux: "ack (i, k) < ack (Suc (i +i'), k)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   184
  apply (induct i k rule: ack.induct)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   185
    apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   186
   prefer 2
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   187
   apply (blast intro: less_trans ack_less_mono2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   188
  apply (induct_tac i' n rule: ack.induct)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   189
    apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   190
  apply (blast intro: Suc_leI [THEN le_less_trans] ack_less_mono2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   191
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   192
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   193
lemma ack_less_mono1: "i < j ==> ack (i, k) < ack (j, k)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   194
  apply (drule less_imp_Suc_add)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   195
  apply (blast intro!: ack_less_mono1_aux)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   196
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   197
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   198
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   199
text {* PROPERTY A 7', monotonicity for @{text "\<le>"} *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   200
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   201
lemma ack_le_mono1: "i \<le> j ==> ack (i, k) \<le> ack (j, k)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   202
  apply (simp add: order_le_less)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   203
  apply (blast intro: ack_less_mono1)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   204
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   205
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   206
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   207
text {* PROPERTY A 10 *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   208
11704
3c50a2cd6f00 * sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm
parents: 11701
diff changeset
   209
lemma ack_nest_bound: "ack(i1, ack (i2, j)) < ack (2 + (i1 + i2), j)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   210
  apply (simp add: numerals)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   211
  apply (rule ack2_le_ack1 [THEN [2] less_le_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   212
  apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   213
  apply (rule le_add1 [THEN ack_le_mono1, THEN le_less_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   214
  apply (rule ack_less_mono1 [THEN ack_less_mono2])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   215
  apply (simp add: le_imp_less_Suc le_add2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   216
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   217
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   218
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   219
text {* PROPERTY A 11 *}
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   220
11704
3c50a2cd6f00 * sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm
parents: 11701
diff changeset
   221
lemma ack_add_bound: "ack (i1, j) + ack (i2, j) < ack (4 + (i1 + i2), j)"
11701
3d51fbf81c17 sane numerals (stage 1): added generic 1, removed 1' and 2 on nat,
wenzelm
parents: 11464
diff changeset
   222
  apply (rule_tac j = "ack (Suc (Suc 0), ack (i1 + i2, j))" in less_trans)
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   223
   prefer 2
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   224
   apply (rule ack_nest_bound [THEN less_le_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   225
   apply (simp add: Suc3_eq_add_3)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   226
  apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   227
  apply (cut_tac i = i1 and m1 = i2 and k = j in le_add1 [THEN ack_le_mono1])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   228
  apply (cut_tac i = "i2" and m1 = i1 and k = j in le_add2 [THEN ack_le_mono1])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   229
  apply auto
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   230
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   231
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   232
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   233
text {* PROPERTY A 12.  Article uses existential quantifier but the ALF proof
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   234
  used @{text "k + 4"}.  Quantified version must be nested @{text
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   235
  "\<exists>k'. \<forall>i j. ..."} *}
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   236
11704
3c50a2cd6f00 * sane numerals (stage 2): plain "num" syntax (removed "#");
wenzelm
parents: 11701
diff changeset
   237
lemma ack_add_bound2: "i < ack (k, j) ==> i + j < ack (4 + k, j)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   238
  apply (rule_tac j = "ack (k, j) + ack (0, j)" in less_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   239
   prefer 2
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   240
   apply (rule ack_add_bound [THEN less_le_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   241
   apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   242
  apply (rule add_less_mono less_ack2 | assumption)+
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   243
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   244
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   245
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   246
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   247
text {* Inductive definition of the @{term PR} functions *}
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   248
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   249
text {* MAIN RESULT *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   250
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   251
lemma SC_case: "SC l < ack (1, list_add l)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   252
  apply (unfold SC_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   253
  apply (induct l)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   254
  apply (simp_all add: le_add1 le_imp_less_Suc)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   255
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   256
19676
187234ec6050 renamed CONST to CONSTANT;
wenzelm
parents: 16731
diff changeset
   257
lemma CONSTANT_case: "CONSTANT k l < ack (k, list_add l)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   258
  apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   259
  done
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   260
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   261
lemma PROJ_case [rule_format]: "\<forall>i. PROJ i l < ack (0, list_add l)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   262
  apply (simp add: PROJ_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   263
  apply (induct l)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   264
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   265
  apply (rule allI)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   266
  apply (case_tac i)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   267
  apply (simp (no_asm_simp) add: le_add1 le_imp_less_Suc)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   268
  apply (simp (no_asm_simp))
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   269
  apply (blast intro: less_le_trans intro!: le_add2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   270
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   271
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   272
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   273
text {* @{term COMP} case *}
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   274
22944
1d471b8dec4e Got rid of listsp
nipkow
parents: 22283
diff changeset
   275
lemma COMP_map_aux: "\<forall>f \<in> set fs. PRIMREC f \<and> (\<exists>kf. \<forall>l. f l < ack (kf, list_add l))
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   276
  ==> \<exists>k. \<forall>l. list_add (map (\<lambda>f. f l) fs) < ack (k, list_add l)"
22944
1d471b8dec4e Got rid of listsp
nipkow
parents: 22283
diff changeset
   277
  apply (induct fs)
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   278
  apply (rule_tac x = 0 in exI)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   279
   apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   280
  apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   281
  apply (blast intro: add_less_mono ack_add_bound less_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   282
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   283
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   284
lemma COMP_case:
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   285
  "\<forall>l. g l < ack (kg, list_add l) ==>
22944
1d471b8dec4e Got rid of listsp
nipkow
parents: 22283
diff changeset
   286
  \<forall>f \<in> set fs. PRIMREC f \<and> (\<exists>kf. \<forall>l. f l < ack(kf, list_add l))
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   287
  ==> \<exists>k. \<forall>l. COMP g fs  l < ack(k, list_add l)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   288
  apply (unfold COMP_def)
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   289
    --{*Now, if meson tolerated map, we could finish with
16731
124b4782944f fixed antiquotation;
wenzelm
parents: 16588
diff changeset
   290
  @{text "(drule COMP_map_aux, meson ack_less_mono2 ack_nest_bound less_trans)"} *}
16588
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   291
  apply (erule COMP_map_aux [THEN exE])
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   292
  apply (rule exI)
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   293
  apply (rule allI)
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   294
  apply (drule spec)+
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   295
  apply (erule less_trans)
8de758143786 stricter first-order check for meson
paulson
parents: 16563
diff changeset
   296
  apply (blast intro: ack_less_mono2 ack_nest_bound less_trans)
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   297
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   298
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   299
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   300
text {* @{term PREC} case *}
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   301
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   302
lemma PREC_case_aux:
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   303
  "\<forall>l. f l + list_add l < ack (kf, list_add l) ==>
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   304
    \<forall>l. g l + list_add l < ack (kg, list_add l) ==>
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   305
    PREC f g l + list_add l < ack (Suc (kf + kg), list_add l)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   306
  apply (unfold PREC_def)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   307
  apply (case_tac l)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   308
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   309
   apply (blast intro: less_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   310
  apply (erule ssubst) -- {* get rid of the needless assumption *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   311
  apply (induct_tac a)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   312
   apply simp_all
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   313
   txt {* base case *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   314
   apply (blast intro: le_add1 [THEN le_imp_less_Suc, THEN ack_less_mono1] less_trans)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   315
  txt {* induction step *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   316
  apply (rule Suc_leI [THEN le_less_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   317
   apply (rule le_refl [THEN add_le_mono, THEN le_less_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   318
    prefer 2
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   319
    apply (erule spec)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   320
   apply (simp add: le_add2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   321
  txt {* final part of the simplification *}
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   322
  apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   323
  apply (rule le_add2 [THEN ack_le_mono1, THEN le_less_trans])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   324
  apply (erule ack_less_mono2)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   325
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   326
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   327
lemma PREC_case:
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   328
  "\<forall>l. f l < ack (kf, list_add l) ==>
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   329
    \<forall>l. g l < ack (kg, list_add l) ==>
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   330
    \<exists>k. \<forall>l. PREC f g l < ack (k, list_add l)"
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   331
  apply (rule exI)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   332
  apply (rule allI)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   333
  apply (rule le_less_trans [OF le_add1 PREC_case_aux])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   334
   apply (blast intro: ack_add_bound2)+
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   335
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   336
22283
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
   337
lemma ack_bounds_PRIMREC: "PRIMREC f ==> \<exists>k. \<forall>l. f l < ack (k, list_add l)"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   338
  apply (erule PRIMREC.induct)
19676
187234ec6050 renamed CONST to CONSTANT;
wenzelm
parents: 16731
diff changeset
   339
      apply (blast intro: SC_case CONSTANT_case PROJ_case COMP_case PREC_case)+
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   340
  done
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   341
22283
26140713540b Adapted to new inductive definition package.
berghofe
parents: 21404
diff changeset
   342
lemma ack_not_PRIMREC: "\<not> PRIMREC (\<lambda>l. case l of [] => 0 | x # l' => ack (x, x))"
11024
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   343
  apply (rule notI)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   344
  apply (erule ack_bounds_PRIMREC [THEN exE])
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   345
  apply (rule less_irrefl)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   346
  apply (drule_tac x = "[x]" in spec)
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   347
  apply simp
23bf8d787b04 converted to new-style theories;
wenzelm
parents: 8703
diff changeset
   348
  done
3335
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   349
b0139b83a5ee New example ported from ZF
paulson
parents:
diff changeset
   350
end