src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML
changeset 42094 e6867e9c6d10
parent 41228 e1fce873b814
child 42361 23f352990944
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML	Thu Mar 24 10:39:47 2011 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_aux.ML	Thu Mar 24 15:29:31 2011 +0100
@@ -51,6 +51,7 @@
   val is_predT : typ -> bool
   val is_constrt : theory -> term -> bool
   val is_constr : Proof.context -> string -> bool
+  val strip_ex : term -> (string * typ) list * term
   val focus_ex : term -> Name.context -> ((string * typ) list * term) * Name.context
   val strip_all : term -> (string * typ) list * term
   val strip_intro_concl : thm -> term * term list