src/HOL/Codatatype/Tools/bnf_lfp.ML
changeset 49125 5fc5211cf104
parent 49124 968e1b7de057
child 49126 1bbd7a37fc29
equal deleted inserted replaced
49124:968e1b7de057 49125:5fc5211cf104
     6 Datatype construction.
     6 Datatype construction.
     7 *)
     7 *)
     8 
     8 
     9 signature BNF_LFP =
     9 signature BNF_LFP =
    10 sig
    10 sig
    11   val bnf_lfp: binding list -> typ list list -> BNF_Def.BNF list -> Proof.context ->
    11   val bnf_lfp: binding list -> typ list list -> BNF_Def.BNF list -> local_theory ->
    12     (term list * term list * thm list * thm list) * Proof.context
    12     (term list * term list * thm list * thm list) * local_theory
    13 end;
    13 end;
    14 
    14 
    15 structure BNF_LFP : BNF_LFP =
    15 structure BNF_LFP : BNF_LFP =
    16 struct
    16 struct
    17 
    17