changeset 128 | 89669c58e506 |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/Finite.thy Thu Aug 25 11:01:45 1994 +0200 @@ -0,0 +1,17 @@ +(* Title: HOL/Finite.thy + ID: $Id$ + Author: Lawrence C Paulson, Cambridge University Computer Laboratory + Copyright 1994 University of Cambridge + +Finite powerset operator +*) + +Finite = Lfp + +consts Fin :: "'a set => 'a set set" + +inductive "Fin(A)" + intrs + emptyI "{} : Fin(A)" + insertI "[| a: A; b: Fin(A) |] ==> insert(a,b) : Fin(A)" + +end