src/HOL/UNITY/Comp/Priority.thy
changeset 60773 d09c66a0ea10
parent 58889 5b7a9633cfa8
child 61941 31f2105521ee
--- a/src/HOL/UNITY/Comp/Priority.thy	Thu Jul 23 16:40:47 2015 +0200
+++ b/src/HOL/UNITY/Comp/Priority.thy	Thu Jul 23 22:13:42 2015 +0200
@@ -65,7 +65,7 @@
      the vertex 'UNIV' is finite by assumption *)
   
 definition system :: "state program"
-  where "system = (JN i. Component i)"
+  where "system = (\<Squnion>i. Component i)"
 
 
 declare highest_def [simp] lowest_def [simp]