TFL/rules.new.sml
changeset 3391 5e45dd3b64e9
parent 3379 7091ffa99c93
child 3405 2cccd0e3e9ea
--- a/TFL/rules.new.sml	Tue Jun 03 10:56:04 1997 +0200
+++ b/TFL/rules.new.sml	Tue Jun 03 11:08:08 1997 +0200
@@ -6,7 +6,7 @@
 Emulation of HOL inference rules for TFL
 *)
 
-structure FastRules : Rules_sig = 
+structure Rules : Rules_sig = 
 struct
 
 open Utils;
@@ -17,7 +17,7 @@
 structure D = Dcterm;
 
 
-fun RULES_ERR{func,mesg} = Utils.ERR{module = "FastRules",func=func,mesg=mesg};
+fun RULES_ERR{func,mesg} = Utils.ERR{module = "Rules",func=func,mesg=mesg};
 
 
 fun cconcl thm = D.drop_prop(#prop(crep_thm thm));
@@ -502,7 +502,7 @@
                 val (f,args) = S.strip_comb (get_lhs eq)
                 val (vstrl,_) = S.strip_abs f
                 val names  = map (#1 o dest_Free)
-                                 (variants (S.free_vars body) vstrl)
+                                 (variants (term_frees body) vstrl)
             in get (rst, n+1, (names,n)::L)
             end handle _ => get (rst, n+1, L);
 
@@ -750,8 +750,8 @@
               val dummy = print_thms "cntxt:\n" cntxt
               val {prop = Const("==>",_) $ (Const("Trueprop",_) $ A) $ _,
                    sign,...} = rep_thm thm
-              fun genl tm = let val vlist = U.set_diff (curry(op aconv))
-                                           (add_term_frees(tm,[])) [func,R]
+              fun genl tm = let val vlist = gen_rems (op aconv)
+                                           (add_term_frees(tm,[]), [func,R])
                             in U.itlist Forall vlist tm
                             end
               (*--------------------------------------------------------------