src/CCL/Type.thy
changeset 14765 bafb24c150c1
parent 3837 d7f033c74b38
child 17456 bcf7544875b2
equal deleted inserted replaced
14764:5d8a9900cabc 14765:bafb24c150c1
    25   TEx           :: "(i set => i set) => i set"       (binder "TEX " 55)
    25   TEx           :: "(i set => i set) => i set"       (binder "TEX " 55)
    26   Lift          :: "i set => i set"                  ("(3[_])")
    26   Lift          :: "i set => i set"                  ("(3[_])")
    27 
    27 
    28   SPLIT         :: "[i, [i, i] => i set] => i set"
    28   SPLIT         :: "[i, [i, i] => i set] => i set"
    29 
    29 
       
    30 syntax
    30   "@Pi"         :: "[idt, i set, i set] => i set"    ("(3PROD _:_./ _)"
    31   "@Pi"         :: "[idt, i set, i set] => i set"    ("(3PROD _:_./ _)"
    31                                 [0,0,60] 60)
    32                                 [0,0,60] 60)
    32 
    33 
    33   "@Sigma"      :: "[idt, i set, i set] => i set"    ("(3SUM _:_./ _)"
    34   "@Sigma"      :: "[idt, i set, i set] => i set"    ("(3SUM _:_./ _)"
    34                                 [0,0,60] 60)
    35                                 [0,0,60] 60)