| author | paulson | 
| Thu, 03 May 2001 10:27:37 +0200 | |
| changeset 11280 | 6fdc4c4ccec1 | 
| parent 10816 | 8b2eafed6183 | 
| child 12137 | 6123958975b8 | 
| permissions | -rw-r--r-- | 
| 9460 | 1 | (* Title: Pure/logic.ML | 
| 0 | 2 | ID: $Id$ | 
| 9460 | 3 | Author: Lawrence C Paulson, Cambridge University Computer Laboratory | 
| 0 | 4 | Copyright Cambridge University 1992 | 
| 5 | ||
| 9460 | 6 | Abstract syntax operations of the Pure meta-logic. | 
| 0 | 7 | *) | 
| 8 | ||
| 9 | infix occs; | |
| 10 | ||
| 9460 | 11 | signature LOGIC = | 
| 4345 | 12 | sig | 
| 5041 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 13 | val is_all : term -> bool | 
| 9460 | 14 | val mk_equals : term * term -> term | 
| 15 | val dest_equals : term -> term * term | |
| 3963 
29c5ec9ecbaa
Corrected alphabetical order of entries in signature.
 nipkow parents: 
3915diff
changeset | 16 | val is_equals : term -> bool | 
| 9460 | 17 | val mk_implies : term * term -> term | 
| 18 | val dest_implies : term -> term * term | |
| 5041 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 19 | val is_implies : term -> bool | 
| 9460 | 20 | val list_implies : term list * term -> term | 
| 21 | val strip_imp_prems : term -> term list | |
| 22 | val strip_imp_concl : term -> term | |
| 23 | val strip_prems : int * term list * term -> term list * term | |
| 24 | val count_prems : term * int -> int | |
| 25 | val mk_flexpair : term * term -> term | |
| 26 | val dest_flexpair : term -> term * term | |
| 27 | val list_flexpairs : (term*term)list * term -> term | |
| 28 | val rule_of : (term*term)list * term list * term -> term | |
| 29 | val strip_flexpairs : term -> (term*term)list * term | |
| 30 | val skip_flexpairs : term -> term | |
| 31 | val strip_horn : term -> (term*term)list * term list * term | |
| 32 | val mk_cond_defpair : term list -> term * term -> string * term | |
| 33 | val mk_defpair : term * term -> string * term | |
| 34 | val mk_type : typ -> term | |
| 35 | val dest_type : term -> typ | |
| 36 | val mk_inclass : typ * class -> term | |
| 37 | val dest_inclass : term -> typ * class | |
| 38 | val goal_const : term | |
| 39 | val mk_goal : term -> term | |
| 40 | val dest_goal : term -> term | |
| 41 | val occs : term * term -> bool | |
| 42 | val close_form : term -> term | |
| 43 | val incr_indexes : typ list * int -> term -> term | |
| 44 | val lift_fns : term * int -> (term -> term) * (term -> term) | |
| 45 | val strip_assums_hyp : term -> term list | |
| 46 | val strip_assums_concl: term -> term | |
| 47 | val strip_params : term -> (string * typ) list | |
| 10816 | 48 | val is_norm_hhf : term -> bool | 
| 9667 | 49 | val has_meta_prems : term -> int -> bool | 
| 9460 | 50 | val flatten_params : int -> term -> term | 
| 51 | val auto_rename : bool ref | |
| 52 | val set_rename_prefix : string -> unit | |
| 0 | 53 | val list_rename_params: string list * term -> term | 
| 9460 | 54 | val assum_pairs : term -> (term*term)list | 
| 55 | val varify : term -> term | |
| 56 | val unvarify : term -> term | |
| 4345 | 57 | end; | 
| 0 | 58 | |
| 1500 | 59 | structure Logic : LOGIC = | 
| 0 | 60 | struct | 
| 398 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 61 | |
| 4345 | 62 | |
| 0 | 63 | (*** Abstract syntax operations on the meta-connectives ***) | 
| 64 | ||
| 5041 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 65 | (** all **) | 
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 66 | |
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 67 | fun is_all (Const ("all", _) $ _) = true
 | 
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 68 | | is_all _ = false; | 
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 69 | |
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 70 | |
| 0 | 71 | (** equality **) | 
| 72 | ||
| 1835 | 73 | (*Make an equality. DOES NOT CHECK TYPE OF u*) | 
| 64 
0bbe5d86cb38
logic/mk_equals,mk_flexpair: now calls fastype_of instead of type_of.
 lcp parents: 
0diff
changeset | 74 | fun mk_equals(t,u) = equals(fastype_of t) $ t $ u; | 
| 0 | 75 | |
| 76 | fun dest_equals (Const("==",_) $ t $ u)  =  (t,u)
 | |
| 77 |   | dest_equals t = raise TERM("dest_equals", [t]);
 | |
| 78 | ||
| 637 | 79 | fun is_equals (Const ("==", _) $ _ $ _) = true
 | 
| 80 | | is_equals _ = false; | |
| 81 | ||
| 82 | ||
| 0 | 83 | (** implies **) | 
| 84 | ||
| 85 | fun mk_implies(A,B) = implies $ A $ B; | |
| 86 | ||
| 87 | fun dest_implies (Const("==>",_) $ A $ B)  =  (A,B)
 | |
| 88 |   | dest_implies A = raise TERM("dest_implies", [A]);
 | |
| 89 | ||
| 5041 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 90 | fun is_implies (Const ("==>", _) $ _ $ _) = true
 | 
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 91 | | is_implies _ = false; | 
| 
a1d0a6d555cd
Goals may now contain assumptions, which are not returned.
 nipkow parents: 
4822diff
changeset | 92 | |
| 4822 | 93 | |
| 0 | 94 | (** nested implications **) | 
| 95 | ||
| 96 | (* [A1,...,An], B goes to A1==>...An==>B *) | |
| 97 | fun list_implies ([], B) = B : term | |
| 98 | | list_implies (A::AS, B) = implies $ A $ list_implies(AS,B); | |
| 99 | ||
| 100 | (* A1==>...An==>B goes to [A1,...,An], where B is not an implication *) | |
| 101 | fun strip_imp_prems (Const("==>", _) $ A $ B) = A :: strip_imp_prems B
 | |
| 102 | | strip_imp_prems _ = []; | |
| 103 | ||
| 104 | (* A1==>...An==>B goes to B, where B is not an implication *) | |
| 105 | fun strip_imp_concl (Const("==>", _) $ A $ B) = strip_imp_concl B
 | |
| 106 | | strip_imp_concl A = A : term; | |
| 107 | ||
| 108 | (*Strip and return premises: (i, [], A1==>...Ai==>B) | |
| 9460 | 109 | goes to ([Ai, A(i-1),...,A1] , B) (REVERSED) | 
| 0 | 110 | if i<0 or else i too big then raises TERM*) | 
| 9460 | 111 | fun strip_prems (0, As, B) = (As, B) | 
| 112 |   | strip_prems (i, As, Const("==>", _) $ A $ B) =
 | |
| 113 | strip_prems (i-1, A::As, B) | |
| 0 | 114 |   | strip_prems (_, As, A) = raise TERM("strip_prems", A::As);
 | 
| 115 | ||
| 116 | (*Count premises -- quicker than (length ostrip_prems) *) | |
| 117 | fun count_prems (Const("==>", _) $ A $ B, n) = count_prems (B,n+1)
 | |
| 118 | | count_prems (_,n) = n; | |
| 119 | ||
| 4822 | 120 | |
| 0 | 121 | (** flex-flex constraints **) | 
| 122 | ||
| 64 
0bbe5d86cb38
logic/mk_equals,mk_flexpair: now calls fastype_of instead of type_of.
 lcp parents: 
0diff
changeset | 123 | (*Make a constraint.*) | 
| 
0bbe5d86cb38
logic/mk_equals,mk_flexpair: now calls fastype_of instead of type_of.
 lcp parents: 
0diff
changeset | 124 | fun mk_flexpair(t,u) = flexpair(fastype_of t) $ t $ u; | 
| 0 | 125 | |
| 126 | fun dest_flexpair (Const("=?=",_) $ t $ u)  =  (t,u)
 | |
| 127 |   | dest_flexpair t = raise TERM("dest_flexpair", [t]);
 | |
| 128 | ||
| 129 | (*make flexflex antecedents: ( [(a1,b1),...,(an,bn)] , C ) | |
| 130 | goes to (a1=?=b1) ==>...(an=?=bn)==>C *) | |
| 131 | fun list_flexpairs ([], A) = A | |
| 132 | | list_flexpairs ((t,u)::pairs, A) = | |
| 9460 | 133 | implies $ (mk_flexpair(t,u)) $ list_flexpairs(pairs,A); | 
| 0 | 134 | |
| 135 | (*Make the object-rule tpairs==>As==>B *) | |
| 136 | fun rule_of (tpairs, As, B) = list_flexpairs(tpairs, list_implies(As, B)); | |
| 137 | ||
| 9460 | 138 | (*Remove and return flexflex pairs: | 
| 139 | (a1=?=b1)==>...(an=?=bn)==>C to ( [(a1,b1),...,(an,bn)] , C ) | |
| 0 | 140 | [Tail recursive in order to return a pair of results] *) | 
| 141 | fun strip_flex_aux (pairs, Const("==>", _) $ (Const("=?=",_)$t$u) $ C) =
 | |
| 142 | strip_flex_aux ((t,u)::pairs, C) | |
| 143 | | strip_flex_aux (pairs,C) = (rev pairs, C); | |
| 144 | ||
| 145 | fun strip_flexpairs A = strip_flex_aux([], A); | |
| 146 | ||
| 147 | (*Discard flexflex pairs*) | |
| 148 | fun skip_flexpairs (Const("==>", _) $ (Const("=?=",_)$_$_) $ C) =
 | |
| 9460 | 149 | skip_flexpairs C | 
| 0 | 150 | | skip_flexpairs C = C; | 
| 151 | ||
| 9460 | 152 | (*strip a proof state (Horn clause): | 
| 0 | 153 | (a1==b1)==>...(am==bm)==>B1==>...Bn==>C | 
| 154 | goes to ( [(a1,b1),...,(am,bm)] , [B1,...,Bn] , C) *) | |
| 155 | fun strip_horn A = | |
| 9460 | 156 | let val (tpairs,horn) = strip_flexpairs A | 
| 0 | 157 | in (tpairs, strip_imp_prems horn, strip_imp_concl horn) end; | 
| 158 | ||
| 4822 | 159 | |
| 160 | (** definitions **) | |
| 161 | ||
| 162 | fun mk_cond_defpair As (lhs, rhs) = | |
| 163 | (case Term.head_of lhs of | |
| 164 | Const (name, _) => | |
| 165 | (Sign.base_name name ^ "_def", list_implies (As, mk_equals (lhs, rhs))) | |
| 166 |   | _ => raise TERM ("Malformed definition: head of lhs not a constant", [lhs, rhs]));
 | |
| 167 | ||
| 168 | fun mk_defpair lhs_rhs = mk_cond_defpair [] lhs_rhs; | |
| 169 | ||
| 170 | ||
| 398 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 171 | (** types as terms **) | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 172 | |
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 173 | fun mk_type ty = Const ("TYPE", itselfT ty);
 | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 174 | |
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 175 | fun dest_type (Const ("TYPE", Type ("itself", [ty]))) = ty
 | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 176 |   | dest_type t = raise TERM ("dest_type", [t]);
 | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 177 | |
| 4822 | 178 | |
| 447 | 179 | (** class constraints **) | 
| 398 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 180 | |
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 181 | fun mk_inclass (ty, c) = | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 182 | Const (Sign.const_of_class c, itselfT ty --> propT) $ mk_type ty; | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 183 | |
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 184 | fun dest_inclass (t as Const (c_class, _) $ ty) = | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 185 | ((dest_type ty, Sign.class_of_const c_class) | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 186 |         handle TERM _ => raise TERM ("dest_inclass", [t]))
 | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 187 |   | dest_inclass t = raise TERM ("dest_inclass", [t]);
 | 
| 
41f279b477e2
added mk_type, dest_type, mk_inclass, dest_inclass (for axclasses);
 wenzelm parents: 
210diff
changeset | 188 | |
| 0 | 189 | |
| 9460 | 190 | (** atomic goals **) | 
| 191 | ||
| 192 | val goal_const = Const ("Goal", propT --> propT);
 | |
| 193 | fun mk_goal t = goal_const $ t; | |
| 194 | ||
| 195 | fun dest_goal (Const ("Goal", _) $ t) = t
 | |
| 196 |   | dest_goal t = raise TERM ("dest_goal", [t]);
 | |
| 197 | ||
| 198 | ||
| 0 | 199 | (*** Low-level term operations ***) | 
| 200 | ||
| 201 | (*Does t occur in u? Or is alpha-convertible to u? | |
| 202 | The term t must contain no loose bound variables*) | |
| 4631 | 203 | fun t occs u = exists_subterm (fn s => t aconv s) u; | 
| 0 | 204 | |
| 205 | (*Close up a formula over all free variables by quantification*) | |
| 206 | fun close_form A = | |
| 4443 | 207 | list_all_free (sort_wrt fst (map dest_Free (term_frees A)), A); | 
| 0 | 208 | |
| 209 | ||
| 210 | (*** Specialized operations for resolution... ***) | |
| 211 | ||
| 212 | (*For all variables in the term, increment indexnames and lift over the Us | |
| 213 | result is ?Gidx(B.(lev+n-1),...,B.lev) where lev is abstraction level *) | |
| 9460 | 214 | fun incr_indexes (Us: typ list, inc:int) t = | 
| 215 | let fun incr (Var ((a,i), T), lev) = | |
| 216 | Unify.combound (Var((a, i+inc), Us---> incr_tvar inc T), | |
| 217 | lev, length Us) | |
| 218 | | incr (Abs (a,T,body), lev) = | |
| 219 | Abs (a, incr_tvar inc T, incr(body,lev+1)) | |
| 220 | | incr (Const(a,T),_) = Const(a, incr_tvar inc T) | |
| 221 | | incr (Free(a,T),_) = Free(a, incr_tvar inc T) | |
| 222 | | incr (f$t, lev) = incr(f,lev) $ incr(t,lev) | |
| 223 | | incr (t,lev) = t | |
| 0 | 224 | in incr(t,0) end; | 
| 225 | ||
| 226 | (*Make lifting functions from subgoal and increment. | |
| 227 | lift_abs operates on tpairs (unification constraints) | |
| 228 | lift_all operates on propositions *) | |
| 229 | fun lift_fns (B,inc) = | |
| 230 |   let fun lift_abs (Us, Const("==>", _) $ _ $ B) u = lift_abs (Us,B) u
 | |
| 9460 | 231 |         | lift_abs (Us, Const("all",_)$Abs(a,T,t)) u =
 | 
| 232 | Abs(a, T, lift_abs (T::Us, t) u) | |
| 233 | | lift_abs (Us, _) u = incr_indexes(rev Us, inc) u | |
| 0 | 234 |       fun lift_all (Us, Const("==>", _) $ A $ B) u =
 | 
| 9460 | 235 | implies $ A $ lift_all (Us,B) u | 
| 236 |         | lift_all (Us, Const("all",_)$Abs(a,T,t)) u =
 | |
| 237 | all T $ Abs(a, T, lift_all (T::Us,t) u) | |
| 238 | | lift_all (Us, _) u = incr_indexes(rev Us, inc) u; | |
| 0 | 239 | in (lift_abs([],B), lift_all([],B)) end; | 
| 240 | ||
| 241 | (*Strips assumptions in goal, yielding list of hypotheses. *) | |
| 242 | fun strip_assums_hyp (Const("==>", _) $ H $ B) = H :: strip_assums_hyp B
 | |
| 243 |   | strip_assums_hyp (Const("all",_)$Abs(a,T,t)) = strip_assums_hyp t
 | |
| 244 | | strip_assums_hyp B = []; | |
| 245 | ||
| 246 | (*Strips assumptions in goal, yielding conclusion. *) | |
| 247 | fun strip_assums_concl (Const("==>", _) $ H $ B) = strip_assums_concl B
 | |
| 248 |   | strip_assums_concl (Const("all",_)$Abs(a,T,t)) = strip_assums_concl t
 | |
| 249 | | strip_assums_concl B = B; | |
| 250 | ||
| 251 | (*Make a list of all the parameters in a subgoal, even if nested*) | |
| 252 | fun strip_params (Const("==>", _) $ H $ B) = strip_params B
 | |
| 253 |   | strip_params (Const("all",_)$Abs(a,T,t)) = (a,T) :: strip_params t
 | |
| 254 | | strip_params B = []; | |
| 255 | ||
| 10816 | 256 | (*test for HHF normal form*) | 
| 257 | fun is_norm_hhf (Const ("==>", _) $ _ $ (Const ("all", _) $ _)) = false
 | |
| 258 | | is_norm_hhf (t $ u) = is_norm_hhf t andalso is_norm_hhf u | |
| 259 | | is_norm_hhf (Abs (_, _, t)) = is_norm_hhf t | |
| 260 | | is_norm_hhf _ = true; | |
| 261 | ||
| 9667 | 262 | (*test for meta connectives in prems of a 'subgoal'*) | 
| 263 | fun has_meta_prems prop i = | |
| 264 | let | |
| 265 |     fun is_meta (Const ("==>", _) $ _ $ _) = true
 | |
| 10442 | 266 |       | is_meta (Const ("==", _) $ _ $ _) = true
 | 
| 9667 | 267 |       | is_meta (Const ("all", _) $ _) = true
 | 
| 268 | | is_meta _ = false; | |
| 269 | val horn = skip_flexpairs prop; | |
| 270 | in | |
| 271 | (case strip_prems (i, [], horn) of | |
| 272 | (B :: _, _) => exists is_meta (strip_assums_hyp B) | |
| 273 | | _ => false) handle TERM _ => false | |
| 274 | end; | |
| 9483 | 275 | |
| 0 | 276 | (*Removes the parameters from a subgoal and renumber bvars in hypotheses, | 
| 9460 | 277 | where j is the total number of parameters (precomputed) | 
| 0 | 278 | If n>0 then deletes assumption n. *) | 
| 9460 | 279 | fun remove_params j n A = | 
| 0 | 280 | if j=0 andalso n<=0 then A (*nothing left to do...*) | 
| 281 | else case A of | |
| 9460 | 282 |         Const("==>", _) $ H $ B =>
 | 
| 283 | if n=1 then (remove_params j (n-1) B) | |
| 284 | else implies $ (incr_boundvars j H) $ (remove_params j (n-1) B) | |
| 0 | 285 |       | Const("all",_)$Abs(a,T,t) => remove_params (j-1) n t
 | 
| 286 |       | _ => if n>0 then raise TERM("remove_params", [A])
 | |
| 287 | else A; | |
| 288 | ||
| 289 | (** Auto-renaming of parameters in subgoals **) | |
| 290 | ||
| 291 | val auto_rename = ref false | |
| 292 | and rename_prefix = ref "ka"; | |
| 293 | ||
| 294 | (*rename_prefix is not exported; it is set by this function.*) | |
| 295 | fun set_rename_prefix a = | |
| 4693 | 296 | if a<>"" andalso forall Symbol.is_letter (Symbol.explode a) | 
| 0 | 297 | then (rename_prefix := a; auto_rename := true) | 
| 298 | else error"rename prefix must be nonempty and consist of letters"; | |
| 299 | ||
| 300 | (*Makes parameters in a goal have distinctive names (not guaranteed unique!) | |
| 301 | A name clash could cause the printer to rename bound vars; | |
| 302 | then res_inst_tac would not work properly.*) | |
| 303 | fun rename_vars (a, []) = [] | |
| 304 | | rename_vars (a, (_,T)::vars) = | |
| 305 | (a,T) :: rename_vars (bump_string a, vars); | |
| 306 | ||
| 307 | (*Move all parameters to the front of the subgoal, renaming them apart; | |
| 308 | if n>0 then deletes assumption n. *) | |
| 309 | fun flatten_params n A = | |
| 310 | let val params = strip_params A; | |
| 9460 | 311 | val vars = if !auto_rename | 
| 312 | then rename_vars (!rename_prefix, params) | |
| 313 | else ListPair.zip (variantlist(map #1 params,[]), | |
| 314 | map #2 params) | |
| 0 | 315 | in list_all (vars, remove_params (length vars) n A) | 
| 316 | end; | |
| 317 | ||
| 318 | (*Makes parameters in a goal have the names supplied by the list cs.*) | |
| 319 | fun list_rename_params (cs, Const("==>", _) $ A $ B) =
 | |
| 320 | implies $ A $ list_rename_params (cs, B) | |
| 9460 | 321 |   | list_rename_params (c::cs, Const("all",_)$Abs(_,T,t)) =
 | 
| 0 | 322 | all T $ Abs(c, T, list_rename_params (cs, t)) | 
| 323 | | list_rename_params (cs, B) = B; | |
| 324 | ||
| 9684 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 325 | (*Strips assumptions in goal yielding ( [HPn,...,HP1], [xm,...,x1], B ). | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 326 | Where HPi has the form (Hi,nparams_i) and x1...xm are the parameters. | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 327 | We need nparams_i only when the parameters aren't flattened; then we | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 328 | must call incr_boundvars to make up the difference. See assum_pairs. | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 329 | Without this refinement we can get the wrong answer, e.g. by | 
| 10816 | 330 | Goal "!!f. EX B. Q(f,B) ==> (!!y. P(f,y))"; | 
| 331 | by (etac exE 1); | |
| 9684 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 332 | *) | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 333 | fun strip_assums_aux (HPs, params, Const("==>", _) $ H $ B) =
 | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 334 | strip_assums_aux ((H,length params)::HPs, params, B) | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 335 |   | strip_assums_aux (HPs, params, Const("all",_)$Abs(a,T,t)) =
 | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 336 | strip_assums_aux (HPs, (a,T)::params, t) | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 337 | | strip_assums_aux (HPs, params, B) = (HPs, params, B); | 
| 0 | 338 | |
| 339 | fun strip_assums A = strip_assums_aux ([],[],A); | |
| 340 | ||
| 341 | ||
| 342 | (*Produces disagreement pairs, one for each assumption proof, in order. | |
| 343 | A is the first premise of the lifted rule, and thus has the form | |
| 344 | H1 ==> ... Hk ==> B and the pairs are (H1,B),...,(Hk,B) *) | |
| 345 | fun assum_pairs A = | |
| 9684 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 346 | let val (HPs, params, B) = strip_assums A | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 347 | val nparams = length params | 
| 0 | 348 | val D = Unify.rlist_abs(params, B) | 
| 10816 | 349 | fun incr_hyp(H,np) = | 
| 350 | Unify.rlist_abs(params, incr_boundvars (nparams-np) H) | |
| 9460 | 351 | fun pairrev ([],pairs) = pairs | 
| 9684 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 352 | | pairrev ((H,np)::HPs, pairs) = | 
| 
6b7d7635a062
fixed strip_assums and assum_pairs, restoring them (essentially) to their
 paulson parents: 
9667diff
changeset | 353 | pairrev(HPs, (incr_hyp(H,np),D) :: pairs) | 
| 10816 | 354 | in pairrev (HPs,[]) | 
| 0 | 355 | end; | 
| 356 | ||
| 357 | (*Converts Frees to Vars and TFrees to TVars so that axioms can be written | |
| 358 | without (?) everywhere*) | |
| 359 | fun varify (Const(a,T)) = Const(a, Type.varifyT T) | |
| 360 | | varify (Free(a,T)) = Var((a,0), Type.varifyT T) | |
| 361 | | varify (Var(ixn,T)) = Var(ixn, Type.varifyT T) | |
| 362 | | varify (Abs (a,T,body)) = Abs (a, Type.varifyT T, varify body) | |
| 363 | | varify (f$t) = varify f $ varify t | |
| 364 | | varify t = t; | |
| 365 | ||
| 546 | 366 | (*Inverse of varify. Converts axioms back to their original form.*) | 
| 585 | 367 | fun unvarify (Const(a,T)) = Const(a, Type.unvarifyT T) | 
| 368 | | unvarify (Var((a,0), T)) = Free(a, Type.unvarifyT T) | |
| 369 | | unvarify (Var(ixn,T)) = Var(ixn, Type.unvarifyT T) (*non-0 index!*) | |
| 370 | | unvarify (Abs (a,T,body)) = Abs (a, Type.unvarifyT T, unvarify body) | |
| 546 | 371 | | unvarify (f$t) = unvarify f $ unvarify t | 
| 372 | | unvarify t = t; | |
| 373 | ||
| 0 | 374 | end; |