--- a/src/HOL/Probability/Discrete_Topology.thy Fri Sep 24 13:40:14 2021 +0200
+++ b/src/HOL/Probability/Discrete_Topology.thy Fri Sep 24 22:23:26 2021 +0200
@@ -32,10 +32,10 @@
instance discrete :: (type) complete_space
proof
- fix X::"nat\<Rightarrow>'a discrete" assume "Cauchy X"
- hence "\<exists>n. \<forall>m\<ge>n. X n = X m"
+ fix X::"nat\<Rightarrow>'a discrete"
+ assume "Cauchy X"
+ then obtain n where "\<forall>m\<ge>n. X n = X m"
by (force simp: dist_discrete_def Cauchy_def split: if_split_asm dest:spec[where x=1])
- then guess n ..
thus "convergent X"
by (intro convergentI[where L="X n"] tendstoI eventually_sequentiallyI[of n])
(simp add: dist_discrete_def)