src/ZF/UNITY/Union.thy
changeset 32960 69916a850301
parent 24893 b8ef7afe3a6b
child 35112 ff6f60e6ab85
--- a/src/ZF/UNITY/Union.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/UNITY/Union.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      ZF/UNITY/Union.thy
-    ID:         $Id$
     Author:     Sidi O Ehmety, Computer Laboratory
     Copyright   2001  University of Cambridge
 
@@ -34,7 +33,7 @@
 definition
   Join :: "[i, i] => i"    (infixl "Join" 65)  where
   "F Join G == mk_program (Init(F) Int Init(G), Acts(F) Un Acts(G),
-				AllowedActs(F) Int AllowedActs(G))"
+                                AllowedActs(F) Int AllowedActs(G))"
 definition
   (*Characterizes safety properties.  Used with specifying AllowedActs*)
   safety_prop :: "i => o"  where