src/HOL/BNF/Tools/bnf_comp.ML
changeset 49585 5c4a12550491
parent 49538 c90818b63599
child 49586 d5e342ffe91e
--- a/src/HOL/BNF/Tools/bnf_comp.ML	Wed Sep 26 10:00:59 2012 +0200
+++ b/src/HOL/BNF/Tools/bnf_comp.ML	Wed Sep 26 10:00:59 2012 +0200
@@ -8,6 +8,9 @@
 
 signature BNF_COMP =
 sig
+  val ID_bnf: BNF_Def.BNF
+  val DEADID_bnf: BNF_Def.BNF
+
   type unfold_set
   val empty_unfolds: unfold_set
   val map_unfolds_of: unfold_set -> thm list
@@ -34,6 +37,10 @@
 open BNF_Tactics
 open BNF_Comp_Tactics
 
+val ID_bnf = the (bnf_of @{context} "Basic_BNFs.ID");
+val DEADID_bnf = the (bnf_of @{context} "Basic_BNFs.DEADID");
+
+(* TODO: Replace by "BNF_Defs.defs list" *)
 type unfold_set = {
   map_unfolds: thm list,
   set_unfoldss: thm list list,
@@ -677,9 +684,6 @@
     ((bnf', deads), lthy')
   end;
 
-val ID_bnf = the (bnf_of @{context} "Basic_BNFs.ID");
-val DEADID_bnf = the (bnf_of @{context} "Basic_BNFs.DEADID");
-
 fun bnf_of_typ _ _ _ (T as TFree _) accum = ((ID_bnf, ([], [T])), accum)
   | bnf_of_typ _ _ _ (TVar _) _ = error "Unexpected schematic variable"
   | bnf_of_typ const_policy qualify' sort (T as Type (C, Ts)) (unfold_set, lthy) =