| author | paulson | 
| Wed, 10 Jan 2001 11:00:17 +0100 | |
| changeset 10840 | 28a53b68a8c0 | 
| parent 10212 | 33fe2d701ddd | 
| child 11954 | 3d1780208bf3 | 
| permissions | -rw-r--r-- | 
| 5181 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 1 | (* Title: HOL/Datatype.thy | 
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 2 | ID: $Id$ | 
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 3 | Author: Stefan Berghofer | 
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 4 | Copyright 1998 TU Muenchen | 
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 5 | *) | 
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 6 | |
| 10212 | 7 | Datatype = Datatype_Universe + | 
| 5181 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 8 | |
| 5759 | 9 | rep_datatype bool | 
| 10 | distinct True_not_False, False_not_True | |
| 11 | induct bool_induct | |
| 12 | ||
| 5181 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 13 | rep_datatype sum | 
| 5714 | 14 | distinct Inl_not_Inr, Inr_not_Inl | 
| 15 | inject Inl_eq, Inr_eq | |
| 5181 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 16 | induct sum_induct | 
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 17 | |
| 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 18 | rep_datatype prod | 
| 5714 | 19 | inject Pair_eq | 
| 20 | induct prod_induct | |
| 5181 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 21 | |
| 5759 | 22 | rep_datatype unit | 
| 23 | induct unit_induct | |
| 24 | ||
| 5181 
4ba3787d9709
New theory Datatype. Needed as an ancestor when defining datatypes.
 berghofe parents: diff
changeset | 25 | end |