src/HOL/Inductive.thy
changeset 14981 e73f8140af78
parent 13705 934d6c1421f2
child 15131 c69542757a4d
equal deleted inserted replaced
14980:267cc670317a 14981:e73f8140af78
     1 (*  Title:      HOL/Inductive.thy
     1 (*  Title:      HOL/Inductive.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Markus Wenzel, TU Muenchen
     3     Author:     Markus Wenzel, TU Muenchen
     4     License:    GPL (GNU GENERAL PUBLIC LICENSE)
       
     5 *)
     4 *)
     6 
     5 
     7 header {* Support for inductive sets and types *}
     6 header {* Support for inductive sets and types *}
     8 
     7 
     9 theory Inductive = Gfp + Sum_Type + Relation + Record
     8 theory Inductive = Gfp + Sum_Type + Relation + Record