src/HOL/Inductive.thy
changeset 11990 c1daefc08eff
parent 11825 ef7d619e2c88
child 12023 d982f98e0f0d
equal deleted inserted replaced
11989:d4bcba4e080e 11990:c1daefc08eff
    60   subset_refl imp_refl disj_mono conj_mono ex_mono all_mono if_def2
    60   subset_refl imp_refl disj_mono conj_mono ex_mono all_mono if_def2
    61   Collect_mono in_mono vimage_mono
    61   Collect_mono in_mono vimage_mono
    62   imp_conv_disj not_not de_Morgan_disj de_Morgan_conj
    62   imp_conv_disj not_not de_Morgan_disj de_Morgan_conj
    63   not_all not_ex
    63   not_all not_ex
    64   Ball_def Bex_def
    64   Ball_def Bex_def
    65   inductive_rulify2
    65   induct_rulify2
    66 
    66 
    67 
    67 
    68 subsubsection {* Inductive datatypes and primitive recursion *}
    68 subsubsection {* Inductive datatypes and primitive recursion *}
    69 
    69 
    70 text {* Package setup. *}
    70 text {* Package setup. *}