PIPDefs.thy
changeset 204 5191a09d9928
parent 197 ca4ddf26a7c7
--- a/PIPDefs.thy	Mon Jan 15 11:35:56 2018 +0000
+++ b/PIPDefs.thy	Tue Feb 06 14:38:31 2018 +0000
@@ -269,7 +269,7 @@
 *}
 
 abbreviation
-  "all_unlocked \<equiv> \<lambda>_::cs. ([]::thread list)"
+  "all_unlocked \<equiv> \<lambda>cs::cs. ([]::thread list)"
 
 
 text {*