diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Quickcheck_Examples/Quickcheck_Lattice_Examples.thy --- a/src/HOL/Quickcheck_Examples/Quickcheck_Lattice_Examples.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Quickcheck_Examples/Quickcheck_Lattice_Examples.thy Fri Sep 20 19:51:08 2024 +0200 @@ -13,12 +13,12 @@ the standard default type \<^typ>\int\ is insufficient.\ notation - less_eq (infix "\" 50) and - less (infix "\" 50) and - top ("\") and - bot ("\") and - inf (infixl "\" 70) and - sup (infixl "\" 65) + less_eq (infix \\\ 50) and + less (infix \\\ 50) and + top (\\\) and + bot (\\\) and + inf (infixl \\\ 70) and + sup (infixl \\\ 65) declare [[quickcheck_narrowing_active = false, quickcheck_timeout = 3600]] @@ -133,11 +133,11 @@ no_notation - less_eq (infix "\" 50) and - less (infix "\" 50) and - inf (infixl "\" 70) and - sup (infixl "\" 65) and - top ("\") and - bot ("\") + less_eq (infix \\\ 50) and + less (infix \\\ 50) and + inf (infixl \\\ 70) and + sup (infixl \\\ 65) and + top (\\\) and + bot (\\\) end