src/CTT/CTT.thy
changeset 17782 b3846df9d643
parent 17441 5b5feca0344a
child 19761 5cd82054c2c6
equal deleted inserted replaced
17781:32bb237158a5 17782:b3846df9d643
    62   "@-->"    :: "[t,t]=>t"           ("(_ -->/ _)" [31,30] 30)
    62   "@-->"    :: "[t,t]=>t"           ("(_ -->/ _)" [31,30] 30)
    63   "@*"      :: "[t,t]=>t"           ("(_ */ _)" [51,50] 50)
    63   "@*"      :: "[t,t]=>t"           ("(_ */ _)" [51,50] 50)
    64 
    64 
    65 translations
    65 translations
    66   "PROD x:A. B" => "Prod(A, %x. B)"
    66   "PROD x:A. B" => "Prod(A, %x. B)"
    67   "A --> B"     => "Prod(A, _K(B))"
    67   "A --> B"     => "Prod(A, %_. B)"
    68   "SUM x:A. B"  => "Sum(A, %x. B)"
    68   "SUM x:A. B"  => "Sum(A, %x. B)"
    69   "A * B"       => "Sum(A, _K(B))"
    69   "A * B"       => "Sum(A, %_. B)"
    70 
    70 
    71 print_translation {*
    71 print_translation {*
    72   [("Prod", dependent_tr' ("@PROD", "@-->")),
    72   [("Prod", dependent_tr' ("@PROD", "@-->")),
    73    ("Sum", dependent_tr' ("@SUM", "@*"))]
    73    ("Sum", dependent_tr' ("@SUM", "@*"))]
    74 *}
    74 *}