src/HOL/Presburger.thy
changeset 14758 af3b71a46a1c
parent 14738 83f1a514dcb4
child 14941 1edb674e0c33
--- a/src/HOL/Presburger.thy	Wed May 19 11:21:19 2004 +0200
+++ b/src/HOL/Presburger.thy	Wed May 19 11:23:59 2004 +0200
@@ -978,11 +978,11 @@
   \medskip Specific instances of congruence rules, to prevent
   simplifier from looping. *}
 
-theorem imp_le_cong: "(0 <= x \<Longrightarrow> P = P') \<Longrightarrow> (0 <= (x::nat) \<longrightarrow> P) = (0 <= x \<longrightarrow> P')"
+theorem imp_le_cong: "(0 <= x \<Longrightarrow> P = P') \<Longrightarrow> (0 <= (x::int) \<longrightarrow> P) = (0 <= x \<longrightarrow> P')"
   by simp
 
-theorem conj_le_cong: "(0 <= x \<Longrightarrow> P = P') \<Longrightarrow> (0 <= (x::nat) \<and> P) = (0 <= x \<and> P')"
-  by simp
+theorem conj_le_cong: "(0 <= x \<Longrightarrow> P = P') \<Longrightarrow> (0 <= (x::int) \<and> P) = (0 <= x \<and> P')"
+  by (simp cong: conj_cong)
 
 use "cooper_dec.ML"
 use "cooper_proof.ML"