explicit is better than implicit;
authorwenzelm
Thu, 05 Jul 2012 17:18:55 +0200
changeset 48196 b7313810b6e6
parent 48195 3127f9ce52fb
child 48197 b13dd10ebc77
explicit is better than implicit;
src/HOL/Word/Word.thy
--- a/src/HOL/Word/Word.thy	Thu Jul 05 16:58:03 2012 +0200
+++ b/src/HOL/Word/Word.thy	Thu Jul 05 17:18:55 2012 +0200
@@ -2344,7 +2344,10 @@
   fixes x' :: "'a::len0 word"
   shows "(w' = (x' AND y')) \<Longrightarrow> (x' = (x' OR w'))" by auto 
 
-lemmas word_ao_equiv = leao [COMP leoa [COMP iffI]]
+lemma word_ao_equiv:
+  fixes w w' :: "'a::len0 word"
+  shows "(w = w OR w') = (w' = w AND w')"
+  by (auto intro: leoa leao)
 
 lemma le_word_or2: "x <= x OR (y::'a::len0 word)"
   unfolding word_le_def uint_or