src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
changeset 48400 f08425165cca
parent 48396 dd82d190c2af
child 48406 b002cc16aa99
equal deleted inserted replaced
48399:4bacc8983b3d 48400:f08425165cca
   236                  s' :: taken)
   236                  s' :: taken)
   237               end)
   237               end)
   238           (Term.add_vars t [] |> sort_wrt (fst o fst))
   238           (Term.add_vars t [] |> sort_wrt (fst o fst))
   239   |> fst
   239   |> fst
   240 
   240 
   241 fun backquote_thm th =
   241 fun backquote_term thy t =
   242   th |> prop_of |> close_form
   242   t |> close_form
   243      |> hackish_string_for_term (theory_of_thm th)
   243     |> hackish_string_for_term thy
   244      |> backquote
   244     |> backquote
       
   245 
       
   246 fun backquote_thm th = backquote_term (theory_of_thm th) (prop_of th)
   245 
   247 
   246 fun clasimpset_rule_table_of ctxt =
   248 fun clasimpset_rule_table_of ctxt =
   247   let
   249   let
   248     val thy = Proof_Context.theory_of ctxt
   250     val thy = Proof_Context.theory_of ctxt
   249     val atomize = HOLogic.mk_Trueprop o Object_Logic.atomize_term thy
   251     val atomize = HOLogic.mk_Trueprop o Object_Logic.atomize_term thy