author | wenzelm |
Mon, 29 Nov 1999 15:52:49 +0100 | |
changeset 8039 | a901bafe4578 |
parent 5184 | 9b8547a9496a |
child 11703 | 6e5de8d4290a |
permissions | -rw-r--r-- |
(* File: TLA/ex/inc/Pcount.thy Author: Stephan Merz Copyright: 1997 University of Munich Theory Name: Pcount Logic Image: TLA Data type "program counter" for the increment example. Isabelle/HOL's datatype package generates useful simplifications and case distinction tactics. *) Pcount = Datatype + datatype pcount = a | b | g end ML