diff -r 6ce0c8d59f5a -r ec121999a9cb src/HOL/Boolean_Algebras.thy --- a/src/HOL/Boolean_Algebras.thy Sun Oct 06 22:56:07 2024 +0200 +++ b/src/HOL/Boolean_Algebras.thy Tue Oct 08 12:10:35 2024 +0200 @@ -14,7 +14,7 @@ locale abstract_boolean_algebra = conj: abel_semigroup \(\<^bold>\)\ + disj: abel_semigroup \(\<^bold>\)\ for conj :: \'a \ 'a \ 'a\ (infixr \\<^bold>\\ 70) and disj :: \'a \ 'a \ 'a\ (infixr \\<^bold>\\ 65) + - fixes compl :: \'a \ 'a\ (\\<^bold>- _\ [81] 80) + fixes compl :: \'a \ 'a\ (\(\open_block notation=\prefix \<^bold>-\\\<^bold>- _)\ [81] 80) and zero :: \'a\ (\\<^bold>0\) and one :: \'a\ (\\<^bold>1\) assumes conj_disj_distrib: \x \<^bold>\ (y \<^bold>\ z) = (x \<^bold>\ y) \<^bold>\ (x \<^bold>\ z)\