changeset 81091 | c007e6d9941d |
parent 81089 | 8042869c2072 |
child 81095 | 49c04500c5f9 |
--- a/src/HOL/HOLCF/ConvexPD.thy Mon Sep 30 23:32:26 2024 +0200 +++ b/src/HOL/HOLCF/ConvexPD.thy Tue Oct 01 20:39:16 2024 +0200 @@ -180,8 +180,6 @@ syntax "_convex_pd" :: "args \<Rightarrow> logic" (\<open>(\<open>indent=1 notation=\<open>mixfix convex_pd enumeration\<close>\<close>{_}\<natural>)\<close>) -syntax_consts - convex_add translations "{x,xs}\<natural>" == "{x}\<natural> \<union>\<natural> {xs}\<natural>" "{x}\<natural>" == "CONST convex_unit\<cdot>x"