doc-src/IsarRef/Thy/Spec.thy
changeset 30546 b3b1f4184ae4
parent 30526 7f9a9ec1c94d
child 31047 c13b0406c039
equal deleted inserted replaced
30545:8209a7196389 30546:b3b1f4184ae4
   876       Attrib.thms >> (fn ths =>
   876       Attrib.thms >> (fn ths =>
   877         Thm.rule_attribute (fn context: Context.generic => fn th: thm =>
   877         Thm.rule_attribute (fn context: Context.generic => fn th: thm =>
   878           let val th' = th OF ths
   878           let val th' = th OF ths
   879           in th' end)) *}  "my rule"
   879           in th' end)) *}  "my rule"
   880 
   880 
   881     attribute_setup my_declatation = {*
   881     attribute_setup my_declaration = {*
   882       Attrib.thms >> (fn ths =>
   882       Attrib.thms >> (fn ths =>
   883         Thm.declaration_attribute (fn th: thm => fn context: Context.generic =>
   883         Thm.declaration_attribute (fn th: thm => fn context: Context.generic =>
   884           let val context' = context
   884           let val context' = context
   885           in context' end)) *}  "my declaration"
   885           in context' end)) *}  "my declaration"
   886 
   886