diff -r 4c51ab632cda -r 2b8c2a7547ab src/ZF/Finite.thy --- a/src/ZF/Finite.thy Mon Feb 05 21:33:14 1996 +0100 +++ b/src/ZF/Finite.thy Tue Feb 06 12:27:17 1996 +0100 @@ -1,6 +1,6 @@ -(* Title: ZF/Finite.thy +(* Title: ZF/Finite.thy ID: $Id$ - Author: Lawrence C Paulson, Cambridge University Computer Laboratory + Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1994 University of Cambridge Finite powerset operator @@ -8,8 +8,8 @@ Finite = Arith + Inductive + consts - Fin :: i=>i - FiniteFun :: [i,i]=>i ("(_ -||>/ _)" [61, 60] 60) + Fin :: i=>i + FiniteFun :: [i,i]=>i ("(_ -||>/ _)" [61, 60] 60) inductive domains "Fin(A)" <= "Pow(A)" @@ -24,6 +24,6 @@ intrs emptyI "0 : A -||> B" consI "[| a: A; b: B; h: A -||> B; a ~: domain(h) - |] ==> cons(,h) : A -||> B" + |] ==> cons(,h) : A -||> B" type_intrs "Fin.intrs" end