src/HOL/Auth/Public.thy
changeset 14133 4cd1a7e7edac
parent 14126 28824746d046
child 14200 d8598e24f8fa
--- a/src/HOL/Auth/Public.thy	Thu Jul 24 18:23:17 2003 +0200
+++ b/src/HOL/Auth/Public.thy	Fri Jul 25 10:52:15 2003 +0200
@@ -52,7 +52,10 @@
     "publicKey b A = publicKey c A' ==> b=c & A=A'"
    apply (rule exI [of _ "%b A. 2 * agent_case 0 (\<lambda>n. n + 2) 1 A + (if b then 1 else 0)"]) 
    apply (auto simp add: inj_on_def split: agent.split) 
+   apply presburger+
+(*faster would be this:
    apply (drule_tac f="%x. x mod 2" in arg_cong, simp add: mod_Suc)+
+*)
    done