doc-src/IsarRef/Thy/Generic.thy
changeset 27071 614c045c5fd4
parent 27044 c4eaa7140532
child 27092 3d79bbdaf2ef
equal deleted inserted replaced
27070:3fcfa8cfa0d5 27071:614c045c5fd4
   210   \item [@{method subst}~@{text "(i \<dots> j) eq"}] performs several
   210   \item [@{method subst}~@{text "(i \<dots> j) eq"}] performs several
   211   substitutions in the conclusion. The numbers @{text i} to @{text j}
   211   substitutions in the conclusion. The numbers @{text i} to @{text j}
   212   indicate the positions to substitute at.  Positions are ordered from
   212   indicate the positions to substitute at.  Positions are ordered from
   213   the top of the term tree moving down from left to right. For
   213   the top of the term tree moving down from left to right. For
   214   example, in @{text "(a + b) + (c + d)"} there are three positions
   214   example, in @{text "(a + b) + (c + d)"} there are three positions
   215   where commutativity of @{text "+"} is applicable: 1 refers to the
   215   where commutativity of @{text "+"} is applicable: 1 refers to
   216   whole term, 2 to @{text "a + b"} and 3 to @{text "c + d"}.
   216   @{text "a + b"}, 2 to the whole term, and 3 to @{text "c + d"}.
   217 
   217 
   218   If the positions in the list @{text "(i \<dots> j)"} are non-overlapping
   218   If the positions in the list @{text "(i \<dots> j)"} are non-overlapping
   219   (e.g.\ @{text "(2 3)"} in @{text "(a + b) + (c + d)"}) you may
   219   (e.g.\ @{text "(2 3)"} in @{text "(a + b) + (c + d)"}) you may
   220   assume all substitutions are performed simultaneously.  Otherwise
   220   assume all substitutions are performed simultaneously.  Otherwise
   221   the behaviour of @{text subst} is not specified.
   221   the behaviour of @{text subst} is not specified.
   222 
   222 
   223   \item [@{method subst}~@{text "(asm) (i \<dots> j) eq"}] performs the
   223   \item [@{method subst}~@{text "(asm) (i \<dots> j) eq"}] performs the
   224   substitutions in the assumptions.  Positions @{text "1 \<dots> i\<^sub>1"}
   224   substitutions in the assumptions. The positions refer to the
   225   refer to assumption 1, positions @{text "i\<^sub>1 + 1 \<dots> i\<^sub>2"}
   225   assumptions in order from left to right.  For example, given in a
   226   to assumption 2, and so on.
   226   goal of the form @{text "P (a + b) \<Longrightarrow> P (c + d) \<Longrightarrow> \<dots>"}, position 1 of
       
   227   commutativity of @{text "+"} is the subterm @{text "a + b"} and
       
   228   position 2 is the subterm @{text "c + d"}.
   227 
   229 
   228   \item [@{method hypsubst}] performs substitution using some
   230   \item [@{method hypsubst}] performs substitution using some
   229   assumption; this only works for equations of the form @{text "x =
   231   assumption; this only works for equations of the form @{text "x =
   230   t"} where @{text x} is a free or bound variable.
   232   t"} where @{text x} is a free or bound variable.
   231 
   233