src/HOL/Real_Vector_Spaces.thy
changeset 76055 8d56461f85ec
parent 74475 409ca22dee4c
child 77138 c8597292cd41
--- a/src/HOL/Real_Vector_Spaces.thy	Sat Jun 25 13:21:27 2022 +0200
+++ b/src/HOL/Real_Vector_Spaces.thy	Sat Jun 25 13:34:41 2022 +0200
@@ -2154,7 +2154,7 @@
     for n x y
     by metis
   have "antimono P"
-    using P(4) unfolding decseq_Suc_iff le_fun_def by blast
+    using P(4) by (rule decseq_SucI)
 
   obtain X where X: "P n (X n)" for n
     using P(1)[THEN eventually_happens'[OF \<open>F \<noteq> bot\<close>]] by metis