src/HOL/Integ/IntDef.thy
changeset 20217 25b068a99d2b
parent 20186 56207a6f4cc5
child 20254 58b71535ed00
equal deleted inserted replaced
20216:f30b73385060 20217:25b068a99d2b
   385     "nat z == contents (\<Union>(x,y) \<in> Rep_Integ z. { x-y })"
   385     "nat z == contents (\<Union>(x,y) \<in> Rep_Integ z. { x-y })"
   386 
   386 
   387 lemma nat: "nat (Abs_Integ (intrel``{(x,y)})) = x-y"
   387 lemma nat: "nat (Abs_Integ (intrel``{(x,y)})) = x-y"
   388 proof -
   388 proof -
   389   have "(\<lambda>(x,y). {x-y}) respects intrel"
   389   have "(\<lambda>(x,y). {x-y}) respects intrel"
   390     by (simp add: congruent_def, arith) 
   390     by (simp add: congruent_def, arith)
   391   thus ?thesis
   391   thus ?thesis
   392     by (simp add: nat_def UN_equiv_class [OF equiv_intrel])
   392     by (simp add: nat_def UN_equiv_class [OF equiv_intrel])
   393 qed
   393 qed
   394 
   394 
   395 lemma nat_int [simp]: "nat(int n) = n"
   395 lemma nat_int [simp]: "nat(int n) = n"