src/HOL/Wellfounded.thy
changeset 64632 9df24b8b6c0a
parent 63982 4c4049e3bad8
child 66952 80985b62029d
--- a/src/HOL/Wellfounded.thy	Wed Dec 21 21:26:25 2016 +0100
+++ b/src/HOL/Wellfounded.thy	Wed Dec 21 21:26:26 2016 +0100
@@ -308,7 +308,7 @@
   done
 
 lemma wfP_SUP:
-  "\<forall>i. wfP (r i) \<Longrightarrow> \<forall>i j. r i \<noteq> r j \<longrightarrow> inf (DomainP (r i)) (RangeP (r j)) = bot \<Longrightarrow>
+  "\<forall>i. wfP (r i) \<Longrightarrow> \<forall>i j. r i \<noteq> r j \<longrightarrow> inf (Domainp (r i)) (Rangep (r j)) = bot \<Longrightarrow>
     wfP (SUPREMUM UNIV r)"
   by (rule wf_UN[to_pred]) simp_all