moved spurious auxiliary lemma here
authorhaftmann
Wed, 18 Aug 2010 14:55:10 +0200
changeset 38527 f2709bc1e41f
parent 38526 a9ce311eb6b9
child 38546 5c69afe3df06
moved spurious auxiliary lemma here
src/HOL/Word/Word.thy
--- a/src/HOL/Word/Word.thy	Wed Aug 18 14:55:10 2010 +0200
+++ b/src/HOL/Word/Word.thy	Wed Aug 18 14:55:10 2010 +0200
@@ -4034,6 +4034,11 @@
   "length (rotater n xs) = length xs"
   by (simp add : rotater_rev)
 
+lemma restrict_to_left:
+  assumes "x = y"
+  shows "(x = z) = (y = z)"
+  using assms by simp
+
 lemmas rrs0 = rotate_eqs [THEN restrict_to_left, 
   simplified rotate_gal [symmetric] rotate_gal' [symmetric], standard]
 lemmas rrs1 = rrs0 [THEN refl [THEN rev_iffD1]]