src/ZF/AC/Hartog.thy
author lcp
Fri, 28 Jul 1995 11:02:22 +0200
changeset 1203 a39bec971684
parent 1123 5dfdc1464966
child 1401 0c439768f45c
permissions -rw-r--r--
Ran expandshort and changed spelling of Grabczewski

(*  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