src/HOL/UNITY/Traces.thy
changeset 4837 eab729051897
parent 4776 1f9362e769c1
child 5111 8f4b72f0c15d
--- a/src/HOL/UNITY/Traces.thy	Mon Apr 27 19:29:19 1998 +0200
+++ b/src/HOL/UNITY/Traces.thy	Mon Apr 27 19:30:40 1998 +0200
@@ -15,7 +15,6 @@
 
 inductive "reachable Init Acts"
   intrs 
-         (*Initial trace is empty*)
     Init  "s: Init ==> s : reachable Init Acts"
 
     Acts  "[| act: Acts;  s : reachable Init Acts;  (s,s'): act |]