src/ZF/IntArith.thy
changeset 46953 2b6e55924af3
parent 46821 ff6b0c1087f2
child 48891 c0eafbd55de3
equal deleted inserted replaced
46952:5e1bcfdcb175 46953:2b6e55924af3
    32 (** Combining of literal coefficients in sums of products **)
    32 (** Combining of literal coefficients in sums of products **)
    33 
    33 
    34 lemma zless_iff_zdiff_zless_0: "(x $< y) \<longleftrightarrow> (x$-y $< #0)"
    34 lemma zless_iff_zdiff_zless_0: "(x $< y) \<longleftrightarrow> (x$-y $< #0)"
    35   by (simp add: zcompare_rls)
    35   by (simp add: zcompare_rls)
    36 
    36 
    37 lemma eq_iff_zdiff_eq_0: "[| x: int; y: int |] ==> (x = y) \<longleftrightarrow> (x$-y = #0)"
    37 lemma eq_iff_zdiff_eq_0: "[| x \<in> int; y \<in> int |] ==> (x = y) \<longleftrightarrow> (x$-y = #0)"
    38   by (simp add: zcompare_rls)
    38   by (simp add: zcompare_rls)
    39 
    39 
    40 lemma zle_iff_zdiff_zle_0: "(x $<= y) \<longleftrightarrow> (x$-y $<= #0)"
    40 lemma zle_iff_zdiff_zle_0: "(x $<= y) \<longleftrightarrow> (x$-y $<= #0)"
    41   by (simp add: zcompare_rls)
    41   by (simp add: zcompare_rls)
    42 
    42