src/HOL/Word/BinGeneral.thy
changeset 25134 3d4953e88449
parent 24465 70f0214b3ecc
child 25349 0d46bea01741
--- a/src/HOL/Word/BinGeneral.thy	Sun Oct 21 14:21:54 2007 +0200
+++ b/src/HOL/Word/BinGeneral.thy	Sun Oct 21 14:53:44 2007 +0200
@@ -457,7 +457,7 @@
   we get a version for when the word length is given literally *)
 
 lemmas nat_non0_gr = 
-  trans [OF iszero_def [THEN Not_eq_iff [THEN iffD2]] neq0_conv, standard]
+  trans [OF iszero_def [THEN Not_eq_iff [THEN iffD2]] refl, standard]
 
 lemmas bintrunc_pred_simps [simp] = 
   bintrunc_minus_simps [of "number_of bin", simplified nobm1, standard]