eliminated dead code;
authorwenzelm
Tue, 09 Jun 2015 15:28:06 +0200
changeset 60405 990c9fea6773
parent 60404 422b63ef0147
child 60406 12cc54fac9b0
eliminated dead code;
src/Pure/Isar/isar_cmd.ML
--- a/src/Pure/Isar/isar_cmd.ML	Tue Jun 09 13:42:58 2015 +0200
+++ b/src/Pure/Isar/isar_cmd.ML	Tue Jun 09 15:28:06 2015 +0200
@@ -173,17 +173,6 @@
   |> Context.proof_map;
 
 
-(* goals *)
-
-fun goal opt_chain goal stmt int =
-  opt_chain #> goal NONE (K I) stmt int;
-
-val have = goal I Proof.have_cmd;
-val hence = goal Proof.chain Proof.have_cmd;
-val show = goal I Proof.show_cmd;
-val thus = goal Proof.chain Proof.show_cmd;
-
-
 (* local endings *)
 
 fun local_qed m = Toplevel.proof (Proof.local_qed (m, true));