src/ZF/Inductive_ZF.thy
changeset 26190 cf51a23c0cd0
parent 26189 9808cca5c54d
child 26480 544cef16045b
equal deleted inserted replaced
26189:9808cca5c54d 26190:cf51a23c0cd0
    40 
    40 
    41 setup IndCases.setup
    41 setup IndCases.setup
    42 setup DatatypeTactics.setup
    42 setup DatatypeTactics.setup
    43 
    43 
    44 ML_setup {*
    44 ML_setup {*
    45 val iT = Ind_Syntax.iT
       
    46 and oT = FOLogic.oT;
       
    47 
       
    48 structure Lfp =
    45 structure Lfp =
    49   struct
    46   struct
    50   val oper      = @{const lfp}
    47   val oper      = @{const lfp}
    51   val bnd_mono  = @{const bnd_mono}
    48   val bnd_mono  = @{const bnd_mono}
    52   val bnd_monoI = @{thm bnd_monoI}
    49   val bnd_monoI = @{thm bnd_monoI}