# HG changeset patch # User wenzelm # Date 1727731946 -7200 # Node ID 843dba3d307acc0e41fefa17300459e2a80abc1e # Parent 8042869c2072f3b80952b252dcd128c78466d079 clarified syntax: use outer block (with indent); diff -r 8042869c2072 -r 843dba3d307a src/Doc/Datatypes/Datatypes.thy --- a/src/Doc/Datatypes/Datatypes.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/Doc/Datatypes/Datatypes.thy Mon Sep 30 23:32:26 2024 +0200 @@ -454,7 +454,7 @@ \ (*<*) no_syntax - "_list" :: "args => 'a list" (\[(\notation=\mixfix list enumeration\\_)]\) + "_list" :: "args => 'a list" (\(\indent=1 notation=\mixfix list enumeration\\[_])\) (*>*) syntax "_list" :: "args \ 'a list" (\[(_)]\) diff -r 8042869c2072 -r 843dba3d307a src/HOL/Codegenerator_Test/Code_Lazy_Test.thy --- a/src/HOL/Codegenerator_Test/Code_Lazy_Test.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Codegenerator_Test/Code_Lazy_Test.thy Mon Sep 30 23:32:26 2024 +0200 @@ -24,7 +24,7 @@ no_notation lazy_llist (\_\) syntax - "_llist" :: "args => 'a list" (\\<^bold>[(\notation=\mixfix lazy list enumeration\\_)\<^bold>]\) + "_llist" :: "args => 'a list" (\(\indent=1 notation=\mixfix lazy list enumeration\\\<^bold>[_\<^bold>])\) syntax_consts lazy_llist translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Computational_Algebra/Polynomial.thy --- a/src/HOL/Computational_Algebra/Polynomial.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Computational_Algebra/Polynomial.thy Mon Sep 30 23:32:26 2024 +0200 @@ -349,7 +349,7 @@ subsection \List-style syntax for polynomials\ syntax - "_poly" :: "args \ 'a poly" (\[:(\notation=\mixfix polynomial enumeration\\_):]\) + "_poly" :: "args \ 'a poly" (\(\indent=2 notation=\mixfix polynomial enumeration\\[:_:])\) syntax_consts pCons translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Library/FSet.thy --- a/src/HOL/Library/FSet.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Library/FSet.thy Mon Sep 30 23:32:26 2024 +0200 @@ -165,7 +165,7 @@ by simp syntax - "_fset" :: "args => 'a fset" (\{|(\notation=\mixfix finite set enumeration\\_)|}\) + "_fset" :: "args => 'a fset" (\(\indent=2 notation=\mixfix finite set enumeration\\{|_|})\) syntax_consts finsert translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Library/Multiset.thy Mon Sep 30 23:32:26 2024 +0200 @@ -92,7 +92,7 @@ by (rule add_mset_in_multiset) syntax - "_multiset" :: "args \ 'a multiset" (\{#(\notation=\mixfix multiset enumeration\\_)#}\) + "_multiset" :: "args \ 'a multiset" (\(\indent=2 notation=\mixfix multiset enumeration\\{#_#})\) syntax_consts add_mset translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/List.thy --- a/src/HOL/List.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/List.thy Mon Sep 30 23:32:26 2024 +0200 @@ -46,7 +46,7 @@ text \List enumeration\ syntax - "_list" :: "args => 'a list" (\[(\notation=\mixfix list enumeration\\_)]\) + "_list" :: "args => 'a list" (\(\indent=1 notation=\mixfix list enumeration\\[_])\) syntax_consts Cons translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Prolog/Test.thy --- a/src/HOL/Prolog/Test.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Prolog/Test.thy Mon Sep 30 23:32:26 2024 +0200 @@ -19,7 +19,7 @@ text \List enumeration\ syntax - "_list" :: "args => 'a list" (\[(\notation=\mixfix list enumeration\\_)]\) + "_list" :: "args => 'a list" (\(\indent=1 notation=\mixfix list enumeration\\[_])\) syntax_consts Cons translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Quotient_Examples/Lift_FSet.thy --- a/src/HOL/Quotient_Examples/Lift_FSet.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Quotient_Examples/Lift_FSet.thy Mon Sep 30 23:32:26 2024 +0200 @@ -96,7 +96,7 @@ end syntax - "_fset" :: "args => 'a fset" (\{|(\notation=\mixfix finite set enumeration\\_)|}\) + "_fset" :: "args => 'a fset" (\(\indent=2 notation=\mixfix finite set enumeration\\{|_|})\) syntax_consts fcons translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Quotient_Examples/Quotient_FSet.thy --- a/src/HOL/Quotient_Examples/Quotient_FSet.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Quotient_Examples/Quotient_FSet.thy Mon Sep 30 23:32:26 2024 +0200 @@ -289,7 +289,7 @@ is "Cons" by auto syntax - "_fset" :: "args => 'a fset" (\{|(\notation=\mixfix finite set enumeration\\_)|}\) + "_fset" :: "args => 'a fset" (\(\indent=2 notation=\mixfix finite set enumeration\\{|_|})\) syntax_consts insert_fset translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/Set.thy --- a/src/HOL/Set.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/Set.thy Mon Sep 30 23:32:26 2024 +0200 @@ -144,7 +144,7 @@ where insert_compr: "insert a B = {x. x = a \ x \ B}" syntax - "_Finset" :: "args \ 'a set" (\{(\notation=\mixfix set enumeration\\_)}\) + "_Finset" :: "args \ 'a set" (\(\indent=1 notation=\mixfix set enumeration\\{_})\) syntax_consts insert translations diff -r 8042869c2072 -r 843dba3d307a src/HOL/ex/Code_Lazy_Demo.thy --- a/src/HOL/ex/Code_Lazy_Demo.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/HOL/ex/Code_Lazy_Demo.thy Mon Sep 30 23:32:26 2024 +0200 @@ -40,7 +40,7 @@ | LCons (lhd: 'a) (ltl: "'a llist") (infixr \###\ 65) syntax - "_llist" :: "args => 'a list" (\\<^bold>\(\notation=\mixfix lazy list enumeration\\_)\<^bold>\\) + "_llist" :: "args => 'a list" (\(\indent=1 notation=\mixfix lazy list enumeration\\\<^bold>\_\<^bold>\)\) syntax_consts LCons translations diff -r 8042869c2072 -r 843dba3d307a src/ZF/List.thy --- a/src/ZF/List.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/ZF/List.thy Mon Sep 30 23:32:26 2024 +0200 @@ -16,7 +16,7 @@ notation Nil (\[]\) syntax - "_List" :: "is \ i" (\[(\notation=\mixfix list enumeration\\_)]\) + "_List" :: "is \ i" (\(\indent=1 notation=\mixfix list enumeration\\[_])\) syntax_consts Cons translations diff -r 8042869c2072 -r 843dba3d307a src/ZF/ZF_Base.thy --- a/src/ZF/ZF_Base.thy Mon Sep 30 22:57:45 2024 +0200 +++ b/src/ZF/ZF_Base.thy Mon Sep 30 23:32:26 2024 +0200 @@ -133,7 +133,7 @@ syntax "" :: "i \ is" (\_\) "_Enum" :: "[i, is] \ is" (\_,/ _\) - "_Finset" :: "is \ i" (\{(\notation=\mixfix set enumeration\\_)}\) + "_Finset" :: "is \ i" (\(\indent=1 notation=\mixfix set enumeration\\{_})\) syntax_consts cons translations @@ -196,7 +196,7 @@ syntax "" :: "i \ tuple_args" (\_\) "_Tuple_args" :: "[i, tuple_args] \ tuple_args" (\_,/ _\) - "_Tuple" :: "[i, tuple_args] \ i" (\\(\notation=\mixfix tuple enumeration\\_,/ _)\\) + "_Tuple" :: "[i, tuple_args] \ i" (\(\indent=1 notation=\mixfix tuple enumeration\\\_,/ _\)\) syntax_consts Pair translations