author | wenzelm |
Fri, 18 Feb 2022 23:12:13 +0100 | |
changeset 75103 | a29d49a636ed |
parent 75101 | f0e2023f361a (diff) |
parent 75102 | 678fae02f9b3 (current diff) |
child 75104 | 08bb0d32b2e3 |
--- a/src/HOL/Set_Interval.thy Fri Feb 18 23:10:33 2022 +0100 +++ b/src/HOL/Set_Interval.thy Fri Feb 18 23:12:13 2022 +0100 @@ -1728,6 +1728,9 @@ "bij_betw of_nat N A \<longleftrightarrow> of_nat ` N = A" by (simp add: bij_betw_def) +lemma Nats_infinite: "infinite (\<nat> :: 'a set)" + by (metis Nats_def finite_imageD infinite_UNIV_char_0 inj_on_of_nat) + end context comm_monoid_set