src/ZF/Sum.thy
changeset 1478 2b8c2a7547ab
parent 1401 0c439768f45c
child 2469 b50b8c0eec01
--- a/src/ZF/Sum.thy	Mon Feb 05 21:33:14 1996 +0100
+++ b/src/ZF/Sum.thy	Tue Feb 06 12:27:17 1996 +0100
@@ -1,6 +1,6 @@
-(*  Title: 	ZF/sum.thy
+(*  Title:      ZF/sum.thy
     ID:         $Id$
-    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1993  University of Cambridge
 
 Disjoint sums in Zermelo-Fraenkel Set Theory 
@@ -9,7 +9,7 @@
 
 Sum = Bool + "simpdata" +
 consts
-    "+"    	:: [i,i]=>i      		(infixr 65)
+    "+"         :: [i,i]=>i                     (infixr 65)
     Inl,Inr     :: i=>i
     case        :: [i=>i, i=>i, i]=>i
     Part        :: [i,i=>i] => i
@@ -21,5 +21,5 @@
     case_def    "case(c,d) == (%<y,z>. cond(y, d(z), c(z)))"
 
   (*operator for selecting out the various summands*)
-    Part_def	"Part(A,h) == {x: A. EX z. x = h(z)}"
+    Part_def    "Part(A,h) == {x: A. EX z. x = h(z)}"
 end