oops;
authorwenzelm
Wed, 20 Jul 2016 16:18:10 +0200
changeset 63529 58980a8b2faf
parent 63528 0f39f59317c1
child 63530 045490f55f69
oops;
src/Doc/Isar_Ref/Proof.thy
--- a/src/Doc/Isar_Ref/Proof.thy	Wed Jul 20 16:02:00 2016 +0200
+++ b/src/Doc/Isar_Ref/Proof.thy	Wed Jul 20 16:18:10 2016 +0200
@@ -189,8 +189,8 @@
   "and"}; the resulting list of current facts consists of all of these
   concatenated.
 
-  A structured assumption like \<^theory_text>\<open>assume "B x" and "A x" for x\<close> is equivalent
-  to \<^theory_text>\<open>assume "\<And>x. A x \<Longrightarrow> B x"\<close>, but vacuous quantification is avoided: a
+  A structured assumption like \<^theory_text>\<open>assume "B x" if "A x" for x\<close> is equivalent to
+  \<^theory_text>\<open>assume "\<And>x. A x \<Longrightarrow> B x"\<close>, but vacuous quantification is avoided: a
   for-context only effects propositions according to actual use of variables.
 
   \<^descr> \<^theory_text>\<open>define x where "x = t"\<close> introduces a local (non-polymorphic) definition.