src/HOL/Main.thy
changeset 68980 5717fbc55521
parent 67385 deb9b0283259
child 69275 9bbd5497befd
equal deleted inserted replaced
68979:e2244e5707dd 68980:5717fbc55521
    20 no_notation
    20 no_notation
    21   bot ("\<bottom>") and
    21   bot ("\<bottom>") and
    22   top ("\<top>") and
    22   top ("\<top>") and
    23   inf (infixl "\<sqinter>" 70) and
    23   inf (infixl "\<sqinter>" 70) and
    24   sup (infixl "\<squnion>" 65) and
    24   sup (infixl "\<squnion>" 65) and
    25   Inf ("\<Sqinter>_" [900] 900) and
    25   Inf ("\<Sqinter> _" [900] 900) and
    26   Sup ("\<Squnion>_" [900] 900) and
    26   Sup ("\<Squnion> _" [900] 900) and
    27   ordLeq2 (infix "<=o" 50) and
    27   ordLeq2 (infix "<=o" 50) and
    28   ordLeq3 (infix "\<le>o" 50) and
    28   ordLeq3 (infix "\<le>o" 50) and
    29   ordLess2 (infix "<o" 50) and
    29   ordLess2 (infix "<o" 50) and
    30   ordIso2 (infix "=o" 50) and
    30   ordIso2 (infix "=o" 50) and
    31   card_of ("|_|") and
    31   card_of ("|_|") and