src/HOL/Algebra/Order.thy
changeset 67613 ce654b0e6d69
parent 67399 eab6ce8368fa
child 68004 a8a20be7053a
child 68072 493b818e8e10
--- a/src/HOL/Algebra/Order.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/Algebra/Order.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -379,7 +379,7 @@
 proof -
   have "Upper L A \<subseteq> carrier L" by simp
   moreover from above L have "s \<in> Upper L A" by (simp add: Upper_def)
-  moreover from below have "ALL x : Upper L A. s \<sqsubseteq> x" by fast
+  moreover from below have "\<forall>x \<in> Upper L A. s \<sqsubseteq> x" by fast
   ultimately show ?thesis by (simp add: least_def)
 qed
 
@@ -439,7 +439,7 @@
 proof -
   have "Lower L A \<subseteq> carrier L" by simp
   moreover from below L have "i \<in> Lower L A" by (simp add: Lower_def)
-  moreover from above have "ALL x : Lower L A. x \<sqsubseteq> i" by fast
+  moreover from above have "\<forall>x \<in> Lower L A. x \<sqsubseteq> i" by fast
   ultimately show ?thesis by (simp add: greatest_def)
 qed