src/HOL/Inductive.thy
changeset 10312 4c5a03649af7
parent 10212 33fe2d701ddd
child 10402 5e82d6cafb5f
equal deleted inserted replaced
10311:3b53ed2c846f 10312:4c5a03649af7
    16 setup InductMethod.setup
    16 setup InductMethod.setup
    17 setup InductivePackage.setup
    17 setup InductivePackage.setup
    18 setup DatatypePackage.setup
    18 setup DatatypePackage.setup
    19 setup PrimrecPackage.setup
    19 setup PrimrecPackage.setup
    20 
    20 
    21 theorems [mono] =
    21 theorems basic_monos [mono] =
    22    subset_refl imp_refl disj_mono conj_mono ex_mono all_mono
    22    subset_refl imp_refl disj_mono conj_mono ex_mono all_mono
    23    Collect_mono in_mono vimage_mono
    23    Collect_mono in_mono vimage_mono
    24    imp_conv_disj not_not de_Morgan_disj de_Morgan_conj
    24    imp_conv_disj not_not de_Morgan_disj de_Morgan_conj
    25    not_all not_ex
    25    not_all not_ex
    26    Ball_def Bex_def
    26    Ball_def Bex_def
    27 
    27 
       
    28 (*belongs to theory Transitive_Closure*)
       
    29 declare rtrancl_induct [induct set: rtrancl]
       
    30 declare rtranclE [cases set: rtrancl]
       
    31 declare trancl_induct [induct set: trancl]
       
    32 declare tranclE [cases set: trancl]
       
    33 
    28 end
    34 end