# HG changeset patch # User wenzelm # Date 1727473665 -7200 # Node ID 2cc651d3ce8ed78de991439c461736575e2a8208 # Parent 7638776e097724b474e8e69d238b83d7edeab60a partial revert of d97fdabd9e2b, to build old documentation more reliably; diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/CTL/CTL.thy --- a/src/Doc/Tutorial/CTL/CTL.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/CTL/CTL.thy Fri Sep 27 23:47:45 2024 +0200 @@ -35,7 +35,7 @@ a new datatype and a new function.} \ (*<*) -primrec valid :: "state \ formula \ bool" (\(_ \ _)\ [80,80] 80) where +primrec valid :: "state \ formula \ bool" ("(_ \ _)" [80,80] 80) where "s \ Atom a = (a \ L s)" | "s \ Neg f = (~(s \ f))" | "s \ And f g = (s \ f \ s \ g)" | diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/CTL/PDL.thy --- a/src/Doc/Tutorial/CTL/PDL.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/CTL/PDL.thy Fri Sep 27 23:47:45 2024 +0200 @@ -26,7 +26,7 @@ \hbox{\valid s f\}. The definition is by recursion over the syntax: \ -primrec valid :: "state \ formula \ bool" (\(_ \ _)\ [80,80] 80) +primrec valid :: "state \ formula \ bool" ("(_ \ _)" [80,80] 80) where "s \ Atom a = (a \ L s)" | "s \ Neg f = (\(s \ f))" | diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/Documents/Documents.thy --- a/src/Doc/Tutorial/Documents/Documents.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/Documents/Documents.thy Fri Sep 27 23:47:45 2024 +0200 @@ -37,7 +37,7 @@ operation on boolean values illustrates typical infix declarations. \ -definition xor :: "bool \ bool \ bool" (infixl \[+]\ 60) +definition xor :: "bool \ bool \ bool" (infixl "[+]" 60) where "A [+] B \ (A \ \ B) \ (\ A \ B)" text \ @@ -138,7 +138,7 @@ hide_const xor setup \Sign.add_path "version1"\ (*>*) -definition xor :: "bool \ bool \ bool" (infixl \\\ 60) +definition xor :: "bool \ bool \ bool" (infixl "\" 60) where "A \ B \ (A \ \ B) \ (\ A \ B)" (*<*) setup \Sign.local_path\ @@ -156,10 +156,10 @@ hide_const xor setup \Sign.add_path "version2"\ (*>*) -definition xor :: "bool \ bool \ bool" (infixl \[+]\\ 60) +definition xor :: "bool \ bool \ bool" (infixl "[+]\" 60) where "A [+]\ B \ (A \ \ B) \ (\ A \ B)" -notation (xsymbols) xor (infixl \\\\ 60) +notation (xsymbols) xor (infixl "\\" 60) (*<*) setup \Sign.local_path\ (*>*) @@ -186,10 +186,10 @@ \ datatype currency = - Euro nat (\\\) - | Pounds nat (\\\) - | Yen nat (\\\) - | Dollar nat (\$\) + Euro nat ("\") + | Pounds nat ("\") + | Yen nat ("\") + | Dollar nat ("$") text \ \noindent Here the mixfix annotations on the rightmost column happen @@ -223,7 +223,7 @@ \x \ y\. We assume that a constant \sim\ of type \<^typ>\('a \ 'a) set\ has been introduced at this point.\ (*<*)consts sim :: "('a \ 'a) set"(*>*) -abbreviation sim2 :: "'a \ 'a \ bool" (infix \\\ 50) +abbreviation sim2 :: "'a \ 'a \ bool" (infix "\" 50) where "x \ y \ (x, y) \ sim" text \\noindent The given meta-equality is used as a rewrite rule @@ -238,10 +238,10 @@ stems from Isabelle/HOL itself: \ -abbreviation not_equal :: "'a \ 'a \ bool" (infixl \~=\\ 50) +abbreviation not_equal :: "'a \ 'a \ bool" (infixl "~=\" 50) where "x ~=\ y \ \ (x = y)" -notation (xsymbols) not_equal (infix \\\\ 50) +notation (xsymbols) not_equal (infix "\\" 50) text \\noindent The notation \\\ is introduced separately to restrict it to the \emph{xsymbols} mode. diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/Inductive/Star.thy --- a/src/Doc/Tutorial/Inductive/Star.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/Inductive/Star.thy Fri Sep 27 23:47:45 2024 +0200 @@ -15,7 +15,7 @@ \ inductive_set - rtc :: "('a \ 'a)set \ ('a \ 'a)set" (\_*\ [1000] 999) + rtc :: "('a \ 'a)set \ ('a \ 'a)set" ("_*" [1000] 999) for r :: "('a \ 'a)set" where rtc_refl[iff]: "(x,x) \ r*" diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/Misc/fakenat.thy --- a/src/Doc/Tutorial/Misc/fakenat.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/Misc/fakenat.thy Fri Sep 27 23:47:45 2024 +0200 @@ -8,7 +8,7 @@ It behaves approximately as if it were declared like this: \ -datatype nat = zero (\0\) | Suc nat +datatype nat = zero ("0") | Suc nat (*<*) end (*>*) diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/Protocol/Message.thy --- a/src/Doc/Tutorial/Protocol/Message.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/Protocol/Message.thy Fri Sep 27 23:47:45 2024 +0200 @@ -81,9 +81,9 @@ text\Concrete syntax: messages appear as \\A,B,NA\\, etc...\ nonterminal mtuple_args syntax - "" :: "'a \ mtuple_args" (\_\) - "_MTuple_args" :: "'a \ mtuple_args \ mtuple_args" (\_,/ _\) - "_MTuple" :: "['a, mtuple_args] \ 'a * 'b" (\(2\_,/ _\)\) + "" :: "'a \ mtuple_args" ("_") + "_MTuple_args" :: "'a \ mtuple_args \ mtuple_args" ("_,/ _") + "_MTuple" :: "['a, mtuple_args] \ 'a * 'b" ("(2\_,/ _\)") syntax_consts "_MTuple_args" "_MTuple" \ MPair translations diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/ToyList/ToyList.thy --- a/src/Doc/Tutorial/ToyList/ToyList.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/ToyList/ToyList.thy Fri Sep 27 23:47:45 2024 +0200 @@ -9,12 +9,12 @@ the concrete syntax and name space of theory \<^theory>\Main\ as follows. \ -no_notation Nil (\[]\) and Cons (infixr \#\ 65) and append (infixr \@\ 65) +no_notation Nil ("[]") and Cons (infixr "#" 65) and append (infixr "@" 65) hide_type list hide_const rev -datatype 'a list = Nil (\[]\) - | Cons 'a "'a list" (infixr \#\ 65) +datatype 'a list = Nil ("[]") + | Cons 'a "'a list" (infixr "#" 65) text\\noindent The datatype\index{datatype@\isacommand {datatype} (command)} @@ -47,7 +47,7 @@ in this order, because Isabelle insists on definition before use: \ -primrec app :: "'a list \ 'a list \ 'a list" (infixr \@\ 65) where +primrec app :: "'a list \ 'a list \ 'a list" (infixr "@" 65) where "[] @ ys = ys" | "(x # xs) @ ys = x # (xs @ ys)" diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/Types/Axioms.thy --- a/src/Doc/Tutorial/Types/Axioms.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/Types/Axioms.thy Fri Sep 27 23:47:45 2024 +0200 @@ -84,7 +84,7 @@ parameter \neutral\ together with its property:\ class monoidl = semigroup + - fixes neutral :: "'a" (\\\) + fixes neutral :: "'a" ("\") assumes neutl: "\ \ x = x" text \\noindent Again, we prove some instances, by providing @@ -140,7 +140,7 @@ text \\noindent To finish our small algebra example, we add a \group\ class:\ class group = monoidl + - fixes inv :: "'a \ 'a" (\\
_\ [81] 80) + fixes inv :: "'a \ 'a" ("\
_" [81] 80) assumes invl: "\
x \ x = \" text \\noindent We continue with a further example for abstract diff -r 7638776e0977 -r 2cc651d3ce8e src/Doc/Tutorial/Types/Overloading.thy --- a/src/Doc/Tutorial/Types/Overloading.thy Fri Sep 27 22:44:30 2024 +0200 +++ b/src/Doc/Tutorial/Types/Overloading.thy Fri Sep 27 23:47:45 2024 +0200 @@ -11,7 +11,7 @@ for arbitrary types by means of a type class:\ class plus = - fixes plus :: "'a \ 'a \ 'a" (infixl \\\ 70) + fixes plus :: "'a \ 'a \ 'a" (infixl "\" 70) text \\noindent This introduces a new class @{class [source] plus}, along with a constant @{const [source] plus} with nice infix syntax.