src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
changeset 48400 f08425165cca
parent 48396 dd82d190c2af
child 48406 b002cc16aa99
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML	Fri Jul 20 22:19:46 2012 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML	Fri Jul 20 22:19:46 2012 +0200
@@ -238,10 +238,12 @@
           (Term.add_vars t [] |> sort_wrt (fst o fst))
   |> fst
 
-fun backquote_thm th =
-  th |> prop_of |> close_form
-     |> hackish_string_for_term (theory_of_thm th)
-     |> backquote
+fun backquote_term thy t =
+  t |> close_form
+    |> hackish_string_for_term thy
+    |> backquote
+
+fun backquote_thm th = backquote_term (theory_of_thm th) (prop_of th)
 
 fun clasimpset_rule_table_of ctxt =
   let