doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 42626 6ac8c55c657e
parent 42617 77d239840285
child 42627 8749742785b8
--- a/doc-src/IsarRef/Thy/HOL_Specific.thy	Mon May 02 20:14:19 2011 +0200
+++ b/doc-src/IsarRef/Thy/HOL_Specific.thy	Mon May 02 20:34:34 2011 +0200
@@ -896,7 +896,7 @@
   ``@{text "!"}'' indicator refers to ``safe'' rules, which may be
   applied aggressively (without considering back-tracking later).
   Rules declared with ``@{text "?"}'' are ignored in proof search (the
-  single-step @{method rule} method still observes these).  An
+  single-step @{method (Pure) rule} method still observes these).  An
   explicit weight annotation may be given as well; otherwise the
   number of rule premises will be taken into account here.
 *}
@@ -1419,7 +1419,7 @@
     @{command_def (HOL) "code_library"} & : & @{text "theory \<rightarrow> theory"} \\
     @{command_def (HOL) "consts_code"} & : & @{text "theory \<rightarrow> theory"} \\
     @{command_def (HOL) "types_code"} & : & @{text "theory \<rightarrow> theory"} \\
-    @{attribute_def (HOL) code} & : & @{text attribute} \\
+    @{attribute_def code} & : & @{text attribute} \\
   \end{matharray}
 
   @{rail "
@@ -1452,7 +1452,7 @@
   attachment: 'attach' modespec? '{' @{syntax text} '}'
   ;
 
-  @@{attribute (HOL) code} (name)?
+  @@{attribute code} name?
   "}
 *}