| author | wenzelm | 
| Sat, 01 Apr 2000 20:21:39 +0200 | |
| changeset 8657 | b9475dad85ed | 
| parent 5759 | bf5d9e5b8cdf | 
| child 10212 | 33fe2d701ddd | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Datatype.thy ID: $Id$ Author: Stefan Berghofer Copyright 1998 TU Muenchen *) Datatype = Univ + rep_datatype bool distinct True_not_False, False_not_True induct bool_induct rep_datatype sum distinct Inl_not_Inr, Inr_not_Inl inject Inl_eq, Inr_eq induct sum_induct rep_datatype prod inject Pair_eq induct prod_induct rep_datatype unit induct unit_induct end