tuned header
authorhaftmann
Mon, 21 Sep 2009 15:35:14 +0200
changeset 32692 90c8af39e215
parent 32691 cdf70f1fc9f9
child 32693 6c6b1ba5e71e
tuned header
src/HOL/UNITY/Simple/Common.thy
--- a/src/HOL/UNITY/Simple/Common.thy	Mon Sep 21 15:35:14 2009 +0200
+++ b/src/HOL/UNITY/Simple/Common.thy	Mon Sep 21 15:35:14 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      HOL/UNITY/Common
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
@@ -10,7 +9,9 @@
 From Misra, "A Logic for Concurrent Programming" (1994), sections 5.1 and 13.1.
 *)
 
-theory Common imports "../UNITY_Main" begin
+theory Common
+imports "../UNITY_Main"
+begin
 
 consts
   ftime :: "nat=>nat"