diff -r 422ac6888c7f -r d139b03fcac2 src/HOL/UNITY/Alloc.thy --- a/src/HOL/UNITY/Alloc.thy Thu Oct 28 14:55:23 1999 +0200 +++ b/src/HOL/UNITY/Alloc.thy Thu Oct 28 16:04:57 1999 +0200 @@ -161,8 +161,6 @@ allocAsk = allocAsk s, allocRel = allocRel s, client = y |)" -(*** "sysOfAlloc == %(s,y). s(|client := y|)" TYPE DOESN'T CHANGE***) - sysOfClient :: "((nat => clientState) * allocState ) => systemState" "sysOfClient == %(x,y). sysOfAlloc(y,x)"