author | wenzelm |
Thu, 07 Aug 2008 19:21:41 +0200 | |
changeset 27779 | 4569003b8813 |
parent 27378 | 0968c0d0b969 |
child 27809 | a1e409db516b |
permissions | -rw-r--r-- |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
1 |
(* Title: Pure/Isar/rule_insts.ML |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
2 |
ID: $Id$ |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
3 |
Author: Makarius |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
4 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
5 |
Rule instantiations -- operations within a rule/subgoal context. |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
6 |
*) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
7 |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
8 |
signature BASIC_RULE_INSTS = |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
9 |
sig |
27236 | 10 |
val read_instantiate: Proof.context -> (indexname * string) list -> thm -> thm |
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
11 |
val instantiate_tac: Proof.context -> (indexname * string) list -> tactic |
27120 | 12 |
val res_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic |
13 |
val eres_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
14 |
val cut_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
15 |
val forw_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
16 |
val dres_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
17 |
val thin_tac: Proof.context -> string -> int -> tactic |
27219 | 18 |
val subgoal_tac: Proof.context -> string -> int -> tactic |
19 |
val subgoals_tac: Proof.context -> string list -> int -> tactic |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
20 |
end; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
21 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
22 |
signature RULE_INSTS = |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
23 |
sig |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
24 |
include BASIC_RULE_INSTS |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
25 |
val make_elim_preserve: thm -> thm |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
26 |
end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
27 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
28 |
structure RuleInsts: RULE_INSTS = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
29 |
struct |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
30 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
31 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
32 |
(** reading instantiations **) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
33 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
34 |
local |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
35 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
36 |
fun is_tvar (x, _) = String.isPrefix "'" x; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
37 |
|
22681
9d42e5365ad1
cleaned/simplified Sign.read_typ, Thm.read_cterm etc.;
wenzelm
parents:
21879
diff
changeset
|
38 |
fun error_var msg xi = error (msg ^ Term.string_of_vname xi); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
39 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
40 |
fun the_sort tvars xi = the (AList.lookup (op =) tvars xi) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
41 |
handle Option.Option => error_var "No such type variable in theorem: " xi; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
42 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
43 |
fun the_type vars xi = the (AList.lookup (op =) vars xi) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
44 |
handle Option.Option => error_var "No such variable in theorem: " xi; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
45 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
46 |
fun unify_vartypes thy vars (xi, u) (unifier, maxidx) = |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
47 |
let |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
48 |
val T = the_type vars xi; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
49 |
val U = Term.fastype_of u; |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
50 |
val maxidx' = Term.maxidx_term u (Int.max (#2 xi, maxidx)); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
51 |
in |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
52 |
Sign.typ_unify thy (T, U) (unifier, maxidx') |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
53 |
handle Type.TUNIFY => error_var "Incompatible type for instantiation of " xi |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
54 |
end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
55 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
56 |
fun instantiate inst = |
20509 | 57 |
TermSubst.instantiate ([], map (fn (xi, t) => ((xi, Term.fastype_of t), t)) inst) #> |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
58 |
Envir.beta_norm; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
59 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
60 |
fun make_instT f v = |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
61 |
let |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
62 |
val T = TVar v; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
63 |
val T' = f T; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
64 |
in if T = T' then NONE else SOME (T, T') end; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
65 |
|
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
66 |
fun make_inst f v = |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
67 |
let |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
68 |
val t = Var v; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
69 |
val t' = f t; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
70 |
in if t aconv t' then NONE else SOME (t, t') end; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
71 |
|
27282 | 72 |
val add_used = |
73 |
(Thm.fold_terms o fold_types o fold_atyps) |
|
74 |
(fn TFree (a, _) => insert (op =) a |
|
75 |
| TVar ((a, _), _) => insert (op =) a |
|
76 |
| _ => I); |
|
77 |
||
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
78 |
in |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
79 |
|
25333 | 80 |
fun read_termTs ctxt schematic ss Ts = |
25329 | 81 |
let |
82 |
fun parse T = if T = propT then Syntax.parse_prop ctxt else Syntax.parse_term ctxt; |
|
83 |
val ts = map2 parse Ts ss; |
|
84 |
val ts' = |
|
85 |
map2 (TypeInfer.constrain o TypeInfer.paramify_vars) Ts ts |
|
25333 | 86 |
|> Syntax.check_terms ((schematic ? ProofContext.set_mode ProofContext.mode_schematic) ctxt) |
25329 | 87 |
|> Variable.polymorphic ctxt; |
88 |
val Ts' = map Term.fastype_of ts'; |
|
89 |
val tyenv = fold Type.raw_match (Ts ~~ Ts') Vartab.empty; |
|
90 |
in (ts', map (apsnd snd) (Vartab.dest tyenv)) end; |
|
91 |
||
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
92 |
fun read_insts ctxt mixed_insts (tvars, vars) = |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
93 |
let |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
94 |
val thy = ProofContext.theory_of ctxt; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
95 |
val cert = Thm.cterm_of thy; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
96 |
val certT = Thm.ctyp_of thy; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
97 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
98 |
val (type_insts, term_insts) = List.partition (is_tvar o fst) mixed_insts; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
99 |
val internal_insts = term_insts |> map_filter |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
100 |
(fn (xi, Args.Term t) => SOME (xi, t) |
21500 | 101 |
| (_, Args.Text _) => NONE |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
102 |
| (xi, _) => error_var "Term argument expected for " xi); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
103 |
val external_insts = term_insts |> map_filter |
21500 | 104 |
(fn (xi, Args.Text s) => SOME (xi, s) | _ => NONE); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
105 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
106 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
107 |
(* mixed type instantiations *) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
108 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
109 |
fun readT (xi, arg) = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
110 |
let |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
111 |
val S = the_sort tvars xi; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
112 |
val T = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
113 |
(case arg of |
25333 | 114 |
Args.Text s => Syntax.read_typ ctxt s |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
115 |
| Args.Typ T => T |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
116 |
| _ => error_var "Type argument expected for " xi); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
117 |
in |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
118 |
if Sign.of_sort thy (T, S) then ((xi, S), T) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
119 |
else error_var "Incompatible sort for typ instantiation of " xi |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
120 |
end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
121 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
122 |
val type_insts1 = map readT type_insts; |
20509 | 123 |
val instT1 = TermSubst.instantiateT type_insts1; |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
124 |
val vars1 = map (apsnd instT1) vars; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
125 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
126 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
127 |
(* internal term instantiations *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
128 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
129 |
val instT2 = Envir.norm_type |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
130 |
(#1 (fold (unify_vartypes thy vars1) internal_insts (Vartab.empty, 0))); |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
131 |
val vars2 = map (apsnd instT2) vars1; |
20548
8ef25fe585a8
renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
wenzelm
parents:
20509
diff
changeset
|
132 |
val internal_insts2 = map (apsnd (map_types instT2)) internal_insts; |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
133 |
val inst2 = instantiate internal_insts2; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
134 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
135 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
136 |
(* external term instantiations *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
137 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
138 |
val (xs, strs) = split_list external_insts; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
139 |
val Ts = map (the_type vars2) xs; |
25354 | 140 |
val (ts, inferred) = read_termTs ctxt false strs Ts; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
141 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
142 |
val instT3 = Term.typ_subst_TVars inferred; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
143 |
val vars3 = map (apsnd instT3) vars2; |
20548
8ef25fe585a8
renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
wenzelm
parents:
20509
diff
changeset
|
144 |
val internal_insts3 = map (apsnd (map_types instT3)) internal_insts2; |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
145 |
val external_insts3 = xs ~~ ts; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
146 |
val inst3 = instantiate external_insts3; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
147 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
148 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
149 |
(* results *) |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
150 |
|
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
151 |
val type_insts3 = map (fn ((a, _), T) => (a, instT3 (instT2 T))) type_insts1; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
152 |
val term_insts3 = internal_insts3 @ external_insts3; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
153 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
154 |
val inst_tvars = map_filter (make_instT (instT3 o instT2 o instT1)) tvars; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
155 |
val inst_vars = map_filter (make_inst (inst3 o inst2)) vars3; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
156 |
in |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
157 |
((type_insts3, term_insts3), |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
158 |
(map (pairself certT) inst_tvars, map (pairself cert) inst_vars)) |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
159 |
end; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
160 |
|
27236 | 161 |
fun read_instantiate_mixed ctxt mixed_insts thm = |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
162 |
let |
20487
6ac7a4fc32a0
read_instantiate: declare names of TVars as well (temporary workaround for no-freeze feature of type inference);
wenzelm
parents:
20343
diff
changeset
|
163 |
val ctxt' = ctxt |> Variable.declare_thm thm |
27282 | 164 |
|> fold (fn a => Variable.declare_names (Logic.mk_type (TFree (a, dummyS)))) (add_used thm []); (* FIXME tmp *) |
22692 | 165 |
val tvars = Thm.fold_terms Term.add_tvars thm []; |
166 |
val vars = Thm.fold_terms Term.add_vars thm []; |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
167 |
val ((type_insts, term_insts), insts) = read_insts ctxt' (map snd mixed_insts) (tvars, vars); |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
168 |
|
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
169 |
val _ = (*assign internalized values*) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
170 |
mixed_insts |> List.app (fn (arg, (xi, _)) => |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
171 |
if is_tvar xi then |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
172 |
Args.assign (SOME (Args.Typ (the (AList.lookup (op =) type_insts xi)))) arg |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
173 |
else |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
174 |
Args.assign (SOME (Args.Term (the (AList.lookup (op =) term_insts xi)))) arg); |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
175 |
in |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
176 |
Drule.instantiate insts thm |> RuleCases.save thm |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
177 |
end; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
178 |
|
27236 | 179 |
fun read_instantiate_mixed' ctxt (args, concl_args) thm = |
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
180 |
let |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
181 |
fun zip_vars _ [] = [] |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
182 |
| zip_vars (_ :: xs) ((_, NONE) :: rest) = zip_vars xs rest |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
183 |
| zip_vars ((x, _) :: xs) ((arg, SOME t) :: rest) = (arg, (x, t)) :: zip_vars xs rest |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
184 |
| zip_vars [] _ = error "More instantiations than variables in theorem"; |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
185 |
val insts = |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
186 |
zip_vars (rev (Term.add_vars (Thm.full_prop_of thm) [])) args @ |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
187 |
zip_vars (rev (Term.add_vars (Thm.concl_of thm) [])) concl_args; |
27236 | 188 |
in read_instantiate_mixed ctxt insts thm end; |
189 |
||
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
190 |
end; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
191 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
192 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
193 |
(* instantiation of rule or goal state *) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
194 |
|
27236 | 195 |
fun read_instantiate ctxt args thm = |
196 |
read_instantiate_mixed (ctxt |> ProofContext.set_mode ProofContext.mode_schematic) (* FIXME !? *) |
|
197 |
(map (fn (x, y) => (Args.eof, (x, Args.Text y))) args) thm; |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
198 |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
199 |
fun instantiate_tac ctxt args = PRIMITIVE (read_instantiate ctxt args); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
200 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
201 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
202 |
|
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
203 |
(** attributes **) |
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
204 |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
205 |
(* where: named instantiation *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
206 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
207 |
local |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
208 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
209 |
val value = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
210 |
Args.internal_typ >> Args.Typ || |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
211 |
Args.internal_term >> Args.Term || |
21500 | 212 |
Args.name >> Args.Text; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
213 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
214 |
val inst = Args.var -- (Args.$$$ "=" |-- Args.ahead -- value) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
215 |
>> (fn (xi, (a, v)) => (a, (xi, v))); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
216 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
217 |
in |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
218 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
219 |
val where_att = Attrib.syntax (Args.and_list (Scan.lift inst) >> (fn args => |
27236 | 220 |
Thm.rule_attribute (fn context => read_instantiate_mixed (Context.proof_of context) args))); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
221 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
222 |
end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
223 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
224 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
225 |
(* of: positional instantiation (terms only) *) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
226 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
227 |
local |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
228 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
229 |
val value = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
230 |
Args.internal_term >> Args.Term || |
21500 | 231 |
Args.name >> Args.Text; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
232 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
233 |
val inst = Args.ahead -- Args.maybe value; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
234 |
val concl = Args.$$$ "concl" -- Args.colon; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
235 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
236 |
val insts = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
237 |
Scan.repeat (Scan.unless concl inst) -- |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
238 |
Scan.optional (concl |-- Scan.repeat inst) []; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
239 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
240 |
in |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
241 |
|
20343
e093a54bf25e
reworked read_instantiate -- separate read_insts;
wenzelm
parents:
20336
diff
changeset
|
242 |
val of_att = Attrib.syntax (Scan.lift insts >> (fn args => |
27236 | 243 |
Thm.rule_attribute (fn context => read_instantiate_mixed' (Context.proof_of context) args))); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
244 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
245 |
end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
246 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
247 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
248 |
(* setup *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
249 |
|
26463 | 250 |
val _ = Context.>> (Context.map_theory |
251 |
(Attrib.add_attributes |
|
252 |
[("where", where_att, "named instantiation of theorem"), |
|
253 |
("of", of_att, "positional instantiation of theorem")])); |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
254 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
255 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
256 |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
257 |
(** tactics **) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
258 |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
259 |
(* resolution after lifting and instantation; may refer to parameters of the subgoal *) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
260 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
261 |
(* FIXME cleanup this mess!!! *) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
262 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
263 |
fun bires_inst_tac bires_flag ctxt insts thm = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
264 |
let |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
265 |
val thy = ProofContext.theory_of ctxt; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
266 |
(* Separate type and term insts *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
267 |
fun has_type_var ((x, _), _) = (case Symbol.explode x of |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
268 |
"'"::cs => true | cs => false); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
269 |
val Tinsts = List.filter has_type_var insts; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
270 |
val tinsts = filter_out has_type_var insts; |
25333 | 271 |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
272 |
(* Tactic *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
273 |
fun tac i st = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
274 |
let |
25333 | 275 |
val (_, _, Bi, _) = Thm.dest_state (st, i); |
276 |
val params = Logic.strip_params Bi; (*params of subgoal i as string typ pairs*) |
|
277 |
val params = rev (Term.rename_wrt_term Bi params) |
|
278 |
(*as they are printed: bound variables with*) |
|
279 |
(*the same name are renamed during printing*) |
|
280 |
||
281 |
val (param_names, ctxt') = ctxt |
|
282 |
|> Variable.declare_thm thm |
|
283 |
|> Thm.fold_terms Variable.declare_constraints st |
|
284 |
|> ProofContext.add_fixes_i (map (fn (x, T) => (x, SOME T, NoSyn)) params); |
|
285 |
||
286 |
(* Process type insts: Tinsts_env *) |
|
287 |
fun absent xi = error |
|
288 |
("No such variable in theorem: " ^ Term.string_of_vname xi); |
|
289 |
val (rtypes, rsorts) = Drule.types_sorts thm; |
|
290 |
fun readT (xi, s) = |
|
291 |
let val S = case rsorts xi of SOME S => S | NONE => absent xi; |
|
292 |
val T = Syntax.read_typ ctxt' s; |
|
293 |
val U = TVar (xi, S); |
|
294 |
in if Sign.typ_instance thy (T, U) then (U, T) |
|
295 |
else error ("Instantiation of " ^ Term.string_of_vname xi ^ " fails") |
|
296 |
end; |
|
297 |
val Tinsts_env = map readT Tinsts; |
|
298 |
(* Preprocess rule: extract vars and their types, apply Tinsts *) |
|
299 |
fun get_typ xi = |
|
300 |
(case rtypes xi of |
|
301 |
SOME T => typ_subst_atomic Tinsts_env T |
|
302 |
| NONE => absent xi); |
|
303 |
val (xis, ss) = Library.split_list tinsts; |
|
304 |
val Ts = map get_typ xis; |
|
305 |
||
306 |
val (ts, envT) = read_termTs ctxt' true ss Ts; |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
307 |
val envT' = map (fn (ixn, T) => |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
308 |
(TVar (ixn, the (rsorts ixn)), T)) envT @ Tinsts_env; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
309 |
val cenv = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
310 |
map |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
311 |
(fn (xi, t) => |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
312 |
pairself (Thm.cterm_of thy) (Var (xi, fastype_of t), t)) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
313 |
(distinct |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
314 |
(fn ((x1, t1), (x2, t2)) => x1 = x2 andalso t1 aconv t2) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
315 |
(xis ~~ ts)); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
316 |
(* Lift and instantiate rule *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
317 |
val {maxidx, ...} = rep_thm st; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
318 |
val paramTs = map #2 params |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
319 |
and inc = maxidx+1 |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
320 |
fun liftvar (Var ((a,j), T)) = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
321 |
Var((a, j+inc), paramTs ---> Logic.incr_tvar inc T) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
322 |
| liftvar t = raise TERM("Variable expected", [t]); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
323 |
fun liftterm t = list_abs_free |
25333 | 324 |
(param_names ~~ paramTs, Logic.incr_indexes(paramTs,inc) t) |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
325 |
fun liftpair (cv,ct) = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
326 |
(cterm_fun liftvar cv, cterm_fun liftterm ct) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
327 |
val lifttvar = pairself (ctyp_of thy o Logic.incr_tvar inc); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
328 |
val rule = Drule.instantiate |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
329 |
(map lifttvar envT', map liftpair cenv) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
330 |
(Thm.lift_rule (Thm.cprem_of st i) thm) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
331 |
in |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
332 |
if i > nprems_of st then no_tac st |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
333 |
else st |> |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
334 |
compose_tac (bires_flag, rule, nprems_of thm) i |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
335 |
end |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
336 |
handle TERM (msg,_) => (warning msg; no_tac st) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
337 |
| THM (msg,_,_) => (warning msg; no_tac st); |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
338 |
in tac end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
339 |
|
27120 | 340 |
val res_inst_tac = bires_inst_tac false; |
341 |
val eres_inst_tac = bires_inst_tac true; |
|
342 |
||
343 |
||
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
344 |
(* forward resolution *) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
345 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
346 |
fun make_elim_preserve rl = |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
347 |
let |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
348 |
val cert = Thm.cterm_of (Thm.theory_of_thm rl); |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
349 |
val maxidx = Thm.maxidx_of rl; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
350 |
fun cvar xi = cert (Var (xi, propT)); |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
351 |
val revcut_rl' = |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
352 |
instantiate ([], [(cvar ("V", 0), cvar ("V", maxidx + 1)), |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
353 |
(cvar ("W", 0), cvar ("W", maxidx + 1))]) Drule.revcut_rl; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
354 |
in |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
355 |
(case Seq.list_of (bicompose false (false, rl, Thm.nprems_of rl) 1 revcut_rl') of |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
356 |
[th] => th |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
357 |
| _ => raise THM ("make_elim_preserve", 1, [rl])) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
358 |
end; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
359 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
360 |
(*instantiate and cut -- for atomic fact*) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
361 |
fun cut_inst_tac ctxt insts rule = res_inst_tac ctxt insts (make_elim_preserve rule); |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
362 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
363 |
(*forward tactic applies a rule to an assumption without deleting it*) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
364 |
fun forw_inst_tac ctxt insts rule = cut_inst_tac ctxt insts rule THEN' assume_tac; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
365 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
366 |
(*dresolve tactic applies a rule to replace an assumption*) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
367 |
fun dres_inst_tac ctxt insts rule = eres_inst_tac ctxt insts (make_elim_preserve rule); |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
368 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
369 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
370 |
(* derived tactics *) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
371 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
372 |
(*deletion of an assumption*) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
373 |
fun thin_tac ctxt s = eres_inst_tac ctxt [(("V", 0), s)] Drule.thin_rl; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
374 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
375 |
(*Introduce the given proposition as lemma and subgoal*) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
376 |
fun subgoal_tac ctxt A = DETERM o res_inst_tac ctxt [(("psi", 0), A)] cut_rl; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
377 |
fun subgoals_tac ctxt As = EVERY' (map (subgoal_tac ctxt) As); |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
378 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
379 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
380 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
381 |
(** methods **) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
382 |
|
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
383 |
(* rule_tac etc. -- refer to dynamic goal state! *) |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
384 |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
385 |
local |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
386 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
387 |
fun gen_inst _ tac _ (quant, ([], thms)) = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
388 |
Method.METHOD (fn facts => quant (Method.insert_tac facts THEN' tac thms)) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
389 |
| gen_inst inst_tac _ ctxt (quant, (insts, [thm])) = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
390 |
Method.METHOD (fn facts => |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
391 |
quant (Method.insert_tac facts THEN' inst_tac ctxt insts thm)) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
392 |
| gen_inst _ _ _ _ = error "Cannot have instantiations with multiple rules"; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
393 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
394 |
in |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
395 |
|
27120 | 396 |
val res_inst_meth = gen_inst res_inst_tac Tactic.resolve_tac; |
397 |
val eres_inst_meth = gen_inst eres_inst_tac Tactic.eresolve_tac; |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
398 |
val cut_inst_meth = gen_inst cut_inst_tac Tactic.cut_rules_tac; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
399 |
val dres_inst_meth = gen_inst dres_inst_tac Tactic.dresolve_tac; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
400 |
val forw_inst_meth = gen_inst forw_inst_tac Tactic.forward_tac; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
401 |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
402 |
end; |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
403 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
404 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
405 |
(* method syntax *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
406 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
407 |
val insts = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
408 |
Scan.optional |
27378 | 409 |
(Args.and_list1 (Scan.lift (Args.name -- (Args.$$$ "=" |-- Args.!!! Args.name))) --| |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
410 |
Scan.lift (Args.$$$ "in")) [] -- Attrib.thms; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
411 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
412 |
fun inst_args f src ctxt = |
21879 | 413 |
f ctxt (fst (Method.syntax (Args.goal_spec HEADGOAL -- insts) src ctxt)); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
414 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
415 |
val insts_var = |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
416 |
Scan.optional |
27378 | 417 |
(Args.and_list1 (Scan.lift (Args.var -- (Args.$$$ "=" |-- Args.!!! Args.name))) --| |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
418 |
Scan.lift (Args.$$$ "in")) [] -- Attrib.thms; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
419 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
420 |
fun inst_args_var f src ctxt = |
21879 | 421 |
f ctxt (fst (Method.syntax (Args.goal_spec HEADGOAL -- insts_var) src ctxt)); |
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
422 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
423 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
424 |
(* setup *) |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
425 |
|
26463 | 426 |
val _ = Context.>> (Context.map_theory |
427 |
(Method.add_methods |
|
428 |
[("rule_tac", inst_args_var res_inst_meth, |
|
429 |
"apply rule (dynamic instantiation)"), |
|
430 |
("erule_tac", inst_args_var eres_inst_meth, |
|
431 |
"apply rule in elimination manner (dynamic instantiation)"), |
|
432 |
("drule_tac", inst_args_var dres_inst_meth, |
|
433 |
"apply rule in destruct manner (dynamic instantiation)"), |
|
434 |
("frule_tac", inst_args_var forw_inst_meth, |
|
435 |
"apply rule in forward manner (dynamic instantiation)"), |
|
436 |
("cut_tac", inst_args_var cut_inst_meth, |
|
437 |
"cut rule (dynamic instantiation)"), |
|
438 |
("subgoal_tac", Method.goal_args_ctxt (Scan.repeat1 Args.name) subgoals_tac, |
|
439 |
"insert subgoal (dynamic instantiation)"), |
|
440 |
("thin_tac", Method.goal_args_ctxt Args.name thin_tac, |
|
441 |
"remove premise (dynamic instantiation)")])); |
|
20336
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
442 |
|
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
443 |
end; |
aac494583949
Rule instantiations -- operations within a rule/subgoal context.
wenzelm
parents:
diff
changeset
|
444 |
|
27245
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
445 |
structure BasicRuleInsts: BASIC_RULE_INSTS = RuleInsts; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
446 |
open BasicRuleInsts; |
817d34377170
added instantiate_tac, cut_inst_tac, forw_inst_tac, dres_inst_tac, make_elim_preserve (from tactic.ML);
wenzelm
parents:
27236
diff
changeset
|
447 |