src/HOL/Word/Word.thy
changeset 38857 97775f3e8722
parent 38527 f2709bc1e41f
child 39198 f967a16dfcdd
equal deleted inserted replaced
38856:168dba35ecf3 38857:97775f3e8722
   951 lemmas word_log_defs = word_and_def word_or_def word_xor_def word_not_def
   951 lemmas word_log_defs = word_and_def word_or_def word_xor_def word_not_def
   952 lemmas word_log_bin_defs = word_log_defs
   952 lemmas word_log_bin_defs = word_log_defs
   953 
   953 
   954 text {* Executable equality *}
   954 text {* Executable equality *}
   955 
   955 
   956 instantiation word :: ("{len0}") eq
   956 instantiation word :: (len0) equal
   957 begin
   957 begin
   958 
   958 
   959 definition eq_word :: "'a word \<Rightarrow> 'a word \<Rightarrow> bool" where
   959 definition equal_word :: "'a word \<Rightarrow> 'a word \<Rightarrow> bool" where
   960   "eq_word k l \<longleftrightarrow> HOL.eq (uint k) (uint l)"
   960   "equal_word k l \<longleftrightarrow> HOL.equal (uint k) (uint l)"
   961 
   961 
   962 instance proof
   962 instance proof
   963 qed (simp add: eq eq_word_def)
   963 qed (simp add: equal equal_word_def)
   964 
   964 
   965 end
   965 end
   966 
   966 
   967 
   967 
   968 subsection {* Word Arithmetic *}
   968 subsection {* Word Arithmetic *}