src/HOL/Tools/BNF/bnf_lift.ML
changeset 61841 4d3527b94f2a
parent 61073 eea21f2ddf16
child 62137 b8dc1fd7d900
--- a/src/HOL/Tools/BNF/bnf_lift.ML	Sat Dec 12 15:37:42 2015 +0100
+++ b/src/HOL/Tools/BNF/bnf_lift.ML	Sun Dec 13 21:56:15 2015 +0100
@@ -345,10 +345,9 @@
   (fn (goals, after_qed, definitions, lthy) =>
     lthy
     |> Proof.theorem NONE after_qed (map (single o rpair []) goals)
-    |> Proof.refine (Method.Basic (fn ctxt => SIMPLE_METHOD (unfold_thms_tac ctxt definitions)))
-    |> Seq.hd
-    |> Proof.refine (Method.primitive_text (K I))
-    |> Seq.hd) oo
+    |> Proof.refine_singleton
+        (Method.Basic (fn ctxt => SIMPLE_METHOD (unfold_thms_tac ctxt definitions)))
+    |> Proof.refine_singleton (Method.primitive_text (K I))) oo
   prepare_common prepare_name prepare_sort prepare_term prepare_thm o apfst (apfst (apsnd SOME));
 
 fun prepare_solve prepare_name prepare_typ prepare_sort prepare_thm tacs =