| changeset 61552 | 980dd46a03fb |
| parent 61531 | ab2e862263e7 |
| child 61609 | 77b453bd616f |
--- a/src/HOL/Int.thy Mon Nov 02 11:56:38 2015 +0100 +++ b/src/HOL/Int.thy Mon Nov 02 16:17:09 2015 +0100 @@ -686,6 +686,9 @@ lemma Ints_1 [simp]: "1 \<in> \<int>" using Ints_of_int [of "1"] by simp +lemma Ints_numeral [simp]: "numeral n \<in> \<int>" + by (subst of_nat_numeral [symmetric], rule Ints_of_nat) + lemma Ints_add [simp]: "a \<in> \<int> \<Longrightarrow> b \<in> \<int> \<Longrightarrow> a + b \<in> \<int>" apply (auto simp add: Ints_def) apply (rule range_eqI)