diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Library/Bit.thy --- a/src/HOL/Library/Bit.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Library/Bit.thy Fri Jan 04 23:22:53 2019 +0100 @@ -87,7 +87,7 @@ by (simp_all add: equal set_iff) -subsection \Type @{typ bit} forms a field\ +subsection \Type \<^typ>\bit\ forms a field\ instantiation bit :: field begin @@ -128,7 +128,7 @@ unfolding plus_bit_def by (simp split: bit.split) -subsection \Numerals at type @{typ bit}\ +subsection \Numerals at type \<^typ>\bit\\ text \All numerals reduce to either 0 or 1.\ @@ -145,7 +145,7 @@ by (simp only: numeral_Bit1 bit_add_self add_0_left) -subsection \Conversion from @{typ bit}\ +subsection \Conversion from \<^typ>\bit\\ context zero_neq_one begin