simplify some proofs
authorhuffman
Thu, 17 Nov 2011 06:04:59 +0100
changeset 45533 af3690f6bd79
parent 45532 74b17a0881b3
child 45534 4ab21521b393
child 45539 787a1a097465
simplify some proofs
src/HOL/Int.thy
--- a/src/HOL/Int.thy	Thu Nov 17 06:01:47 2011 +0100
+++ b/src/HOL/Int.thy	Thu Nov 17 06:04:59 2011 +0100
@@ -1277,22 +1277,13 @@
   by (simp add: Ints_def)
 
 lemma Ints_of_nat [simp]: "of_nat n \<in> \<int>"
-apply (simp add: Ints_def)
-apply (rule range_eqI)
-apply (rule of_int_of_nat_eq [symmetric])
-done
+  using Ints_of_int [of "of_nat n"] by simp
 
 lemma Ints_0 [simp]: "0 \<in> \<int>"
-apply (simp add: Ints_def)
-apply (rule range_eqI)
-apply (rule of_int_0 [symmetric])
-done
+  using Ints_of_int [of "0"] by simp
 
 lemma Ints_1 [simp]: "1 \<in> \<int>"
-apply (simp add: Ints_def)
-apply (rule range_eqI)
-apply (rule of_int_1 [symmetric])
-done
+  using Ints_of_int [of "1"] by simp
 
 lemma Ints_add [simp]: "a \<in> \<int> \<Longrightarrow> b \<in> \<int> \<Longrightarrow> a + b \<in> \<int>"
 apply (auto simp add: Ints_def)