src/FOLP/simp.ML
changeset 32952 aeb1e44fbc19
parent 32740 9dd0a2f83429
child 32957 675c0c7e6a37
--- a/src/FOLP/simp.ML	Thu Oct 15 23:10:35 2009 +0200
+++ b/src/FOLP/simp.ML	Thu Oct 15 23:28:10 2009 +0200
@@ -432,8 +432,8 @@
 fun add_asms(ss,thm,a,anet,ats,cs) =
     let val As = strip_varify(nth_subgoal i thm, a, []);
         val thms = map (trivial o cterm_of(Thm.theory_of_thm thm)) As;
-        val new_rws = List.concat(map mk_rew_rules thms);
-        val rwrls = map mk_trans (List.concat(map mk_rew_rules thms));
+        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
     in  if !tracing andalso not(null new_rws)
         then writeln (cat_lines
@@ -589,7 +589,7 @@
     val T' = Logic.incr_tvar 9 T;
 in mk_cong_type thy (Const(f,T'),T') end;
 
-fun mk_congs thy = List.concat o map (mk_cong_thy thy);
+fun mk_congs thy = maps (mk_cong_thy thy);
 
 fun mk_typed_congs thy =
 let
@@ -599,7 +599,7 @@
       val t = case Sign.const_type thy f of
                   SOME(_) => Const(f,T) | NONE => Free(f,T)
     in (t,T) end
-in List.concat o map (mk_cong_type thy o readfT) end;
+in maps (mk_cong_type thy o readfT) end;
 
 end;
 end;