src/HOL/Wellfounded.thy
changeset 61952 546958347e05
parent 61943 7fba644ed827
child 63088 f2177f5d2aed
--- a/src/HOL/Wellfounded.thy	Mon Dec 28 16:34:26 2015 +0100
+++ b/src/HOL/Wellfounded.thy	Mon Dec 28 17:43:30 2015 +0100
@@ -305,7 +305,7 @@
 lemma wf_Union: 
  "[| ALL r:R. wf r;  
      ALL r:R. ALL s:R. r ~= s --> Domain r Int Range s = {}  
-  |] ==> wf(Union R)"
+  |] ==> wf (\<Union> R)"
   using wf_UN[of R "\<lambda>i. i"] by simp
 
 (*Intuition: we find an (R u S)-min element of a nonempty subset A