doc-src/IsarImplementation/Thy/Logic.thy
changeset 47498 e3fc50c7da13
parent 47174 b9b2e183e94d
equal deleted inserted replaced
47497:c78c6e1ec75d 47498:e3fc50c7da13
  1121   \item @{text "[rule\<^sub>1, \<dots>, rule\<^sub>n] MRS rule"} resolves @{text "rule\<^isub>i"}
  1121   \item @{text "[rule\<^sub>1, \<dots>, rule\<^sub>n] MRS rule"} resolves @{text "rule\<^isub>i"}
  1122   against premise @{text "i"} of @{text "rule"}, for @{text "i = n, \<dots>,
  1122   against premise @{text "i"} of @{text "rule"}, for @{text "i = n, \<dots>,
  1123   1"}.  By working from right to left, newly emerging premises are
  1123   1"}.  By working from right to left, newly emerging premises are
  1124   concatenated in the result, without interfering.
  1124   concatenated in the result, without interfering.
  1125 
  1125 
  1126   \item @{text "rule OF rules"} abbreviates @{text "rules MRS rule"}.
  1126   \item @{text "rule OF rules"} is an alternative notation for @{text
       
  1127   "rules MRS rule"}, which makes rule composition look more like
       
  1128   function application.  Note that the argument @{text "rules"} need
       
  1129   not be atomic.
  1127 
  1130 
  1128   This corresponds to the rule attribute @{attribute OF} in Isar
  1131   This corresponds to the rule attribute @{attribute OF} in Isar
  1129   source language.
  1132   source language.
  1130 
  1133 
  1131   \end{description}
  1134   \end{description}