src/Doc/Isar_Ref/Proof.thy
changeset 59783 00b62aa9f430
parent 59660 49e498cedd02
child 59785 4e6ab5831cc0
--- a/src/Doc/Isar_Ref/Proof.thy	Mon Mar 23 15:54:41 2015 +0100
+++ b/src/Doc/Isar_Ref/Proof.thy	Mon Mar 23 15:55:41 2015 +0100
@@ -432,7 +432,7 @@
   @{rail \<open>
     (@@{command lemma} | @@{command theorem} | @@{command corollary} |
      @@{command schematic_lemma} | @@{command schematic_theorem} |
-     @@{command schematic_corollary}) @{syntax target}? (goal | longgoal)
+     @@{command schematic_corollary}) (goal | longgoal)
     ;
     (@@{command have} | @@{command show} | @@{command hence} | @@{command thus}) goal
     ;
@@ -935,8 +935,7 @@
   \end{matharray}
 
   @{rail \<open>
-    @@{command method_setup} @{syntax target}?
-      @{syntax name} '=' @{syntax text} @{syntax text}?
+    @@{command method_setup} @{syntax name} '=' @{syntax text} @{syntax text}?
   \<close>}
 
   \begin{description}