src/HOL/Word/Word.thy
changeset 69605 a96320074298
parent 69064 5840724b1d71
child 70169 8bb835f10a39
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
  4500   for n :: "'a::len word"
  4500   for n :: "'a::len word"
  4501   by unat_arith
  4501   by unat_arith
  4502 
  4502 
  4503 declare bin_to_bl_def [simp]
  4503 declare bin_to_bl_def [simp]
  4504 
  4504 
  4505 ML_file "Tools/word_lib.ML"
  4505 ML_file \<open>Tools/word_lib.ML\<close>
  4506 ML_file "Tools/smt_word.ML"
  4506 ML_file \<open>Tools/smt_word.ML\<close>
  4507 
  4507 
  4508 hide_const (open) Word
  4508 hide_const (open) Word
  4509 
  4509 
  4510 end
  4510 end