src/HOL/ZF/MainZF.thy
author krauss
Thu, 21 Sep 2006 12:22:05 +0200
changeset 20654 d80502f0d701
parent 19203 778507520684
child 35416 d8d7d1b785af
permissions -rw-r--r--
1. Function package accepts a parameter (default "some_term"), which specifies the functions behaviour outside its domain. 2. Bugfix: An exception occured when a function in a mutual definition was declared but no equation was given.

(*  Title:      HOL/ZF/MainZF.thy
    ID:         $Id$
    Author:     Steven Obua

    Starting point for using HOLZF.
    See "Partizan Games in Isabelle/HOLZF", available from http://www4.in.tum.de/~obua/partizan
*)

theory MainZF
imports Zet LProd
begin
end