diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/SMT_Examples/SMT_Examples_Verit.thy --- a/src/HOL/SMT_Examples/SMT_Examples_Verit.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/SMT_Examples/SMT_Examples_Verit.thy Fri Sep 20 19:51:08 2024 +0200 @@ -683,8 +683,8 @@ fixes piecewise_C1 :: "('real :: {one,zero,ord} \ 'a :: {one,zero,ord}) \ 'real set \ bool" and joinpaths :: "('real \ 'a) \ ('real \ 'a) \ 'real \ 'a" begin -notation piecewise_C1 (infixr "piecewise'_C1'_differentiable'_on" 50) -notation joinpaths (infixr "+++" 75) +notation piecewise_C1 (infixr \piecewise'_C1'_differentiable'_on\ 50) +notation joinpaths (infixr \+++\ 75) lemma \(\v1. \v0. (rec_join v0 = v1 \ @@ -823,7 +823,7 @@ ground_resolution :: "'a \ 'a \ 'a \ bool" and is_least_false_clause :: "'afset \ 'a \ bool" and fset :: "'afset \ 'a set" and - union_fset :: "'afset \ 'afset \ 'afset" (infixr "|\|" 50) + union_fset :: "'afset \ 'afset \ 'afset" (infixr \|\|\ 50) begin term "a |\| b"