src/Pure/simplifier.ML
changeset 46776 8575cc482dfb
parent 46465 5ba52c337cd0
child 47001 a0e370d3d149
--- a/src/Pure/simplifier.ML	Sat Mar 03 21:43:59 2012 +0100
+++ b/src/Pure/simplifier.ML	Sat Mar 03 21:52:15 2012 +0100
@@ -315,7 +315,7 @@
   (Args.context -- Scan.lift add_del) :|-- (fn (ctxt, decl) =>
     Scan.repeat1 (Scan.lift (Args.named_attribute (decl o the_simproc ctxt o check_simproc ctxt))))
   >> (fn atts => Thm.declaration_attribute (fn th =>
-        Library.apply (map (fn att => Thm.attribute_declaration (Morphism.form att) th) atts)));
+        fold (fn att => Thm.attribute_declaration (Morphism.form att) th) atts));
 
 end;