src/HOL/UNITY/UNITY.thy
changeset 13861 0c18f31d901a
parent 13812 91713a1915ee
child 13870 cf947d1ec5ff
--- a/src/HOL/UNITY/UNITY.thy	Fri Mar 14 10:30:15 2003 +0100
+++ b/src/HOL/UNITY/UNITY.thy	Fri Mar 14 10:30:46 2003 +0100
@@ -72,6 +72,9 @@
 lemma insert_Id_Acts [iff]: "insert Id (Acts F) = Acts F"
 by (simp add: insert_absorb Id_in_Acts)
 
+lemma Acts_nonempty [simp]: "Acts F \<noteq> {}"
+by auto
+
 lemma Id_in_AllowedActs [iff]: "Id \<in> AllowedActs F"
 apply (cut_tac x = F in Rep_Program)
 apply (auto simp add: program_typedef)