src/ZF/datatype.thy
author paulson
Thu, 02 Jul 1998 17:58:12 +0200
changeset 5116 8eb343ab5748
parent 124 858ab9a9b047
permissions -rw-r--r--
Renamed expand_if to split_if and setloop split_tac to addsplits, as in HOL

(*Dummy theory to document dependencies *)

Datatype = "constructor" + "inductive" + "coinductive" + Univ + QUniv
               (*this must be capital to avoid conflicts with ML's "datatype" *)