src/HOL/UNITY/Follows.thy
changeset 54859 64ff7f16d5b7
parent 41413 64cd30d6b0b8
child 56248 67dc9549fa15
--- a/src/HOL/UNITY/Follows.thy	Wed Dec 25 10:09:43 2013 +0100
+++ b/src/HOL/UNITY/Follows.thy	Wed Dec 25 15:52:25 2013 +0100
@@ -158,7 +158,7 @@
 lemma Follows_Un: 
     "[| F \<in> f' Fols f;  F \<in> g' Fols g |]  
      ==> F \<in> (%s. (f' s) \<union> (g' s)) Fols (%s. (f s) \<union> (g s))"
-apply (simp add: Follows_def Increasing_Un Always_Un del: Un_subset_iff le_sup_iff, auto)
+apply (simp add: Follows_def Increasing_Un Always_Un del: Un_subset_iff sup.bounded_iff, auto)
 apply (rule LeadsTo_Trans)
 apply (blast intro: Follows_Un_lemma)
 (*Weakening is used to exchange Un's arguments*)