src/Sequents/Modal0.thy
changeset 74302 6bc96f31cafd
parent 69605 a96320074298
equal deleted inserted replaced
74301:ffe269e74bdd 74302:6bc96f31cafd
    18 syntax
    18 syntax
    19   "_Lstar"      :: "two_seqe"   ("(_)|L>(_)" [6,6] 5)
    19   "_Lstar"      :: "two_seqe"   ("(_)|L>(_)" [6,6] 5)
    20   "_Rstar"      :: "two_seqe"   ("(_)|R>(_)" [6,6] 5)
    20   "_Rstar"      :: "two_seqe"   ("(_)|R>(_)" [6,6] 5)
    21 
    21 
    22 ML \<open>
    22 ML \<open>
    23   fun star_tr c [s1, s2] = Const(c, dummyT) $ seq_tr s1 $ seq_tr s2;
    23   fun star_tr c [s1, s2] = Syntax.const c $ seq_tr s1 $ seq_tr s2;
    24   fun star_tr' c [s1, s2] = Const(c, dummyT) $ seq_tr' s1 $ seq_tr' s2;
    24   fun star_tr' c [s1, s2] = Syntax.const c $ seq_tr' s1 $ seq_tr' s2;
    25 \<close>
    25 \<close>
    26 
    26 
    27 parse_translation \<open>
    27 parse_translation \<open>
    28  [(\<^syntax_const>\<open>_Lstar\<close>, K (star_tr \<^const_syntax>\<open>Lstar\<close>)),
    28  [(\<^syntax_const>\<open>_Lstar\<close>, K (star_tr \<^const_syntax>\<open>Lstar\<close>)),
    29   (\<^syntax_const>\<open>_Rstar\<close>, K (star_tr \<^const_syntax>\<open>Rstar\<close>))]
    29   (\<^syntax_const>\<open>_Rstar\<close>, K (star_tr \<^const_syntax>\<open>Rstar\<close>))]