dropped group_simps, ring_simps, field_eq_simps; classes division_ring_inverse_zero, field_inverse_zero, linordered_field_inverse_zero
(* Title: HOL/Word/Word.thy
Author: Gerwin Klein, NICTA
*)
header {* Word Library interface *}
theory Word
imports WordGenLib
begin
text {* see @{text "Examples/WordExamples.thy"} for examples *}
end