src/HOL/Tools/Lifting/lifting_def.ML
changeset 58011 bc6bced136e5
parent 57664 179b9c43fe84
child 58028 e4250d370657
--- a/src/HOL/Tools/Lifting/lifting_def.ML	Tue Aug 19 18:21:29 2014 +0200
+++ b/src/HOL/Tools/Lifting/lifting_def.ML	Tue Aug 19 23:17:51 2014 +0200
@@ -13,7 +13,8 @@
     (binding * mixfix) -> typ -> term -> thm -> thm list -> local_theory -> local_theory
 
   val lift_def_cmd:
-    (binding * string option * mixfix) * string * (Facts.ref * Args.src list) list -> local_theory -> Proof.state
+    (binding * string option * mixfix) * string * (Facts.ref * Token.src list) list ->
+    local_theory -> Proof.state
 
   val can_generate_code_cert: thm -> bool
 end