changeset 81091 | c007e6d9941d |
parent 81090 | 843dba3d307a |
child 81182 | fc5066122e68 |
--- a/src/HOL/Prolog/Test.thy Mon Sep 30 23:32:26 2024 +0200 +++ b/src/HOL/Prolog/Test.thy Tue Oct 01 20:39:16 2024 +0200 @@ -20,8 +20,6 @@ syntax "_list" :: "args => 'a list" (\<open>(\<open>indent=1 notation=\<open>mixfix list enumeration\<close>\<close>[_])\<close>) -syntax_consts - Cons translations "[x, xs]" == "x#[xs]" "[x]" == "x#[]"