src/Pure/Isar/locale.ML
changeset 67714 a0b58be402ab
parent 67694 ab68ca1e80ba
child 67814 c4c4c2f01723
--- a/src/Pure/Isar/locale.ML	Fri Feb 23 20:55:46 2018 +0100
+++ b/src/Pure/Isar/locale.ML	Fri Feb 23 21:12:08 2018 +0100
@@ -49,7 +49,6 @@
   val pretty_name: Proof.context -> string -> Pretty.T
   val defined: theory -> string -> bool
   val params_of: theory -> string -> ((string * typ) * mixfix) list
-  val params_types_of: theory -> string -> string list * typ list
   val intros_of: theory -> string -> thm option * thm option
   val axioms_of: theory -> string -> thm list
   val instance_of: theory -> string -> morphism -> term list
@@ -213,7 +212,6 @@
 (** Primitive operations **)
 
 fun params_of thy = snd o #parameters o the_locale thy;
-fun params_types_of thy loc = split_list (map #1 (params_of thy loc));
 
 fun intros_of thy = (apply2 o Option.map) (Thm.transfer thy) o #intros o the_locale thy;