src/HOL/Inductive.thy
author paulson
Fri, 23 Jul 1999 17:30:27 +0200
changeset 7078 4e64b2bd10ce
parent 6437 9bdfe07ba8e9
child 7357 d0e16da40ea2
permissions -rw-r--r--
now using correctly-typed constants from HOLogic


Inductive = Gfp + Prod + Sum +

setup InductivePackage.setup

end