src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML
changeset 75026 b61949cba32a
parent 75025 f741d55a81e5
child 75031 ae4dc5ac983f
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML	Mon Jan 31 16:09:23 2022 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML	Mon Jan 31 16:09:23 2022 +0100
@@ -14,6 +14,7 @@
   type fact = Sledgehammer_Fact.fact
   type proof_method = Sledgehammer_Proof_Methods.proof_method
   type play_outcome = Sledgehammer_Proof_Methods.play_outcome
+  type base_slice = Sledgehammer_ATP_Systems.base_slice
   type atp_slice = Sledgehammer_ATP_Systems.atp_slice
 
   datatype mode = Auto_Try | Try | Normal | Minimize | MaSh
@@ -62,9 +63,7 @@
      factss : (string * fact list) list,
      found_proof : string -> unit}
 
-  datatype prover_slice =
-    ATP_Slice of atp_slice
-  | SMT_Slice of int * string
+  type prover_slice = base_slice * atp_slice option
 
   type prover_result =
     {outcome : atp_failure option,
@@ -199,9 +198,7 @@
    factss : (string * fact list) list,
    found_proof : string -> unit}
 
-datatype prover_slice =
-  ATP_Slice of atp_slice
-| SMT_Slice of int * string
+type prover_slice = base_slice * atp_slice option
 
 type prover_result =
   {outcome : atp_failure option,