src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML
changeset 59888 27e4d0ab0948
parent 59877 a04ea4709c8d
child 60638 16d80e5ef2dc
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML	Tue Mar 31 23:42:57 2015 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML	Wed Apr 01 10:35:43 2015 +0200
@@ -737,8 +737,6 @@
 
 (*** Isabelle helpers ***)
 
-val local_prefix = Long_Name.localN ^ Long_Name.separator
-
 fun elided_backquote_thm threshold th =
   elide_string threshold (backquote_thm (Proof_Context.init_global (Thm.theory_of_thm th)) th)
 
@@ -748,7 +746,7 @@
   if Thm.has_name_hint th then
     let val hint = Thm.get_name_hint th in
       (* There must be a better way to detect local facts. *)
-      (case try (unprefix local_prefix) hint of
+      (case Long_Name.dest_local hint of
         SOME suf => Long_Name.implode [thy_name_of_thm th, suf, elided_backquote_thm 50 th]
       | NONE => hint)
     end