diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/MicroJava/DFA/Semilat.thy --- a/src/HOL/MicroJava/DFA/Semilat.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/MicroJava/DFA/Semilat.thy Fri Sep 20 19:51:08 2024 +0200 @@ -25,26 +25,26 @@ where "plussub x f y = f x y" notation (ASCII) - "lesub" ("(_ /<='__ _)" [50, 1000, 51] 50) and - "lesssub" ("(_ /<'__ _)" [50, 1000, 51] 50) and - "plussub" ("(_ /+'__ _)" [65, 1000, 66] 65) + "lesub" (\(_ /<='__ _)\ [50, 1000, 51] 50) and + "lesssub" (\(_ /<'__ _)\ [50, 1000, 51] 50) and + "plussub" (\(_ /+'__ _)\ [65, 1000, 66] 65) notation - "lesub" ("(_ /\\<^bsub>_\<^esub> _)" [50, 0, 51] 50) and - "lesssub" ("(_ /\\<^bsub>_\<^esub> _)" [50, 0, 51] 50) and - "plussub" ("(_ /\\<^bsub>_\<^esub> _)" [65, 0, 66] 65) + "lesub" (\(_ /\\<^bsub>_\<^esub> _)\ [50, 0, 51] 50) and + "lesssub" (\(_ /\\<^bsub>_\<^esub> _)\ [50, 0, 51] 50) and + "plussub" (\(_ /\\<^bsub>_\<^esub> _)\ [65, 0, 66] 65) (* allow \ instead of \..\ *) abbreviation (input) - lesub1 :: "'a \ 'a ord \ 'a \ bool" ("(_ /\\<^sub>_ _)" [50, 1000, 51] 50) + lesub1 :: "'a \ 'a ord \ 'a \ bool" (\(_ /\\<^sub>_ _)\ [50, 1000, 51] 50) where "x \\<^sub>r y == x \\<^bsub>r\<^esub> y" abbreviation (input) - lesssub1 :: "'a \ 'a ord \ 'a \ bool" ("(_ /\\<^sub>_ _)" [50, 1000, 51] 50) + lesssub1 :: "'a \ 'a ord \ 'a \ bool" (\(_ /\\<^sub>_ _)\ [50, 1000, 51] 50) where "x \\<^sub>r y == x \\<^bsub>r\<^esub> y" abbreviation (input) - plussub1 :: "'a \ ('a \ 'b \ 'c) \ 'b \ 'c" ("(_ /\\<^sub>_ _)" [65, 1000, 66] 65) + plussub1 :: "'a \ ('a \ 'b \ 'c) \ 'b \ 'c" (\(_ /\\<^sub>_ _)\ [65, 1000, 66] 65) where "x \\<^sub>f y == x \\<^bsub>f\<^esub> y" definition ord :: "('a \ 'a) set \ 'a ord" where