removed obsolete/unused Proof.match_bind;
authorwenzelm
Sun, 25 Apr 2010 16:10:05 +0200
changeset 36324 7cd5057a5bb8
parent 36323 655e2d74de3a
child 36325 8715343af626
removed obsolete/unused Proof.match_bind;
src/Pure/Isar/proof.ML
--- a/src/Pure/Isar/proof.ML	Sun Apr 25 15:52:03 2010 +0200
+++ b/src/Pure/Isar/proof.ML	Sun Apr 25 16:10:05 2010 +0200
@@ -41,8 +41,6 @@
   val raw_goal: state -> {context: context, facts: thm list, goal: thm}
   val goal: state -> {context: context, facts: thm list, goal: thm}
   val simple_goal: state -> {context: context, goal: thm}
-  val match_bind: (term list * term) list -> state -> state
-  val match_bind_cmd: (string list * string) list -> state -> state
   val let_bind: (term list * term) list -> state -> state
   val let_bind_cmd: (string list * string) list -> state -> state
   val fix: (binding * typ option * mixfix) list -> state -> state
@@ -523,22 +521,20 @@
 
 (** context elements **)
 
-(* bindings *)
+(* let bindings *)
 
 local
 
 fun gen_bind bind args state =
   state
   |> assert_forward
-  |> map_context (bind args #> snd)
+  |> map_context (bind true args #> snd)
   |> put_facts NONE;
 
 in
 
-val match_bind = gen_bind (ProofContext.match_bind_i false);
-val match_bind_cmd = gen_bind (ProofContext.match_bind false);
-val let_bind = gen_bind (ProofContext.match_bind_i true);
-val let_bind_cmd = gen_bind (ProofContext.match_bind true);
+val let_bind = gen_bind ProofContext.match_bind_i;
+val let_bind_cmd = gen_bind ProofContext.match_bind;
 
 end;