src/ZF/Induct/FoldSet.thy
changeset 32960 69916a850301
parent 24893 b8ef7afe3a6b
child 46822 95f1e700b712
--- a/src/ZF/Induct/FoldSet.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/Induct/FoldSet.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,8 +1,6 @@
 (*  Title:      ZF/Induct/FoldSet.thy
-    ID:         $Id$
     Author:     Sidi O Ehmety, Cambridge University Computer Laboratory
 
-
 A "fold" functional for finite sets.  For n non-negative we have
 fold f e {x1,...,xn} = f x1 (... (f xn e)) where f is at
 least left-commutative.  
@@ -17,7 +15,7 @@
   intros
     emptyI: "e\<in>B ==> <0, e>\<in>fold_set(A, B, f,e)"
     consI:  "[| x\<in>A; x \<notin>C;  <C,y> : fold_set(A, B,f,e); f(x,y):B |]
-		==>  <cons(x,C), f(x,y)>\<in>fold_set(A, B, f, e)"
+                ==>  <cons(x,C), f(x,y)>\<in>fold_set(A, B, f, e)"
   type_intros Fin.intros
   
 definition