src/HOL/Topological_Spaces.thy
changeset 73411 1f1366966296
parent 71827 5e315defb038
child 73832 9db620f007fa
--- a/src/HOL/Topological_Spaces.thy	Thu Mar 11 07:05:29 2021 +0000
+++ b/src/HOL/Topological_Spaces.thy	Thu Mar 11 07:05:38 2021 +0000
@@ -853,7 +853,7 @@
     and at_within_Icc_at_left:  "at b within {a..b} = at_left b"
   using order_tendstoD(2)[OF tendsto_ident_at assms, of "{a<..}"]
   using order_tendstoD(1)[OF tendsto_ident_at assms, of "{..<b}"]
-  by (auto intro!: order_class.antisym filter_leI
+  by (auto intro!: order_class.order_antisym filter_leI
       simp: eventually_at_filter less_le
       elim: eventually_elim2)