src/HOL/Int.thy
changeset 69700 7a92cbec7030
parent 69605 a96320074298
child 69791 195aeee8b30a
--- a/src/HOL/Int.thy	Sun Jan 20 17:15:49 2019 +0000
+++ b/src/HOL/Int.thy	Mon Jan 21 14:44:23 2019 +0000
@@ -1441,7 +1441,7 @@
    apply auto
   done
 
-lemma infinite_UNIV_int: "\<not> finite (UNIV::int set)"
+lemma infinite_UNIV_int [simp]: "\<not> finite (UNIV::int set)"
 proof
   assume "finite (UNIV::int set)"
   moreover have "inj (\<lambda>i::int. 2 * i)"