src/HOL/Mirabelle/Tools/mirabelle_metis.ML
changeset 63337 ae9330fdbc16
parent 62519 a564458f94db
--- a/src/HOL/Mirabelle/Tools/mirabelle_metis.ML	Tue Jun 21 11:03:24 2016 +0200
+++ b/src/HOL/Mirabelle/Tools/mirabelle_metis.ML	Tue Jun 21 14:42:47 2016 +0200
@@ -16,7 +16,7 @@
     val names = map Thm.get_name_hint thms
     val add_info = if null names then I else suffix (":\n" ^ commas names)
 
-    val facts = Facts.props (Proof_Context.facts_of (Proof.context_of pre))
+    val facts = map #1 (Facts.props (Proof_Context.facts_of (Proof.context_of pre)))
 
     fun metis ctxt =
       Metis_Tactic.metis_tac [] ATP_Problem_Generate.liftingN ctxt