src/HOL/Main.thy
changeset 55057 6b0fcbeebaba
parent 55056 b5c94200d081
child 55058 4e700eb471d4
equal deleted inserted replaced
55056:b5c94200d081 55057:6b0fcbeebaba
    15   bot ("\<bottom>") and
    15   bot ("\<bottom>") and
    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)
    20   Sup ("\<Squnion>_" [900] 900) and
       
    21   ordLeq2 ("<=o") and
       
    22   ordLeq3 ("\<le>o") and
       
    23   ordLess2 ("<o") and
       
    24   ordIso2 ("=o") and
       
    25   csum (infixr "+c" 65) and
       
    26   cprod (infixr "*c" 80) and
       
    27   cexp (infixr "^c" 90)
    21 
    28 
    22 no_syntax (xsymbols)
    29 no_syntax (xsymbols)
    23   "_INF1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Sqinter>_./ _)" [0, 10] 10)
    30   "_INF1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Sqinter>_./ _)" [0, 10] 10)
    24   "_INF"      :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"  ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10)
    31   "_INF"      :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'b \<Rightarrow> 'b"  ("(3\<Sqinter>_\<in>_./ _)" [0, 0, 10] 10)
    25   "_SUP1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Squnion>_./ _)" [0, 10] 10)
    32   "_SUP1"     :: "pttrns \<Rightarrow> 'b \<Rightarrow> 'b"           ("(3\<Squnion>_./ _)" [0, 10] 10)