src/ZF/ex/Data.thy
author wenzelm
Sat, 20 Oct 2001 20:20:41 +0200
changeset 11852 a528a716a312
parent 11354 9b80fe19407f
permissions -rw-r--r--
added TextIO.stdErr;

(*  Title:      ZF/ex/Data.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1994  University of Cambridge

Sample datatype definition.  
It has four contructors, of arities 0-3, and two parameters A and B.
*)

Data = Main +

consts
  data :: [i,i] => i

datatype
  "data(A,B)" = Con0
              | Con1 ("a \\<in> A")
              | Con2 ("a \\<in> A", "b \\<in> B")
              | Con3 ("a \\<in> A", "b \\<in> B", "d \\<in> data(A,B)")

end