src/HOL/Tools/try0.ML
changeset 54431 e98996c2a32c
parent 54291 709a2bbd7638
child 55177 b7ca9f98faca
--- a/src/HOL/Tools/try0.ML	Thu Nov 14 15:40:06 2013 +0100
+++ b/src/HOL/Tools/try0.ML	Thu Nov 14 15:40:06 2013 +0100
@@ -110,8 +110,9 @@
   let
     val st = st |> Proof.map_context (Config.put Metis_Tactic.verbose false #>
       Config.put Lin_Arith.verbose false)
+    fun trd (_, _, t) = t
     fun par_map f =
-      if mode = Normal then Par_List.map f #> map_filter I #> sort (int_ord o pairself #3)
+      if mode = Normal then Par_List.map f #> map_filter I #> sort (int_ord o pairself trd)
       else Par_List.get_some f #> the_list
   in
     if mode = Normal then