src/HOL/Library/Word.thy
changeset 30960 fec1a04b7220
parent 30224 79136ce06bdb
child 32438 620a5d8cfa78
--- a/src/HOL/Library/Word.thy	Wed Apr 22 19:09:19 2009 +0200
+++ b/src/HOL/Library/Word.thy	Wed Apr 22 19:09:21 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      HOL/Library/Word.thy
-    ID:         $Id$
     Author:     Sebastian Skalberg (TU Muenchen)
 *)
 
@@ -40,10 +39,8 @@
     Zero ("\<zero>")
   | One ("\<one>")
 
-primrec
-  bitval :: "bit => nat"
-where
-  "bitval \<zero> = 0"
+primrec bitval :: "bit => nat" where
+    "bitval \<zero> = 0"
   | "bitval \<one> = 1"
 
 consts
@@ -1531,7 +1528,7 @@
     show ?thesis
       apply simp
       apply (subst power_Suc [symmetric])
-      apply (simp del: power_int.simps)
+      apply simp
       done
   qed
   finally show ?thesis .