src/HOL/Word/Bool_List_Representation.thy
changeset 57492 74bf65a1910a
parent 56073 29e308b56d23
child 57514 bdc2c6b40bf2
--- a/src/HOL/Word/Bool_List_Representation.thy	Wed Jul 02 17:34:45 2014 +0200
+++ b/src/HOL/Word/Bool_List_Representation.thy	Wed Jun 11 14:24:23 2014 +1000
@@ -595,7 +595,7 @@
 
 lemma takefill_same': 
   "l = length xs ==> takefill fill l xs = xs"
-  by clarify (induct xs, auto)
+  by (induct xs arbitrary: l, auto)
  
 lemmas takefill_same [simp] = takefill_same' [OF refl]