diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Parity.thy --- a/src/HOL/Parity.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Parity.thy Fri Jan 04 23:22:53 2019 +0100 @@ -454,7 +454,7 @@ end -subsection \Instance for @{typ nat}\ +subsection \Instance for \<^typ>\nat\\ instance nat :: semiring_parity by standard (simp_all add: dvd_eq_mod_eq_0) @@ -679,7 +679,7 @@ end -subsection \Instance for @{typ int}\ +subsection \Instance for \<^typ>\int\\ instance int :: ring_parity by standard (simp_all add: dvd_eq_mod_eq_0 divide_int_def division_segment_int_def) @@ -706,7 +706,7 @@ begin text \The primary purpose of the following operations is - to avoid ad-hoc simplification of concrete expressions @{term "2 ^ n"}\ + to avoid ad-hoc simplification of concrete expressions \<^term>\2 ^ n\\ definition push_bit :: "nat \ 'a \ 'a" where push_bit_eq_mult: "push_bit n a = a * 2 ^ n"