diff -r 24b17460ee60 -r 714fad33252e src/HOL/Divides.thy --- a/src/HOL/Divides.thy Fri Aug 19 05:49:10 2022 +0000 +++ b/src/HOL/Divides.thy Fri Aug 19 05:49:11 2022 +0000 @@ -62,8 +62,10 @@ text \Enable (lin)arith to deal with \<^const>\divide\ and \<^const>\modulo\ when these are applied to some constant that is of the form \<^term>\numeral k\:\ -declare split_zdiv [of _ _ \numeral k\, linarith_split] for k -declare split_zmod [of _ _ \numeral k\, linarith_split] for k +declare split_zdiv [of _ _ \numeral n\, linarith_split] for n +declare split_zdiv [of _ _ \- numeral n\, linarith_split] for n +declare split_zmod [of _ _ \numeral n\, linarith_split] for n +declare split_zmod [of _ _ \- numeral n\, linarith_split] for n lemma half_nonnegative_int_iff [simp]: \k div 2 \ 0 \ k \ 0\ for k :: int