src/Pure/Isar/isar_thy.ML
changeset 8615 419166fa66d0
parent 8588 b7c3f264f8ac
child 8681 957a5fe9b212
--- a/src/Pure/Isar/isar_thy.ML	Thu Mar 30 14:24:46 2000 +0200
+++ b/src/Pure/Isar/isar_thy.ML	Thu Mar 30 14:25:35 2000 +0200
@@ -76,8 +76,8 @@
   val chain: Comment.text -> ProofHistory.T -> ProofHistory.T
   val fix: ((string list * string option) * Comment.text) list -> ProofHistory.T -> ProofHistory.T
   val fix_i: ((string list * typ option) * Comment.text) list -> ProofHistory.T -> ProofHistory.T
-  val match_bind: ((string list * string) * Comment.text) list -> ProofHistory.T -> ProofHistory.T
-  val match_bind_i: ((term list * term) * Comment.text) list -> ProofHistory.T -> ProofHistory.T
+  val let_bind: ((string list * string) * Comment.text) list -> ProofHistory.T -> ProofHistory.T
+  val let_bind_i: ((term list * term) * Comment.text) list -> ProofHistory.T -> ProofHistory.T
   val invoke_case: (string * Args.src list) * Comment.text -> ProofHistory.T -> ProofHistory.T
   val invoke_case_i: (string * Proof.context attribute list) * Comment.text
     -> ProofHistory.T -> ProofHistory.T
@@ -288,8 +288,8 @@
 
 val fix = ProofHistory.apply o Proof.fix o map Comment.ignore;
 val fix_i = ProofHistory.apply o Proof.fix_i o map Comment.ignore;
-val match_bind = ProofHistory.apply o Proof.match_bind o map Comment.ignore;
-val match_bind_i = ProofHistory.apply o Proof.match_bind_i o map Comment.ignore;
+val let_bind = ProofHistory.apply o Proof.let_bind o map Comment.ignore;
+val let_bind_i = ProofHistory.apply o Proof.let_bind_i o map Comment.ignore;
 
 fun invoke_case ((name, src), comment_ignore) = ProofHistory.apply (fn state =>
   Proof.invoke_case (name, map (Attrib.local_attribute (Proof.theory_of state)) src) state);