diff -r 1a9decb8bfbc -r ae9e6218443d src/HOL/Library/Signed_Division.thy --- a/src/HOL/Library/Signed_Division.thy Mon Apr 10 23:21:47 2023 +0200 +++ b/src/HOL/Library/Signed_Division.thy Tue Apr 11 11:59:02 2023 +0000 @@ -1,7 +1,7 @@ (* Author: Stefan Berghofer et al. *) -subsection \Signed division: negative results rounded towards zero rather than minus infinity.\ +section \Signed division: negative results rounded towards zero rather than minus infinity.\ theory Signed_Division imports Main