src/HOL/UNITY/Channel.thy
changeset 5253 82a5ca6290aa
parent 4776 1f9362e769c1
child 5608 a82a038a3e7a
--- a/src/HOL/UNITY/Channel.thy	Wed Aug 05 10:56:58 1998 +0200
+++ b/src/HOL/UNITY/Channel.thy	Wed Aug 05 10:57:25 1998 +0200
@@ -18,12 +18,12 @@
 
 rules
 
-  skip "id: Acts"
+  skip "id: acts"
 
-  UC1  "constrains Acts (minSet -`` {Some x}) (minSet -`` (Some``atLeast x))"
+  UC1  "constrains acts (minSet -`` {Some x}) (minSet -`` (Some``atLeast x))"
 
-  (*  UC1  "constrains Acts {s. minSet s = x} {s. x <= minSet s}"  *)
+  (*  UC1  "constrains acts {s. minSet s = x} {s. x <= minSet s}"  *)
 
-  UC2  "leadsTo Acts (minSet -`` {Some x}) {s. x ~: s}"
+  UC2  "leadsTo acts (minSet -`` {Some x}) {s. x ~: s}"
 
 end