# HG changeset patch # User Jian Xu # Date 1360940540 -28800 # Node ID bc6b6845d57c596ac71d45a88a08594b98846919 # Parent 3674347dd98ecb9309f6b0f9eb132e50798d8bd7 remove dead code in Abacus_mopup diff -r 3674347dd98e -r bc6b6845d57c thys/Abacus_Mopup.thy --- a/thys/Abacus_Mopup.thy Fri Feb 15 14:07:39 2013 +0000 +++ b/thys/Abacus_Mopup.thy Fri Feb 15 23:02:20 2013 +0800 @@ -666,20 +666,6 @@ lemma mod_ex2: "(a mod (2::nat) = 0) = (\ q. a = 2 * q)" by arith -(* -lemma [simp]: "(a mod 2 \ Suc 0) = (a mod 2 = 0) " -by arith - -lemma [simp]: "(a mod 2 \ 0) = (a mod 2 = Suc 0) " -by arith - - -lemma [simp]: "(2*q - Suc 0) div 2 = (q - 1)" -by arith - -lemma [simp]: "(Suc (2*q)) div 2 = q" -by arith -*) lemma mod_2: "x mod 2 = 0 \ x mod 2 = Suc 0" by arith @@ -858,8 +844,6 @@ done qed -(*we can use Hoare_plus here*) - lemma wf_mopup[intro]: "tm_wf (mopup n, 0)" apply(induct n, simp add: mopup.simps shift.simps mopup_b_def tm_wf.simps) apply(auto simp: mopup.simps shift.simps mopup_b_def tm_wf.simps)