src/HOL/Tools/BNF/bnf_fp_def_sugar.ML
changeset 58230 61e4c96bf2b6
parent 58214 bd1754377965
child 58233 108f9ab5466d
--- a/src/HOL/Tools/BNF/bnf_fp_def_sugar.ML	Mon Sep 08 15:54:33 2014 +0200
+++ b/src/HOL/Tools/BNF/bnf_fp_def_sugar.ML	Mon Sep 08 16:09:10 2014 +0200
@@ -50,6 +50,7 @@
 
   val flat_corec_preds_predsss_gettersss: 'a list -> 'a list list list -> 'a list list list ->
     'a list
+  val liveness_of_fp_bnf: int -> BNF_Def.bnf -> bool list
   val nesting_bnfs: Proof.context -> typ list list list -> typ list -> BNF_Def.bnf list
 
   type lfp_sugar_thms = (thm list * thm * Token.src list) * (thm list list * Token.src list)