src/HOL/Quotient_Examples/Lift_FSet.thy
changeset 81182 fc5066122e68
parent 81091 c007e6d9941d
--- a/src/HOL/Quotient_Examples/Lift_FSet.thy	Fri Oct 18 11:44:05 2024 +0200
+++ b/src/HOL/Quotient_Examples/Lift_FSet.thy	Fri Oct 18 14:20:09 2024 +0200
@@ -97,6 +97,8 @@
 
 syntax
   "_fset" :: "args => 'a fset"  (\<open>(\<open>indent=2 notation=\<open>mixfix finite set enumeration\<close>\<close>{|_|})\<close>)
+syntax_consts
+  "_fset" == fcons
 translations
   "{|x, xs|}" == "CONST fcons x {|xs|}"
   "{|x|}"     == "CONST fcons x {||}"