src/FOLP/simp.ML
changeset 33339 d41f77196338
parent 33317 b4534348b8fd
child 33955 fff6f11b1f09
--- a/src/FOLP/simp.ML	Thu Oct 29 23:49:55 2009 +0100
+++ b/src/FOLP/simp.ML	Thu Oct 29 23:56:33 2009 +0100
@@ -66,7 +66,7 @@
 fun eq_brl ((b1 : bool, th1), (b2, th2)) = b1 = b2 andalso Thm.eq_thm_prop (th1, th2);
 
 (*insert a thm in a discrimination net by its lhs*)
-fun lhs_insert_thm (th,net) =
+fun lhs_insert_thm th net =
     Net.insert_term eq_brl (lhs_of (concl_of th), (false,th)) net
     handle  Net.INSERT => net;
 
@@ -434,7 +434,7 @@
         val thms = map (trivial o cterm_of(Thm.theory_of_thm thm)) As;
         val new_rws = maps mk_rew_rules thms;
         val rwrls = map mk_trans (maps mk_rew_rules thms);
-        val anet' = List.foldr lhs_insert_thm anet rwrls
+        val anet' = fold_rev lhs_insert_thm rwrls anet;
     in  if !tracing andalso not(null new_rws)
         then writeln (cat_lines
           ("Adding rewrites:" :: map Display.string_of_thm_without_context new_rws))