diff -r 82f57315cade -r 7a92cbec7030 src/HOL/Int.thy --- 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: "\ finite (UNIV::int set)" +lemma infinite_UNIV_int [simp]: "\ finite (UNIV::int set)" proof assume "finite (UNIV::int set)" moreover have "inj (\i::int. 2 * i)"