src/HOL/Tools/Sledgehammer/sledgehammer.ML
changeset 59582 0fbed69ff081
parent 59471 ca459352d8c5
child 60548 e6adb8868478
--- a/src/HOL/Tools/Sledgehammer/sledgehammer.ML	Tue Mar 03 19:08:04 2015 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer.ML	Wed Mar 04 19:53:18 2015 +0100
@@ -75,7 +75,7 @@
 
       val {context = ctxt, facts = chained, goal} = Proof.goal state
       val (_, hyp_ts, concl_t) = strip_subgoal goal i ctxt
-      val goal_t = Logic.list_implies (map prop_of chained @ hyp_ts, concl_t)
+      val goal_t = Logic.list_implies (map Thm.prop_of chained @ hyp_ts, concl_t)
 
       fun try_methss [] [] = (used_facts, (preferred_meth, Play_Timed_Out Time.zeroTime))
         | try_methss ress [] =
@@ -305,7 +305,7 @@
             val problem =
               {comment = "", state = state, goal = goal, subgoal = i, subgoal_count = n,
                factss = factss}
-            val learn = mash_learn_proof ctxt params (prop_of goal) all_facts
+            val learn = mash_learn_proof ctxt params (Thm.prop_of goal) all_facts
             val launch = launch_prover params mode output_result only learn
           in
             if mode = Auto_Try then