src/Pure/Isar/isar_syn.ML
changeset 40965 54b6c9e1c157
parent 40960 9e54eb514a46
child 41229 d797baa3d57c
--- a/src/Pure/Isar/isar_syn.ML	Sun Dec 05 13:42:58 2010 +0100
+++ b/src/Pure/Isar/isar_syn.ML	Sun Dec 05 14:02:16 2010 +0100
@@ -513,13 +513,6 @@
     (Parse.begin >> K Proof.begin_notepad);
 
 val _ =
-  Outer_Syntax.local_theory_to_proof "example_proof"
-    "example proof body, without any result" Keyword.thy_schematic_goal
-    (Scan.succeed
-      (Specification.theorem_cmd "" NONE (K I)
-        Attrib.empty_binding [] (Element.Shows []) false #> Proof.enter_forward));
-
-val _ =
   Outer_Syntax.command "have" "state local goal"
     (Keyword.tag_proof Keyword.prf_goal)
     (Parse_Spec.statement >> ((Toplevel.print oo Toplevel.proof') o Isar_Cmd.have));