src/ZF/Datatype.thy
author lcp
Wed, 03 May 1995 13:55:05 +0200
changeset 1091 f55f54a032ce
parent 809 1daa0269eb5d
child 2870 6d6fd10a9fdc
permissions -rw-r--r--
Changed some definitions and proofs to use pattern-matching.

(*Dummy theory to document dependencies *)

Datatype = "constructor" + Inductive + Univ + QUniv

(*Datatype must be capital to avoid conflicts with ML's "datatype" *)