diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/ex/PER.thy --- a/src/HOL/ex/PER.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/ex/PER.thy Fri Sep 20 19:51:08 2024 +0200 @@ -32,7 +32,7 @@ \ class partial_equiv = - fixes eqv :: "'a \ 'a \ bool" (infixl "\" 50) + fixes eqv :: "'a \ 'a \ bool" (infixl \\\ 50) assumes partial_equiv_sym [elim?]: "x \ y \ y \ x" assumes partial_equiv_trans [trans]: "x \ y \ y \ z \ x \ z" @@ -168,7 +168,7 @@ representation of elements of a quotient type. \ -definition eqv_class :: "('a::partial_equiv) \ 'a quot" ("\_\") +definition eqv_class :: "('a::partial_equiv) \ 'a quot" (\\_\\) where "\a\ = Abs_quot {x. a \ x}" theorem quot_rep: "\a. A = \a\"