src/HOL/Library/Z2.thy
changeset 74101 d804e93ae9ff
parent 74097 6d7be1227d02
child 74108 3146646a43a7
--- a/src/HOL/Library/Z2.thy	Sun Aug 01 23:18:13 2021 +0200
+++ b/src/HOL/Library/Z2.thy	Mon Aug 02 10:01:06 2021 +0000
@@ -5,11 +5,11 @@
 section \<open>The Field of Integers mod 2\<close>
 
 theory Z2
-imports Main "HOL-Library.Bit_Operations"
+imports Main
 begin
 
 text \<open>
-  Note that in most cases \<^typ>\<open>bool\<close> is appropriate hen a binary type is needed; the
+  Note that in most cases \<^typ>\<open>bool\<close> is appropriate when a binary type is needed; the
   type provided here, for historical reasons named \<^text>\<open>bit\<close>, is only needed if proper
   field operations are required.
 \<close>