avoid slow proofs due to simp rules from 960509bfd47e;
authorwenzelm
Sat, 28 Oct 2017 16:12:29 +0200
changeset 66930 d4f7c6f14fa2
parent 66929 c19b17b72777
child 66931 4ff031d249b2
avoid slow proofs due to simp rules from 960509bfd47e;
src/HOL/SPARK/Examples/RIPEMD-160/Round.thy
--- a/src/HOL/SPARK/Examples/RIPEMD-160/Round.thy	Fri Oct 27 17:06:30 2017 +0200
+++ b/src/HOL/SPARK/Examples/RIPEMD-160/Round.thy	Sat Oct 28 16:12:29 2017 +0200
@@ -330,7 +330,7 @@
   from this[OF x_lower x_upper x_lower' x_upper' \<open>0 <= 0\<close> \<open>0 <= 79\<close>]
     \<open>0 \<le> ca\<close> \<open>0 \<le> ce\<close> x_lower x_lower'
   show ?thesis unfolding returns(1) returns(2) unfolding returns
-    by simp
+    by (simp del: mod_pos_pos_trivial mod_neg_neg_trivial)
 qed
 
 spark_vc procedure_round_62
@@ -415,7 +415,8 @@
     \<open>0 \<le> cla\<close> \<open>0 \<le> cle\<close> \<open>0 \<le> cra\<close> \<open>0 \<le> cre\<close> x_lower x_lower'
   show ?thesis unfolding \<open>loop__1__j + 1 + 1 = loop__1__j + 2\<close>
     unfolding returns(1) returns(2) unfolding returns
-    by simp
+    by (simp del: mod_pos_pos_trivial mod_neg_neg_trivial)
+
 qed
 
 spark_vc procedure_round_76