src/HOL/Infinite_Set.thy
changeset 16796 140f1e0ea846
parent 16733 236dfafbeb63
child 19313 45c9fc22904b
--- a/src/HOL/Infinite_Set.thy	Wed Jul 13 15:06:04 2005 +0200
+++ b/src/HOL/Infinite_Set.thy	Wed Jul 13 15:06:20 2005 +0200
@@ -127,7 +127,7 @@
     assume "\<not> ?rhs"
     then obtain m where m: "\<forall>n. m<n \<longrightarrow> n\<notin>S" by blast
     hence "S \<subseteq> {..m}"
-      by (auto simp add: sym[OF not_less_iff_le])
+      by (auto simp add: sym[OF linorder_not_less])
     with inf show "False" 
       by (simp add: finite_nat_iff_bounded_le)
   qed