src/HOL/Int.thy
changeset 36719 d396f6f63d94
parent 36716 b09f3ad3208f
child 36749 a8dc19a352e6
--- a/src/HOL/Int.thy	Thu May 06 19:35:43 2010 +0200
+++ b/src/HOL/Int.thy	Thu May 06 23:11:56 2010 +0200
@@ -2025,6 +2025,14 @@
 
 lemmas half_gt_zero [simp] = half_gt_zero_iff [THEN iffD2, standard]
 
+lemma divide_Numeral1:
+  "(x::'a::{field, number_ring}) / Numeral1 = x"
+  by simp
+
+lemma divide_Numeral0:
+  "(x::'a::{field_inverse_zero, number_ring}) / Numeral0 = 0"
+  by simp
+
 
 subsection {* The divides relation *}