changeset 81182 | fc5066122e68 |
parent 81091 | c007e6d9941d |
--- a/src/HOL/Prolog/Test.thy Fri Oct 18 11:44:05 2024 +0200 +++ b/src/HOL/Prolog/Test.thy Fri Oct 18 14:20:09 2024 +0200 @@ -20,6 +20,8 @@ syntax "_list" :: "args => 'a list" (\<open>(\<open>indent=1 notation=\<open>mixfix list enumeration\<close>\<close>[_])\<close>) +syntax_consts + "_list" \<rightleftharpoons> Cons translations "[x, xs]" == "x#[xs]" "[x]" == "x#[]"