author | wenzelm |
Wed, 13 Apr 2005 18:34:22 +0200 | |
changeset 15703 | 727ef1b8b3ee |
parent 15574 | b1d1b5bfc464 |
child 15705 | b5edb9dcec9a |
permissions | -rw-r--r-- |
12191 | 1 |
(* Title: ZF/Tools/inductive_package.ML |
6051 | 2 |
ID: $Id$ |
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1994 University of Cambridge |
|
5 |
||
6 |
Fixedpoint definition module -- for Inductive/Coinductive Definitions |
|
7 |
||
8 |
The functor will be instantiated for normal sums/products (inductive defs) |
|
9 |
and non-standard sums/products (coinductive defs) |
|
10 |
||
11 |
Sums are used only for mutual recursion; |
|
12 |
Products are used only to derive "streamlined" induction rules for relations |
|
13 |
*) |
|
14 |
||
15 |
type inductive_result = |
|
16 |
{defs : thm list, (*definitions made in thy*) |
|
17 |
bnd_mono : thm, (*monotonicity for the lfp definition*) |
|
18 |
dom_subset : thm, (*inclusion of recursive set in dom*) |
|
19 |
intrs : thm list, (*introduction rules*) |
|
20 |
elim : thm, (*case analysis theorem*) |
|
6141 | 21 |
mk_cases : string -> thm, (*generates case theorems*) |
6051 | 22 |
induct : thm, (*main induction rule*) |
23 |
mutual_induct : thm}; (*mutual induction rule*) |
|
24 |
||
25 |
||
26 |
(*Functor's result signature*) |
|
27 |
signature INDUCTIVE_PACKAGE = |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
28 |
sig |
6051 | 29 |
(*Insert definitions for the recursive sets, which |
30 |
must *already* be declared as constants in parent theory!*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
31 |
val add_inductive_i: bool -> term list * term -> |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
32 |
((bstring * term) * theory attribute list) list -> |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
33 |
thm list * thm list * thm list * thm list -> theory -> theory * inductive_result |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
34 |
val add_inductive_x: string list * string -> ((bstring * string) * theory attribute list) list |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
35 |
-> thm list * thm list * thm list * thm list -> theory -> theory * inductive_result |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
36 |
val add_inductive: string list * string -> |
15703 | 37 |
((bstring * string) * Attrib.src list) list -> |
38 |
(thmref * Attrib.src list) list * (thmref * Attrib.src list) list * |
|
39 |
(thmref * Attrib.src list) list * (thmref * Attrib.src list) list -> |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
40 |
theory -> theory * inductive_result |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
41 |
end; |
6051 | 42 |
|
43 |
||
44 |
(*Declares functions to add fixedpoint/constructor defs to a theory. |
|
45 |
Recursive sets must *already* be declared as constants.*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
46 |
functor Add_inductive_def_Fun |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
47 |
(structure Fp: FP and Pr : PR and CP: CARTPROD and Su : SU val coind: bool) |
6051 | 48 |
: INDUCTIVE_PACKAGE = |
49 |
struct |
|
12183 | 50 |
|
6051 | 51 |
open Logic Ind_Syntax; |
52 |
||
12227 | 53 |
val co_prefix = if coind then "co" else ""; |
54 |
||
7695 | 55 |
|
56 |
(* utils *) |
|
57 |
||
58 |
(*make distinct individual variables a1, a2, a3, ..., an. *) |
|
59 |
fun mk_frees a [] = [] |
|
12902 | 60 |
| mk_frees a (T::Ts) = Free(a,T) :: mk_frees (Symbol.bump_string a) Ts; |
7695 | 61 |
|
62 |
||
63 |
(* add_inductive(_i) *) |
|
64 |
||
6051 | 65 |
(*internal version, accepting terms*) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
66 |
fun add_inductive_i verbose (rec_tms, dom_sum) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
67 |
intr_specs (monos, con_defs, type_intrs, type_elims) thy = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
68 |
let |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
69 |
val _ = Theory.requires thy "Inductive" "(co)inductive definitions"; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
70 |
val sign = sign_of thy; |
6051 | 71 |
|
12191 | 72 |
val (intr_names, intr_tms) = split_list (map fst intr_specs); |
73 |
val case_names = RuleCases.case_names intr_names; |
|
6051 | 74 |
|
75 |
(*recT and rec_params should agree for all mutually recursive components*) |
|
76 |
val rec_hds = map head_of rec_tms; |
|
77 |
||
78 |
val dummy = assert_all is_Const rec_hds |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
79 |
(fn t => "Recursive set not previously declared as constant: " ^ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
80 |
Sign.string_of_term sign t); |
6051 | 81 |
|
82 |
(*Now we know they are all Consts, so get their names, type and params*) |
|
83 |
val rec_names = map (#1 o dest_Const) rec_hds |
|
84 |
and (Const(_,recT),rec_params) = strip_comb (hd rec_tms); |
|
85 |
||
86 |
val rec_base_names = map Sign.base_name rec_names; |
|
87 |
val dummy = assert_all Syntax.is_identifier rec_base_names |
|
88 |
(fn a => "Base name of recursive set not an identifier: " ^ a); |
|
89 |
||
90 |
local (*Checking the introduction rules*) |
|
91 |
val intr_sets = map (#2 o rule_concl_msg sign) intr_tms; |
|
92 |
fun intr_ok set = |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
93 |
case head_of set of Const(a,recT) => a mem rec_names | _ => false; |
6051 | 94 |
in |
95 |
val dummy = assert_all intr_ok intr_sets |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
96 |
(fn t => "Conclusion of rule does not name a recursive set: " ^ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
97 |
Sign.string_of_term sign t); |
6051 | 98 |
end; |
99 |
||
100 |
val dummy = assert_all is_Free rec_params |
|
101 |
(fn t => "Param in recursion term not a free variable: " ^ |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
102 |
Sign.string_of_term sign t); |
6051 | 103 |
|
104 |
(*** Construct the fixedpoint definition ***) |
|
15574
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
105 |
val mk_variant = variant (foldr add_term_names [] intr_tms); |
6051 | 106 |
|
107 |
val z' = mk_variant"z" and X' = mk_variant"X" and w' = mk_variant"w"; |
|
108 |
||
109 |
fun dest_tprop (Const("Trueprop",_) $ P) = P |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
110 |
| dest_tprop Q = error ("Ill-formed premise of introduction rule: " ^ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
111 |
Sign.string_of_term sign Q); |
6051 | 112 |
|
113 |
(*Makes a disjunct from an introduction rule*) |
|
114 |
fun fp_part intr = (*quantify over rule's free vars except parameters*) |
|
115 |
let val prems = map dest_tprop (strip_imp_prems intr) |
|
15570 | 116 |
val dummy = List.app (fn rec_hd => List.app (chk_prem rec_hd) prems) rec_hds |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
117 |
val exfrees = term_frees intr \\ rec_params |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
118 |
val zeq = FOLogic.mk_eq (Free(z',iT), #1 (rule_concl intr)) |
15574
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
119 |
in foldr FOLogic.mk_exists |
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
120 |
(fold_bal FOLogic.mk_conj (zeq::prems)) exfrees |
6051 | 121 |
end; |
122 |
||
123 |
(*The Part(A,h) terms -- compose injections to make h*) |
|
124 |
fun mk_Part (Bound 0) = Free(X',iT) (*no mutual rec, no Part needed*) |
|
125 |
| mk_Part h = Part_const $ Free(X',iT) $ Abs(w',iT,h); |
|
126 |
||
127 |
(*Access to balanced disjoint sums via injections*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
128 |
val parts = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
129 |
map mk_Part (accesses_bal (fn t => Su.inl $ t, fn t => Su.inr $ t, Bound 0) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
130 |
(length rec_tms)); |
6051 | 131 |
|
132 |
(*replace each set by the corresponding Part(A,h)*) |
|
133 |
val part_intrs = map (subst_free (rec_tms ~~ parts) o fp_part) intr_tms; |
|
134 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
135 |
val fp_abs = absfree(X', iT, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
136 |
mk_Collect(z', dom_sum, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
137 |
fold_bal FOLogic.mk_disj part_intrs)); |
6051 | 138 |
|
139 |
val fp_rhs = Fp.oper $ dom_sum $ fp_abs |
|
140 |
||
15570 | 141 |
val dummy = List.app (fn rec_hd => deny (rec_hd occs fp_rhs) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
142 |
"Illegal occurrence of recursion operator") |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
143 |
rec_hds; |
6051 | 144 |
|
145 |
(*** Make the new theory ***) |
|
146 |
||
147 |
(*A key definition: |
|
148 |
If no mutual recursion then it equals the one recursive set. |
|
149 |
If mutual recursion then it differs from all the recursive sets. *) |
|
150 |
val big_rec_base_name = space_implode "_" rec_base_names; |
|
151 |
val big_rec_name = Sign.intern_const sign big_rec_base_name; |
|
152 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
153 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
154 |
val dummy = conditional verbose (fn () => |
12243 | 155 |
writeln ((if coind then "Coind" else "Ind") ^ "uctive definition " ^ quote big_rec_name)); |
6051 | 156 |
|
157 |
(*Forbid the inductive definition structure from clashing with a theory |
|
158 |
name. This restriction may become obsolete as ML is de-emphasized.*) |
|
159 |
val dummy = deny (big_rec_base_name mem (Sign.stamp_names_of sign)) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
160 |
("Definition " ^ big_rec_base_name ^ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
161 |
" would clash with the theory of the same name!"); |
6051 | 162 |
|
163 |
(*Big_rec... is the union of the mutually recursive sets*) |
|
164 |
val big_rec_tm = list_comb(Const(big_rec_name,recT), rec_params); |
|
165 |
||
166 |
(*The individual sets must already be declared*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
167 |
val axpairs = map Logic.mk_defpair |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
168 |
((big_rec_tm, fp_rhs) :: |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
169 |
(case parts of |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
170 |
[_] => [] (*no mutual recursion*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
171 |
| _ => rec_tms ~~ (*define the sets as Parts*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
172 |
map (subst_atomic [(Free(X',iT),big_rec_tm)]) parts)); |
6051 | 173 |
|
174 |
(*tracing: print the fixedpoint definition*) |
|
175 |
val dummy = if !Ind_Syntax.trace then |
|
15570 | 176 |
List.app (writeln o Sign.string_of_term sign o #2) axpairs |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
177 |
else () |
6051 | 178 |
|
179 |
(*add definitions of the inductive sets*) |
|
180 |
val thy1 = thy |> Theory.add_path big_rec_base_name |
|
9329 | 181 |
|> (#1 o PureThy.add_defs_i false (map Thm.no_attributes axpairs)) |
6051 | 182 |
|
183 |
||
184 |
(*fetch fp definitions from the theory*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
185 |
val big_rec_def::part_rec_defs = |
6051 | 186 |
map (get_def thy1) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
187 |
(case rec_names of [_] => rec_names |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
188 |
| _ => big_rec_base_name::rec_names); |
6051 | 189 |
|
190 |
||
191 |
val sign1 = sign_of thy1; |
|
192 |
||
193 |
(********) |
|
194 |
val dummy = writeln " Proving monotonicity..."; |
|
195 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
196 |
val bnd_mono = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
197 |
prove_goalw_cterm [] |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
198 |
(cterm_of sign1 |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
199 |
(FOLogic.mk_Trueprop (Fp.bnd_mono $ dom_sum $ fp_abs))) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
200 |
(fn _ => |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
201 |
[rtac (Collect_subset RS bnd_monoI) 1, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
202 |
REPEAT (ares_tac (basic_monos @ monos) 1)]); |
6051 | 203 |
|
204 |
val dom_subset = standard (big_rec_def RS Fp.subs); |
|
205 |
||
206 |
val unfold = standard ([big_rec_def, bnd_mono] MRS Fp.Tarski); |
|
207 |
||
208 |
(********) |
|
209 |
val dummy = writeln " Proving the introduction rules..."; |
|
210 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
211 |
(*Mutual recursion? Helps to derive subset rules for the |
6051 | 212 |
individual sets.*) |
213 |
val Part_trans = |
|
214 |
case rec_names of |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
215 |
[_] => asm_rl |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
216 |
| _ => standard (Part_subset RS subset_trans); |
6051 | 217 |
|
218 |
(*To type-check recursive occurrences of the inductive sets, possibly |
|
219 |
enclosed in some monotonic operator M.*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
220 |
val rec_typechecks = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
221 |
[dom_subset] RL (asm_rl :: ([Part_trans] RL monos)) |
6051 | 222 |
RL [subsetD]; |
223 |
||
224 |
(*Type-checking is hardest aspect of proof; |
|
225 |
disjIn selects the correct disjunct after unfolding*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
226 |
fun intro_tacsf disjIn prems = |
6051 | 227 |
[(*insert prems and underlying sets*) |
228 |
cut_facts_tac prems 1, |
|
229 |
DETERM (stac unfold 1), |
|
230 |
REPEAT (resolve_tac [Part_eqI,CollectI] 1), |
|
231 |
(*Now 2-3 subgoals: typechecking, the disjunction, perhaps equality.*) |
|
232 |
rtac disjIn 2, |
|
233 |
(*Not ares_tac, since refl must be tried before equality assumptions; |
|
234 |
backtracking may occur if the premises have extra variables!*) |
|
235 |
DEPTH_SOLVE_1 (resolve_tac [refl,exI,conjI] 2 APPEND assume_tac 2), |
|
236 |
(*Now solve the equations like Tcons(a,f) = Inl(?b4)*) |
|
237 |
rewrite_goals_tac con_defs, |
|
238 |
REPEAT (rtac refl 2), |
|
239 |
(*Typechecking; this can fail*) |
|
6172 | 240 |
if !Ind_Syntax.trace then print_tac "The type-checking subgoal:" |
6051 | 241 |
else all_tac, |
242 |
REPEAT (FIRSTGOAL ( dresolve_tac rec_typechecks |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
243 |
ORELSE' eresolve_tac (asm_rl::PartE::SigmaE2:: |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
244 |
type_elims) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
245 |
ORELSE' hyp_subst_tac)), |
6051 | 246 |
if !Ind_Syntax.trace then print_tac "The subgoal after monos, type_elims:" |
247 |
else all_tac, |
|
248 |
DEPTH_SOLVE (swap_res_tac (SigmaI::subsetI::type_intrs) 1)]; |
|
249 |
||
250 |
(*combines disjI1 and disjI2 to get the corresponding nested disjunct...*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
251 |
val mk_disj_rls = |
6051 | 252 |
let fun f rl = rl RS disjI1 |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
253 |
and g rl = rl RS disjI2 |
6051 | 254 |
in accesses_bal(f, g, asm_rl) end; |
255 |
||
256 |
fun prove_intr (ct, tacsf) = prove_goalw_cterm part_rec_defs ct tacsf; |
|
257 |
||
258 |
val intrs = ListPair.map prove_intr |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
259 |
(map (cterm_of sign1) intr_tms, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
260 |
map intro_tacsf (mk_disj_rls(length intr_tms))) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
261 |
handle MetaSimplifier.SIMPLIFIER (msg,thm) => (print_thm thm; error msg); |
6051 | 262 |
|
263 |
(********) |
|
264 |
val dummy = writeln " Proving the elimination rule..."; |
|
265 |
||
266 |
(*Breaks down logical connectives in the monotonic function*) |
|
267 |
val basic_elim_tac = |
|
268 |
REPEAT (SOMEGOAL (eresolve_tac (Ind_Syntax.elim_rls @ Su.free_SEs) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
269 |
ORELSE' bound_hyp_subst_tac)) |
6051 | 270 |
THEN prune_params_tac |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
271 |
(*Mutual recursion: collapse references to Part(D,h)*) |
6051 | 272 |
THEN fold_tac part_rec_defs; |
273 |
||
274 |
(*Elimination*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
275 |
val elim = rule_by_tactic basic_elim_tac |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
276 |
(unfold RS Ind_Syntax.equals_CollectD) |
6051 | 277 |
|
278 |
(*Applies freeness of the given constructors, which *must* be unfolded by |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
279 |
the given defs. Cannot simply use the local con_defs because |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
280 |
con_defs=[] for inference systems. |
12175 | 281 |
Proposition A should have the form t:Si where Si is an inductive set*) |
282 |
fun make_cases ss A = |
|
283 |
rule_by_tactic |
|
284 |
(basic_elim_tac THEN ALLGOALS (asm_full_simp_tac ss) THEN basic_elim_tac) |
|
285 |
(Thm.assume A RS elim) |
|
286 |
|> Drule.standard'; |
|
287 |
fun mk_cases a = make_cases (*delayed evaluation of body!*) |
|
288 |
(simpset ()) (read_cterm (Thm.sign_of_thm elim) (a, propT)); |
|
6051 | 289 |
|
290 |
fun induction_rules raw_induct thy = |
|
291 |
let |
|
292 |
val dummy = writeln " Proving the induction rule..."; |
|
293 |
||
294 |
(*** Prove the main induction rule ***) |
|
295 |
||
296 |
val pred_name = "P"; (*name for predicate variables*) |
|
297 |
||
298 |
(*Used to make induction rules; |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
299 |
ind_alist = [(rec_tm1,pred1),...] associates predicates with rec ops |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
300 |
prem is a premise of an intr rule*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
301 |
fun add_induct_prem ind_alist (prem as Const("Trueprop",_) $ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
302 |
(Const("op :",_)$t$X), iprems) = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
303 |
(case gen_assoc (op aconv) (ind_alist, X) of |
15531 | 304 |
SOME pred => prem :: FOLogic.mk_Trueprop (pred $ t) :: iprems |
305 |
| NONE => (*possibly membership in M(rec_tm), for M monotone*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
306 |
let fun mk_sb (rec_tm,pred) = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
307 |
(rec_tm, Ind_Syntax.Collect_const$rec_tm$pred) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
308 |
in subst_free (map mk_sb ind_alist) prem :: iprems end) |
6051 | 309 |
| add_induct_prem ind_alist (prem,iprems) = prem :: iprems; |
310 |
||
311 |
(*Make a premise of the induction rule.*) |
|
312 |
fun induct_prem ind_alist intr = |
|
313 |
let val quantfrees = map dest_Free (term_frees intr \\ rec_params) |
|
15574
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
314 |
val iprems = foldr (add_induct_prem ind_alist) [] |
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
315 |
(Logic.strip_imp_prems intr) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
316 |
val (t,X) = Ind_Syntax.rule_concl intr |
15531 | 317 |
val (SOME pred) = gen_assoc (op aconv) (ind_alist, X) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
318 |
val concl = FOLogic.mk_Trueprop (pred $ t) |
6051 | 319 |
in list_all_free (quantfrees, Logic.list_implies (iprems,concl)) end |
320 |
handle Bind => error"Recursion term not found in conclusion"; |
|
321 |
||
322 |
(*Minimizes backtracking by delivering the correct premise to each goal. |
|
323 |
Intro rules with extra Vars in premises still cause some backtracking *) |
|
324 |
fun ind_tac [] 0 = all_tac |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
325 |
| ind_tac(prem::prems) i = |
13747
bf308fcfd08e
Better treatment of equality in premises of inductive definitions. Less
paulson
parents:
13627
diff
changeset
|
326 |
DEPTH_SOLVE_1 (ares_tac [prem, refl] i) THEN ind_tac prems (i-1); |
6051 | 327 |
|
328 |
val pred = Free(pred_name, Ind_Syntax.iT --> FOLogic.oT); |
|
329 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
330 |
val ind_prems = map (induct_prem (map (rpair pred) rec_tms)) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
331 |
intr_tms; |
6051 | 332 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
333 |
val dummy = if !Ind_Syntax.trace then |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
334 |
(writeln "ind_prems = "; |
15570 | 335 |
List.app (writeln o Sign.string_of_term sign1) ind_prems; |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
336 |
writeln "raw_induct = "; print_thm raw_induct) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
337 |
else (); |
6051 | 338 |
|
339 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
340 |
(*We use a MINIMAL simpset. Even FOL_ss contains too many simpules. |
6051 | 341 |
If the premises get simplified, then the proofs could fail.*) |
342 |
val min_ss = empty_ss |
|
12725 | 343 |
setmksimps (map mk_eq o ZF_atomize o gen_all) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
344 |
setSolver (mk_solver "minimal" |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
345 |
(fn prems => resolve_tac (triv_rls@prems) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
346 |
ORELSE' assume_tac |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
347 |
ORELSE' etac FalseE)); |
6051 | 348 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
349 |
val quant_induct = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
350 |
prove_goalw_cterm part_rec_defs |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
351 |
(cterm_of sign1 |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
352 |
(Logic.list_implies |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
353 |
(ind_prems, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
354 |
FOLogic.mk_Trueprop (Ind_Syntax.mk_all_imp(big_rec_tm,pred))))) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
355 |
(fn prems => |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
356 |
[rtac (impI RS allI) 1, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
357 |
DETERM (etac raw_induct 1), |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
358 |
(*Push Part inside Collect*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
359 |
full_simp_tac (min_ss addsimps [Part_Collect]) 1, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
360 |
(*This CollectE and disjE separates out the introduction rules*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
361 |
REPEAT (FIRSTGOAL (eresolve_tac [CollectE, disjE])), |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
362 |
(*Now break down the individual cases. No disjE here in case |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
363 |
some premise involves disjunction.*) |
13747
bf308fcfd08e
Better treatment of equality in premises of inductive definitions. Less
paulson
parents:
13627
diff
changeset
|
364 |
REPEAT (FIRSTGOAL (eresolve_tac [CollectE, exE, conjE] |
bf308fcfd08e
Better treatment of equality in premises of inductive definitions. Less
paulson
parents:
13627
diff
changeset
|
365 |
ORELSE' bound_hyp_subst_tac)), |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
366 |
ind_tac (rev prems) (length prems) ]); |
6051 | 367 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
368 |
val dummy = if !Ind_Syntax.trace then |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
369 |
(writeln "quant_induct = "; print_thm quant_induct) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
370 |
else (); |
6051 | 371 |
|
372 |
||
373 |
(*** Prove the simultaneous induction rule ***) |
|
374 |
||
375 |
(*Make distinct predicates for each inductive set*) |
|
376 |
||
377 |
(*The components of the element type, several if it is a product*) |
|
378 |
val elem_type = CP.pseudo_type dom_sum; |
|
379 |
val elem_factors = CP.factors elem_type; |
|
380 |
val elem_frees = mk_frees "za" elem_factors; |
|
381 |
val elem_tuple = CP.mk_tuple Pr.pair elem_type elem_frees; |
|
382 |
||
383 |
(*Given a recursive set and its domain, return the "fsplit" predicate |
|
384 |
and a conclusion for the simultaneous induction rule. |
|
385 |
NOTE. This will not work for mutually recursive predicates. Previously |
|
386 |
a summand 'domt' was also an argument, but this required the domain of |
|
387 |
mutual recursion to invariably be a disjoint sum.*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
388 |
fun mk_predpair rec_tm = |
6051 | 389 |
let val rec_name = (#1 o dest_Const o head_of) rec_tm |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
390 |
val pfree = Free(pred_name ^ "_" ^ Sign.base_name rec_name, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
391 |
elem_factors ---> FOLogic.oT) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
392 |
val qconcl = |
15574
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
393 |
foldr FOLogic.mk_all |
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
394 |
(FOLogic.imp $ |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
395 |
(Ind_Syntax.mem_const $ elem_tuple $ rec_tm) |
15574
b1d1b5bfc464
Removed practically all references to Library.foldr.
skalberg
parents:
15570
diff
changeset
|
396 |
$ (list_comb (pfree, elem_frees))) elem_frees |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
397 |
in (CP.ap_split elem_type FOLogic.oT pfree, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
398 |
qconcl) |
6051 | 399 |
end; |
400 |
||
401 |
val (preds,qconcls) = split_list (map mk_predpair rec_tms); |
|
402 |
||
403 |
(*Used to form simultaneous induction lemma*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
404 |
fun mk_rec_imp (rec_tm,pred) = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
405 |
FOLogic.imp $ (Ind_Syntax.mem_const $ Bound 0 $ rec_tm) $ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
406 |
(pred $ Bound 0); |
6051 | 407 |
|
408 |
(*To instantiate the main induction rule*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
409 |
val induct_concl = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
410 |
FOLogic.mk_Trueprop |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
411 |
(Ind_Syntax.mk_all_imp |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
412 |
(big_rec_tm, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
413 |
Abs("z", Ind_Syntax.iT, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
414 |
fold_bal FOLogic.mk_conj |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
415 |
(ListPair.map mk_rec_imp (rec_tms, preds))))) |
6051 | 416 |
and mutual_induct_concl = |
7695 | 417 |
FOLogic.mk_Trueprop(fold_bal FOLogic.mk_conj qconcls); |
6051 | 418 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
419 |
val dummy = if !Ind_Syntax.trace then |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
420 |
(writeln ("induct_concl = " ^ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
421 |
Sign.string_of_term sign1 induct_concl); |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
422 |
writeln ("mutual_induct_concl = " ^ |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
423 |
Sign.string_of_term sign1 mutual_induct_concl)) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
424 |
else (); |
6051 | 425 |
|
426 |
||
427 |
val lemma_tac = FIRST' [eresolve_tac [asm_rl, conjE, PartE, mp], |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
428 |
resolve_tac [allI, impI, conjI, Part_eqI], |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
429 |
dresolve_tac [spec, mp, Pr.fsplitD]]; |
6051 | 430 |
|
431 |
val need_mutual = length rec_names > 1; |
|
432 |
||
433 |
val lemma = (*makes the link between the two induction rules*) |
|
434 |
if need_mutual then |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
435 |
(writeln " Proving the mutual induction rule..."; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
436 |
prove_goalw_cterm part_rec_defs |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
437 |
(cterm_of sign1 (Logic.mk_implies (induct_concl, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
438 |
mutual_induct_concl))) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
439 |
(fn prems => |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
440 |
[cut_facts_tac prems 1, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
441 |
REPEAT (rewrite_goals_tac [Pr.split_eq] THEN |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
442 |
lemma_tac 1)])) |
6051 | 443 |
else (writeln " [ No mutual induction rule needed ]"; |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
444 |
TrueI); |
6051 | 445 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
446 |
val dummy = if !Ind_Syntax.trace then |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
447 |
(writeln "lemma = "; print_thm lemma) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
448 |
else (); |
6051 | 449 |
|
450 |
||
451 |
(*Mutual induction follows by freeness of Inl/Inr.*) |
|
452 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
453 |
(*Simplification largely reduces the mutual induction rule to the |
6051 | 454 |
standard rule*) |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
455 |
val mut_ss = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
456 |
min_ss addsimps [Su.distinct, Su.distinct', Su.inl_iff, Su.inr_iff]; |
6051 | 457 |
|
458 |
val all_defs = con_defs @ part_rec_defs; |
|
459 |
||
460 |
(*Removes Collects caused by M-operators in the intro rules. It is very |
|
461 |
hard to simplify |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
462 |
list({v: tf. (v : t --> P_t(v)) & (v : f --> P_f(v))}) |
6051 | 463 |
where t==Part(tf,Inl) and f==Part(tf,Inr) to list({v: tf. P_t(v)}). |
464 |
Instead the following rules extract the relevant conjunct. |
|
465 |
*) |
|
466 |
val cmonos = [subset_refl RS Collect_mono] RL monos |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
467 |
RLN (2,[rev_subsetD]); |
6051 | 468 |
|
469 |
(*Minimizes backtracking by delivering the correct premise to each goal*) |
|
470 |
fun mutual_ind_tac [] 0 = all_tac |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
471 |
| mutual_ind_tac(prem::prems) i = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
472 |
DETERM |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
473 |
(SELECT_GOAL |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
474 |
( |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
475 |
(*Simplify the assumptions and goal by unfolding Part and |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
476 |
using freeness of the Sum constructors; proves all but one |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
477 |
conjunct by contradiction*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
478 |
rewrite_goals_tac all_defs THEN |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
479 |
simp_tac (mut_ss addsimps [Part_iff]) 1 THEN |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
480 |
IF_UNSOLVED (*simp_tac may have finished it off!*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
481 |
((*simplify assumptions*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
482 |
(*some risk of excessive simplification here -- might have |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
483 |
to identify the bare minimum set of rewrites*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
484 |
full_simp_tac |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
485 |
(mut_ss addsimps conj_simps @ imp_simps @ quant_simps) 1 |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
486 |
THEN |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
487 |
(*unpackage and use "prem" in the corresponding place*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
488 |
REPEAT (rtac impI 1) THEN |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
489 |
rtac (rewrite_rule all_defs prem) 1 THEN |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
490 |
(*prem must not be REPEATed below: could loop!*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
491 |
DEPTH_SOLVE (FIRSTGOAL (ares_tac [impI] ORELSE' |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
492 |
eresolve_tac (conjE::mp::cmonos)))) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
493 |
) i) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
494 |
THEN mutual_ind_tac prems (i-1); |
6051 | 495 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
496 |
val mutual_induct_fsplit = |
6051 | 497 |
if need_mutual then |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
498 |
prove_goalw_cterm [] |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
499 |
(cterm_of sign1 |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
500 |
(Logic.list_implies |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
501 |
(map (induct_prem (rec_tms~~preds)) intr_tms, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
502 |
mutual_induct_concl))) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
503 |
(fn prems => |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
504 |
[rtac (quant_induct RS lemma) 1, |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
505 |
mutual_ind_tac (rev prems) (length prems)]) |
6051 | 506 |
else TrueI; |
507 |
||
508 |
(** Uncurrying the predicate in the ordinary induction rule **) |
|
509 |
||
510 |
(*instantiate the variable to a tuple, if it is non-trivial, in order to |
|
511 |
allow the predicate to be "opened up". |
|
512 |
The name "x.1" comes from the "RS spec" !*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
513 |
val inst = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
514 |
case elem_frees of [_] => I |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
515 |
| _ => instantiate ([], [(cterm_of sign1 (Var(("x",1), Ind_Syntax.iT)), |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
516 |
cterm_of sign1 elem_tuple)]); |
6051 | 517 |
|
518 |
(*strip quantifier and the implication*) |
|
519 |
val induct0 = inst (quant_induct RS spec RSN (2,rev_mp)); |
|
520 |
||
521 |
val Const ("Trueprop", _) $ (pred_var $ _) = concl_of induct0 |
|
522 |
||
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
523 |
val induct = CP.split_rule_var(pred_var, elem_type-->FOLogic.oT, induct0) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
524 |
|> standard |
6051 | 525 |
and mutual_induct = CP.remove_split mutual_induct_fsplit |
8438 | 526 |
|
12191 | 527 |
val (thy', [induct', mutual_induct']) = thy |> PureThy.add_thms |
12227 | 528 |
[((co_prefix ^ "induct", induct), [case_names, InductAttrib.induct_set_global big_rec_name]), |
12191 | 529 |
(("mutual_induct", mutual_induct), [case_names])]; |
12227 | 530 |
in ((thy', induct'), mutual_induct') |
6051 | 531 |
end; (*of induction_rules*) |
532 |
||
533 |
val raw_induct = standard ([big_rec_def, bnd_mono] MRS Fp.induct) |
|
534 |
||
12227 | 535 |
val ((thy2, induct), mutual_induct) = |
536 |
if not coind then induction_rules raw_induct thy1 |
|
537 |
else (thy1 |> PureThy.add_thms [((co_prefix ^ "induct", raw_induct), [])] |> apsnd hd, TrueI) |
|
6051 | 538 |
and defs = big_rec_def :: part_rec_defs |
539 |
||
540 |
||
8438 | 541 |
val (thy3, ([bnd_mono', dom_subset', elim'], [defs', intrs'])) = |
542 |
thy2 |
|
12183 | 543 |
|> IndCases.declare big_rec_name make_cases |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
544 |
|> PureThy.add_thms |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
545 |
[(("bnd_mono", bnd_mono), []), |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
546 |
(("dom_subset", dom_subset), []), |
12191 | 547 |
(("cases", elim), [case_names, InductAttrib.cases_set_global big_rec_name])] |
8438 | 548 |
|>>> (PureThy.add_thmss o map Thm.no_attributes) |
549 |
[("defs", defs), |
|
12175 | 550 |
("intros", intrs)]; |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
551 |
val (thy4, intrs'') = |
12191 | 552 |
thy3 |> PureThy.add_thms ((intr_names ~~ intrs') ~~ map #2 intr_specs) |
12175 | 553 |
|>> Theory.parent_path; |
8438 | 554 |
in |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
555 |
(thy4, |
8438 | 556 |
{defs = defs', |
557 |
bnd_mono = bnd_mono', |
|
558 |
dom_subset = dom_subset', |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
559 |
intrs = intrs'', |
8438 | 560 |
elim = elim', |
561 |
mk_cases = mk_cases, |
|
562 |
induct = induct, |
|
563 |
mutual_induct = mutual_induct}) |
|
564 |
end; |
|
6051 | 565 |
|
566 |
||
567 |
(*external version, accepting strings*) |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
568 |
fun add_inductive_x (srec_tms, sdom_sum) sintrs (monos, con_defs, type_intrs, type_elims) thy = |
8819 | 569 |
let |
570 |
val read = Sign.simple_read_term (Theory.sign_of thy); |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
571 |
val rec_tms = map (read Ind_Syntax.iT) srec_tms; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
572 |
val dom_sum = read Ind_Syntax.iT sdom_sum; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
573 |
val intr_tms = map (read propT o snd o fst) sintrs; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
574 |
val intr_specs = (map (fst o fst) sintrs ~~ intr_tms) ~~ map snd sintrs; |
8819 | 575 |
in |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
576 |
add_inductive_i true (rec_tms, dom_sum) intr_specs |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
577 |
(monos, con_defs, type_intrs, type_elims) thy |
8819 | 578 |
end |
6051 | 579 |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
580 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
581 |
(*source version*) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
582 |
fun add_inductive (srec_tms, sdom_sum) intr_srcs |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
583 |
(raw_monos, raw_con_defs, raw_type_intrs, raw_type_elims) thy = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
584 |
let |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
585 |
val intr_atts = map (map (Attrib.global_attribute thy) o snd) intr_srcs; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
586 |
val (thy', (((monos, con_defs), type_intrs), type_elims)) = thy |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
587 |
|> IsarThy.apply_theorems raw_monos |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
588 |
|>>> IsarThy.apply_theorems raw_con_defs |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
589 |
|>>> IsarThy.apply_theorems raw_type_intrs |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
590 |
|>>> IsarThy.apply_theorems raw_type_elims; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
591 |
in |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
592 |
add_inductive_x (srec_tms, sdom_sum) (map fst intr_srcs ~~ intr_atts) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
593 |
(monos, con_defs, type_intrs, type_elims) thy' |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
594 |
end; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
595 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
596 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
597 |
(* outer syntax *) |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
598 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
599 |
local structure P = OuterParse and K = OuterSyntax.Keyword in |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
600 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
601 |
fun mk_ind (((((doms, intrs), monos), con_defs), type_intrs), type_elims) = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
602 |
#1 o add_inductive doms (map P.triple_swap intrs) (monos, con_defs, type_intrs, type_elims); |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
603 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
604 |
val ind_decl = |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
605 |
(P.$$$ "domains" |-- P.!!! (P.enum1 "+" P.term -- |
12876
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
wenzelm
parents:
12725
diff
changeset
|
606 |
((P.$$$ "\\<subseteq>" || P.$$$ "<=") |-- P.term))) -- |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
607 |
(P.$$$ "intros" |-- |
12876
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
wenzelm
parents:
12725
diff
changeset
|
608 |
P.!!! (Scan.repeat1 (P.opt_thm_name ":" -- P.prop))) -- |
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
wenzelm
parents:
12725
diff
changeset
|
609 |
Scan.optional (P.$$$ "monos" |-- P.!!! P.xthms1) [] -- |
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
wenzelm
parents:
12725
diff
changeset
|
610 |
Scan.optional (P.$$$ "con_defs" |-- P.!!! P.xthms1) [] -- |
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
wenzelm
parents:
12725
diff
changeset
|
611 |
Scan.optional (P.$$$ "type_intros" |-- P.!!! P.xthms1) [] -- |
a70df1e5bf10
got rid of explicit marginal comments (now stripped earlier from input);
wenzelm
parents:
12725
diff
changeset
|
612 |
Scan.optional (P.$$$ "type_elims" |-- P.!!! P.xthms1) [] |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
613 |
>> (Toplevel.theory o mk_ind); |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
614 |
|
12227 | 615 |
val inductiveP = OuterSyntax.command (co_prefix ^ "inductive") |
616 |
("define " ^ co_prefix ^ "inductive sets") K.thy_decl ind_decl; |
|
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
617 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
618 |
val _ = OuterSyntax.add_keywords |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
619 |
["domains", "intros", "monos", "con_defs", "type_intros", "type_elims"]; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
620 |
val _ = OuterSyntax.add_parsers [inductiveP]; |
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
621 |
|
6051 | 622 |
end; |
12132
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
623 |
|
1ef58b332ca9
support co/inductive definitions in new-style theories;
wenzelm
parents:
11680
diff
changeset
|
624 |
end; |