diff -r f6e595e4f608 -r 261cd8722677 src/HOL/Fun.thy --- a/src/HOL/Fun.thy Mon Sep 23 12:59:10 2024 +0200 +++ b/src/HOL/Fun.thy Mon Sep 23 13:32:38 2024 +0200 @@ -45,11 +45,11 @@ subsection \The Composition Operator \f \ g\\ -definition comp :: "('b \ 'c) \ ('a \ 'b) \ 'a \ 'c" (infixl "\" 55) +definition comp :: "('b \ 'c) \ ('a \ 'b) \ 'a \ 'c" (infixl \\\ 55) where "f \ g = (\x. f (g x))" notation (ASCII) - comp (infixl "o" 55) + comp (infixl \o\ 55) lemma comp_apply [simp]: "(f \ g) x = f (g x)" by (simp add: comp_def) @@ -102,7 +102,7 @@ subsection \The Forward Composition Operator \fcomp\\ -definition fcomp :: "('a \ 'b) \ ('b \ 'c) \ 'a \ 'c" (infixl "\>" 60) +definition fcomp :: "('a \ 'b) \ ('b \ 'c) \ 'a \ 'c" (infixl \\>\ 60) where "f \> g = (\x. g (f x))" lemma fcomp_apply [simp]: "(f \> g) x = g (f x)" @@ -123,7 +123,7 @@ code_printing constant fcomp \ (Eval) infixl 1 "#>" -no_notation fcomp (infixl "\>" 60) +no_notation fcomp (infixl \\>\ 60) subsection \Mapping functions\ @@ -841,10 +841,10 @@ nonterminal updbinds and updbind syntax - "_updbind" :: "'a \ 'a \ updbind" ("(2_ :=/ _)") - "" :: "updbind \ updbinds" ("_") - "_updbinds":: "updbind \ updbinds \ updbinds" ("_,/ _") - "_Update" :: "'a \ updbinds \ 'a" ("_/'((_)')" [1000, 0] 900) + "_updbind" :: "'a \ 'a \ updbind" (\(2_ :=/ _)\) + "" :: "updbind \ updbinds" (\_\) + "_updbinds":: "updbind \ updbinds \ updbinds" (\_,/ _\) + "_Update" :: "'a \ updbinds \ 'a" (\_/'((_)')\ [1000, 0] 900) syntax_consts "_updbind" "_updbinds" "_Update" \ fun_upd