changeset 80768 | c7723cc15de8 |
parent 74563 | 042041c0ebeb |
child 80786 | 70076ba563d2 |
--- a/src/HOL/HOLCF/IOA/Sequence.thy Sun Aug 25 20:54:20 2024 +0200 +++ b/src/HOL/HOLCF/IOA/Sequence.thy Sun Aug 25 21:10:01 2024 +0200 @@ -72,6 +72,8 @@ syntax "_totlist" :: "args \<Rightarrow> 'a Seq" ("[(_)!]") "_partlist" :: "args \<Rightarrow> 'a Seq" ("[(_)?]") +syntax_consts + "_totlist" "_partlist" \<rightleftharpoons> Consq translations "[x, xs!]" \<rightleftharpoons> "x \<leadsto> [xs!]" "[x!]" \<rightleftharpoons> "x\<leadsto>nil"