src/Doc/IsarImplementation/Logic.thy
changeset 53200 09e8c42dbb06
parent 53071 1958a5e65ea5
child 54883 dd04a8b654fc
equal deleted inserted replaced
53199:7a9fe70c8b0a 53200:09e8c42dbb06
  1171   THM}.
  1171   THM}.
  1172 
  1172 
  1173   This corresponds to the rule attribute @{attribute THEN} in Isar
  1173   This corresponds to the rule attribute @{attribute THEN} in Isar
  1174   source language.
  1174   source language.
  1175 
  1175 
  1176   \item @{text "rule\<^sub>1 RS rule\<^sub>2"} abbreviates @{text "rule\<^sub>1 RS (1,
  1176   \item @{text "rule\<^sub>1 RS rule\<^sub>2"} abbreviates @{text "rule\<^sub>1 RSN (1,
  1177   rule\<^sub>2)"}.
  1177   rule\<^sub>2)"}.
  1178 
  1178 
  1179   \item @{text "rules\<^sub>1 RLN (i, rules\<^sub>2)"} joins lists of rules.  For
  1179   \item @{text "rules\<^sub>1 RLN (i, rules\<^sub>2)"} joins lists of rules.  For
  1180   every @{text "rule\<^sub>1"} in @{text "rules\<^sub>1"} and @{text "rule\<^sub>2"} in
  1180   every @{text "rule\<^sub>1"} in @{text "rules\<^sub>1"} and @{text "rule\<^sub>2"} in
  1181   @{text "rules\<^sub>2"}, it resolves the conclusion of @{text "rule\<^sub>1"} with
  1181   @{text "rules\<^sub>2"}, it resolves the conclusion of @{text "rule\<^sub>1"} with