src/HOL/Inductive.thy
changeset 58306 117ba6cbe414
parent 58187 d2ddd401d74d
child 58815 fd3f893a40ea
equal deleted inserted replaced
58305:57752a91eec4 58306:117ba6cbe414
     8 imports Complete_Lattices Ctr_Sugar
     8 imports Complete_Lattices Ctr_Sugar
     9 keywords
     9 keywords
    10   "inductive" "coinductive" "inductive_cases" "inductive_simps" :: thy_decl and
    10   "inductive" "coinductive" "inductive_cases" "inductive_simps" :: thy_decl and
    11   "monos" and
    11   "monos" and
    12   "print_inductives" :: diag and
    12   "print_inductives" :: diag and
    13   "rep_datatype" :: thy_goal and
    13   "old_rep_datatype" :: thy_goal and
    14   "primrec" :: thy_decl
    14   "primrec" :: thy_decl
    15 begin
    15 begin
    16 
    16 
    17 subsection {* Least and greatest fixed points *}
    17 subsection {* Least and greatest fixed points *}
    18 
    18