src/HOL/UNITY/Extend.thy
changeset 67613 ce654b0e6d69
parent 63146 f1ecba0272f9
child 69313 b021008c5397
--- a/src/HOL/UNITY/Extend.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/UNITY/Extend.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -49,7 +49,7 @@
   where "project h C F =
        mk_program (project_set h (Init F),
                    project_act h ` Restrict C ` Acts F,
-                   {act. Restrict (project_set h C) act :
+                   {act. Restrict (project_set h C) act \<in>
                          project_act h ` Restrict C ` AllowedActs F})"
 
 locale Extend =
@@ -70,7 +70,7 @@
 subsection\<open>Restrict\<close>
 (*MOVE to Relation.thy?*)
 
-lemma Restrict_iff [iff]: "((x,y): Restrict A r) = ((x,y): r & x \<in> A)"
+lemma Restrict_iff [iff]: "((x,y) \<in> Restrict A r) = ((x,y) \<in> r & x \<in> A)"
 by (unfold Restrict_def, blast)
 
 lemma Restrict_UNIV [simp]: "Restrict UNIV = id"