src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML
changeset 34948 2d5f2a9f7601
parent 33752 9aa8e961f850
child 34954 b206c70ea6f0
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML	Sat Jan 16 21:14:15 2010 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_fun.ML	Wed Jan 20 11:56:45 2010 +0100
@@ -14,31 +14,7 @@
 structure Predicate_Compile_Fun : PREDICATE_COMPILE_FUN =
 struct
 
-fun is_funtype (Type ("fun", [_, _])) = true
-  | is_funtype _ = false;
-
-fun is_Type (Type _) = true
-  | is_Type _ = false
-
-(* returns true if t is an application of an datatype constructor *)
-(* which then consequently would be splitted *)
-(* else false *)
-(*
-fun is_constructor thy t =
-  if (is_Type (fastype_of t)) then
-    (case DatatypePackage.get_datatype thy ((fst o dest_Type o fastype_of) t) of
-      NONE => false
-    | SOME info => (let
-      val constr_consts = maps (fn (_, (_, _, constrs)) => map fst constrs) (#descr info)
-      val (c, _) = strip_comb t
-      in (case c of
-        Const (name, _) => name mem_string constr_consts
-        | _ => false) end))
-  else false
-*)
-
-(* must be exported in code.ML *)
-fun is_constr thy = is_some o Code.get_datatype_of_constr thy;
+open Predicate_Compile_Aux;
 
 (* Table from constant name (string) to term of inductive predicate *)
 structure Pred_Compile_Preproc = Theory_Data