src/Cube/Cube.thy
changeset 52143 36ffe23b25f8
parent 49752 2bbb0013ff82
child 57945 cacb00a569e0
equal deleted inserted replaced
52142:348aed032cda 52143:36ffe23b25f8
    61 syntax (xsymbols)
    61 syntax (xsymbols)
    62   "_Pi" :: "[idt, term, term] => term"    ("(3\<Pi> _:_./ _)" [0, 0] 10)
    62   "_Pi" :: "[idt, term, term] => term"    ("(3\<Pi> _:_./ _)" [0, 0] 10)
    63 
    63 
    64 print_translation {*
    64 print_translation {*
    65   [(@{const_syntax Prod},
    65   [(@{const_syntax Prod},
    66     Syntax_Trans.dependent_tr' (@{syntax_const "_Pi"}, @{syntax_const "_arrow"}))]
    66     fn _ => Syntax_Trans.dependent_tr' (@{syntax_const "_Pi"}, @{syntax_const "_arrow"}))]
    67 *}
    67 *}
    68 
    68 
    69 axiomatization where
    69 axiomatization where
    70   s_b: "*: \<box>"  and
    70   s_b: "*: \<box>"  and
    71 
    71