# HG changeset patch # User smolkas # Date 1354101943 -3600 # Node ID 05f8ec128e838f61f1dcca5fd494cc9de055100b # Parent e0a4d8404c7681f0eadbf118d418b809d96592fb improved readability diff -r e0a4d8404c76 -r 05f8ec128e83 src/HOL/Tools/Sledgehammer/sledgehammer_shrink.ML --- a/src/HOL/Tools/Sledgehammer/sledgehammer_shrink.ML Wed Nov 28 12:25:43 2012 +0100 +++ b/src/HOL/Tools/Sledgehammer/sledgehammer_shrink.ML Wed Nov 28 12:25:43 2012 +0100 @@ -142,10 +142,10 @@ | Assume (_, t) => Skip_Proof.make_thm (Proof_Context.theory_of ctxt) t | _ => error "Internal error: unexpected succedent of case split") - :: map (Skip_Proof.make_thm (Proof_Context.theory_of ctxt) - o (fn Assume (_, a) => Logic.mk_implies(a, t) - | _ => error "Internal error: malformed case split") - o hd) + :: map + (hd #> (fn Assume (_, a) => Logic.mk_implies(a, t) + | _ => error "Internal error: malformed case split") + #> Skip_Proof.make_thm (Proof_Context.theory_of ctxt)) cases val goal = Goal.prove (Config.put Metis_Tactic.verbose debug ctxt) [] [] t