diff -r a9b20bc32fa6 -r ead56ad40e15 src/HOL/Main.thy --- a/src/HOL/Main.thy Mon Sep 20 23:15:02 2021 +0200 +++ b/src/HOL/Main.thy Tue Sep 21 00:20:47 2021 +0200 @@ -19,7 +19,7 @@ GCD begin -text \Namespace cleanup\ +subsection \Namespace cleanup\ hide_const (open) czero cinfinite cfinite csum cone ctwo Csum cprod cexp image2 image2p vimage2p Gr Grp collect @@ -29,15 +29,9 @@ hide_fact (open) id_bnf_def type_definition_id_bnf_UNIV -text \Syntax cleanup\ +subsection \Syntax cleanup\ no_notation - bot ("\") and - top ("\") and - inf (infixl "\" 70) and - sup (infixl "\" 65) and - Inf ("\") and - Sup ("\") and ordLeq2 (infix "<=o" 50) and ordLeq3 (infix "\o" 50) and ordLess2 (infix "(_,/ _)\") -bundle cardinal_syntax begin +bundle cardinal_syntax +begin + notation ordLeq2 (infix "<=o" 50) and ordLeq3 (infix "\o" 50) and @@ -63,8 +59,42 @@ alias czero = BNF_Cardinal_Arithmetic.czero alias cone = BNF_Cardinal_Arithmetic.cone alias ctwo = BNF_Cardinal_Arithmetic.ctwo + end + +subsection \Lattice syntax\ + +bundle lattice_syntax +begin + +notation + bot ("\") and + top ("\") and + inf (infixl "\" 70) and + sup (infixl "\" 65) and + Inf ("\ _" [900] 900) and + Sup ("\ _" [900] 900) + +syntax + "_INF1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) + "_INF" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) + "_SUP1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) + "_SUP" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) + +end + +bundle no_lattice_syntax +begin + +no_notation + bot ("\") and + top ("\") and + inf (infixl "\" 70) and + sup (infixl "\" 65) and + Inf ("\ _" [900] 900) and + Sup ("\ _" [900] 900) + no_syntax "_INF1" :: "pttrns \ 'b \ 'b" ("(3\_./ _)" [0, 10] 10) "_INF" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) @@ -72,3 +102,8 @@ "_SUP" :: "pttrn \ 'a set \ 'b \ 'b" ("(3\_\_./ _)" [0, 0, 10] 10) end + +unbundle no_lattice_syntax +no_notation Inf ("\") and Sup ("\") + +end