src/HOL/UNITY/Simple/Reach.thy
changeset 32960 69916a850301
parent 26825 0373ed6f04b1
child 35416 d8d7d1b785af
--- a/src/HOL/UNITY/Simple/Reach.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/UNITY/Simple/Reach.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,10 +1,9 @@
 (*  Title:      HOL/UNITY/Reach.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
 Reachability in Directed Graphs.  From Chandy and Misra, section 6.4.
-	[this example took only four days!]
+[this example took only four days!]
 *)
 
 theory Reach imports "../UNITY_Main" begin