doc-src/IsarRef/Thy/Proof.thy
changeset 47498 e3fc50c7da13
parent 47484 e94cc23d434a
equal deleted inserted replaced
47497:c78c6e1ec75d 47498:e3fc50c7da13
   782   "Pure.intro"}.
   782   "Pure.intro"}.
   783   
   783   
   784   \item @{attribute (Pure) rule}~@{text del} undeclares introduction,
   784   \item @{attribute (Pure) rule}~@{text del} undeclares introduction,
   785   elimination, or destruct rules.
   785   elimination, or destruct rules.
   786   
   786   
   787   \item @{attribute OF}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} applies some
   787   \item @{attribute OF}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} applies some theorem to all
   788   theorem to all of the given rules @{text "a\<^sub>1, \<dots>, a\<^sub>n"}
   788   of the given rules @{text "a\<^sub>1, \<dots>, a\<^sub>n"} in canonical right-to-left
   789   (in parallel).  This corresponds to the @{ML_op "MRS"} operation in
   789   order, which means that premises stemming from the @{text "a\<^sub>i"}
   790   ML, but note the reversed order.  Positions may be effectively
   790   emerge in parallel in the result, without interfering with each
   791   skipped by including ``@{text _}'' (underscore) as argument.
   791   other.  In many practical situations, the @{text "a\<^sub>i"} do not have
       
   792   premises themselves, so @{text "rule [OF a\<^sub>1 \<dots> a\<^sub>n]"} can be actually
       
   793   read as functional application (modulo unification).
       
   794 
       
   795   Argument positions may be effectively skipped by using ``@{text _}''
       
   796   (underscore), which refers to the propositional identity rule in the
       
   797   Pure theory.
   792   
   798   
   793   \item @{attribute of}~@{text "t\<^sub>1 \<dots> t\<^sub>n"} performs positional
   799   \item @{attribute of}~@{text "t\<^sub>1 \<dots> t\<^sub>n"} performs positional
   794   instantiation of term variables.  The terms @{text "t\<^sub>1, \<dots>, t\<^sub>n"} are
   800   instantiation of term variables.  The terms @{text "t\<^sub>1, \<dots>, t\<^sub>n"} are
   795   substituted for any schematic variables occurring in a theorem from
   801   substituted for any schematic variables occurring in a theorem from
   796   left to right; ``@{text _}'' (underscore) indicates to skip a
   802   left to right; ``@{text _}'' (underscore) indicates to skip a