src/HOL/Library/Infinite_Set.thy
changeset 72097 496cfe488d72
parent 72095 cfb6c22a5636
child 72302 d7d90ed4c74e
--- a/src/HOL/Library/Infinite_Set.thy	Wed Aug 05 21:03:31 2020 +0100
+++ b/src/HOL/Library/Infinite_Set.thy	Thu Aug 06 13:07:23 2020 +0100
@@ -363,6 +363,13 @@
     unfolding bij_betw_def by (auto intro: enumerate_in_set)
 qed
 
+lemma 
+  fixes S :: "nat set"
+  assumes S: "infinite S"
+  shows range_enumerate: "range (enumerate S) = S" 
+    and strict_mono_enumerate: "strict_mono (enumerate S)"
+  by (auto simp add: bij_betw_imp_surj_on bij_enumerate assms strict_mono_def)
+
 text \<open>A pair of weird and wonderful lemmas from HOL Light.\<close>
 lemma finite_transitivity_chain:
   assumes "finite A"