src/HOL/Auth/Kerberos_BAN.thy
changeset 25134 3d4953e88449
parent 25112 98824cc791c0
child 32406 9ea59bd1397a
--- a/src/HOL/Auth/Kerberos_BAN.thy	Sun Oct 21 14:21:54 2007 +0200
+++ b/src/HOL/Auth/Kerberos_BAN.thy	Sun Oct 21 14:53:44 2007 +0200
@@ -35,7 +35,7 @@
 
 text{*The authenticator only for one journey*}
 specification (authlife)
-  authlife_LB [iff]:    "0 < authlife"
+  authlife_LB [iff]:    "authlife \<noteq> 0"
     by blast
 
 abbreviation
@@ -133,7 +133,7 @@
 apply (rule_tac [2]
            bankerberos.Nil [THEN bankerberos.BK1, THEN bankerberos.BK2,
                              THEN bankerberos.BK3, THEN bankerberos.BK4])
-apply (possibility, simp_all (no_asm_simp) add: used_Cons neq0_conv)
+apply (possibility, simp_all (no_asm_simp) add: used_Cons)
 done
 
 subsection{*Lemmas for reasoning about predicate "Issues"*}