src/HOL/Datatype.thy
author paulson
Thu, 01 Oct 1998 18:30:05 +0200
changeset 5601 b6456ccd9e3e
parent 5181 4ba3787d9709
child 5714 b4f2e281a907
permissions -rw-r--r--
revised for new treatment of integers

(*  Title:      HOL/Datatype.thy
    ID:         $Id$
    Author:     Stefan Berghofer
    Copyright   1998  TU Muenchen
*)

Datatype = Univ +

rep_datatype sum
  distinct "[[Inl_not_Inr, Inr_not_Inl]]"
  inject   "[[Inl_eq, Inr_eq]]"
  induct   sum_induct

rep_datatype prod
  distinct "[[]]"
  inject   "[[Pair_eq]]"
  induct   "allI RS (allI RS (split_paired_All RS iffD2)) RS spec"

end