src/Pure/Isar/interpretation.ML
changeset 62680 646b84666a56
parent 61890 f6ded81f5690
child 63068 8b9401bfd9fd
--- a/src/Pure/Isar/interpretation.ML	Mon Mar 21 11:54:45 2016 +0100
+++ b/src/Pure/Isar/interpretation.ML	Mon Mar 21 19:57:56 2016 +0100
@@ -11,10 +11,8 @@
   type 'a rewrites = (Attrib.binding * 'a) list
 
   (*interpretation in proofs*)
-  val interpret: Expression.expression_i ->
-    term rewrites -> bool -> Proof.state -> Proof.state
-  val interpret_cmd: Expression.expression ->
-    string rewrites -> bool -> Proof.state -> Proof.state
+  val interpret: Expression.expression_i -> term rewrites -> Proof.state -> Proof.state
+  val interpret_cmd: Expression.expression -> string rewrites -> Proof.state -> Proof.state
 
   (*interpretation in local theories*)
   val interpretation: Expression.expression_i ->
@@ -160,7 +158,7 @@
 
 local
 
-fun gen_interpret prep_interpretation expression raw_eqns int state =
+fun gen_interpret prep_interpretation expression raw_eqns state =
   let
     val _ = Proof.assert_forward_or_chain state;
     val ctxt = Proof.context_of state;
@@ -168,7 +166,7 @@
       Proof.map_context (after_qed witss eqns) #> Proof.reset_facts;
     fun setup_proof after_qed propss eqns goal_ctxt =
       Element.witness_local_proof_eqs (lift_after_qed after_qed) "interpret"
-        propss eqns goal_ctxt int state;
+        propss eqns goal_ctxt state;
   in
     generic_interpretation prep_interpretation setup_proof
       Attrib.local_notes (Context.proof_map ooo Locale.add_registration) expression raw_eqns ctxt