src/HOLCF/IOA/NTP/Correctness.thy
changeset 3898 f6bf42312e9e
parent 3073 88366253a09a
child 4816 64f075872f69
--- a/src/HOLCF/IOA/NTP/Correctness.thy	Thu Oct 16 14:12:58 1997 +0200
+++ b/src/HOLCF/IOA/NTP/Correctness.thy	Thu Oct 16 14:14:01 1997 +0200
@@ -12,6 +12,6 @@
 
   hom :: 'm impl_state => 'm list
   "hom(s) == rq(rec(s)) @ (if rbit(rec s) = sbit(sen s) then sq(sen s) 
-                          else ttl(sq(sen s)))"
+                           else tl(sq(sen s)))"
 
 end