src/HOL/Isar_examples/BasicLogic.thy
changeset 6881 91a2c8b8269a
parent 6746 cf6ad8d22793
child 6892 4a905b4a39c8
--- a/src/HOL/Isar_examples/BasicLogic.thy	Thu Jul 01 21:28:49 1999 +0200
+++ b/src/HOL/Isar_examples/BasicLogic.thy	Thu Jul 01 21:29:53 1999 +0200
@@ -106,7 +106,7 @@
   proof (rule exE);
     fix a;
     assume "P(f(a))" (is "P(??witness)");
-    show ??thesis; by (rule exI [with P ??witness]);
+    show ??thesis; by (rule exI [of P ??witness]);
   qed;
 qed;