src/HOL/Tools/SMT2/z3_new_isar.ML
changeset 57159 24cbdebba35a
parent 57056 8b2283566f6e
child 57218 7e90e30822a9
--- a/src/HOL/Tools/SMT2/z3_new_isar.ML	Mon Jun 02 17:34:26 2014 +0200
+++ b/src/HOL/Tools/SMT2/z3_new_isar.ML	Mon Jun 02 17:34:27 2014 +0200
@@ -6,11 +6,9 @@
 
 signature Z3_NEW_ISAR =
 sig
-  type ('a, 'b) atp_step = ('a, 'b) ATP_Proof.atp_step
-
   val atp_proof_of_z3_proof: Proof.context -> thm list -> term list -> term ->
     (string * term) list -> int list -> int -> (int * string) list -> Z3_New_Proof.z3_step list ->
-    (term, string) atp_step list
+    (term, string) ATP_Proof.atp_step list
 end;
 
 structure Z3_New_Isar: Z3_NEW_ISAR =