changeset 81091 | c007e6d9941d |
parent 81090 | 843dba3d307a |
child 81130 | 7dd81ffaac72 |
--- a/src/HOL/Quotient_Examples/Quotient_FSet.thy Mon Sep 30 23:32:26 2024 +0200 +++ b/src/HOL/Quotient_Examples/Quotient_FSet.thy Tue Oct 01 20:39:16 2024 +0200 @@ -290,8 +290,6 @@ syntax "_fset" :: "args => 'a fset" (\<open>(\<open>indent=2 notation=\<open>mixfix finite set enumeration\<close>\<close>{|_|})\<close>) -syntax_consts - insert_fset translations "{|x, xs|}" == "CONST insert_fset x {|xs|}" "{|x|}" == "CONST insert_fset x {||}"