src/Doc/Isar_Ref/Spec.thy
changeset 61853 fb7756087101
parent 61823 5daa82ba4078
child 61891 76189756ff65
--- a/src/Doc/Isar_Ref/Spec.thy	Tue Dec 15 16:57:10 2015 +0100
+++ b/src/Doc/Isar_Ref/Spec.thy	Wed Dec 16 16:31:36 2015 +0100
@@ -1066,7 +1066,7 @@
 (*<*)experiment begin(*>*)
   attribute_setup my_rule =
     \<open>Attrib.thms >> (fn ths =>
-      Thm.rule_attribute
+      Thm.rule_attribute ths
         (fn context: Context.generic => fn th: thm =>
           let val th' = th OF ths
           in th' end))\<close>