src/ZF/Induct/Datatypes.thy
changeset 58871 c399ae4b836f
parent 35762 af3ff2ba4c54
child 60770 240563fbf41d
equal deleted inserted replaced
58870:e2c0d8ef29cb 58871:c399ae4b836f
     1 (*  Title:      ZF/Induct/Datatypes.thy
     1 (*  Title:      ZF/Induct/Datatypes.thy
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Copyright   1994  University of Cambridge
     3     Copyright   1994  University of Cambridge
     4 *)
     4 *)
     5 
     5 
     6 header {* Sample datatype definitions *}
     6 section {* Sample datatype definitions *}
     7 
     7 
     8 theory Datatypes imports Main begin
     8 theory Datatypes imports Main begin
     9 
     9 
    10 subsection {* A type with four constructors *}
    10 subsection {* A type with four constructors *}
    11 
    11