equal
deleted
inserted
replaced
16 top ("\<top>") and |
16 top ("\<top>") and |
17 inf (infixl "\<sqinter>" 70) and |
17 inf (infixl "\<sqinter>" 70) and |
18 sup (infixl "\<squnion>" 65) and |
18 sup (infixl "\<squnion>" 65) and |
19 Inf ("\<Sqinter>_" [900] 900) and |
19 Inf ("\<Sqinter>_" [900] 900) and |
20 Sup ("\<Squnion>_" [900] 900) and |
20 Sup ("\<Squnion>_" [900] 900) and |
21 ordLeq2 ("<=o") and |
21 ordLeq2 (infix "<=o" 50) and |
22 ordLeq3 ("\<le>o") and |
22 ordLeq3 (infix "\<le>o" 50) and |
23 ordLess2 ("<o") and |
23 ordLess2 (infix "<o" 50) and |
24 ordIso2 ("=o") and |
24 ordIso2 (infix "=o" 50) and |
25 csum (infixr "+c" 65) and |
25 csum (infixr "+c" 65) and |
26 cprod (infixr "*c" 80) and |
26 cprod (infixr "*c" 80) and |
27 cexp (infixr "^c" 90) |
27 cexp (infixr "^c" 90) |
28 |
28 |
29 no_syntax (xsymbols) |
29 no_syntax (xsymbols) |