src/ZF/AC/Hartog.thy
author clasohm
Sat, 09 Dec 1995 13:36:11 +0100
changeset 1401 0c439768f45c
parent 1203 a39bec971684
child 1478 2b8c2a7547ab
permissions -rw-r--r--
removed quotes from consts and syntax sections

(*  Title: 	ZF/AC/Hartog.thy
    ID:         $Id$
    Author: 	Krzysztof Grabczewski

Hartog's function.
*)

Hartog = Cardinal +

consts

  Hartog :: i => i

defs

  Hartog_def "Hartog(X) == LEAST i. ~i lepoll X"

end