src/CCL/Type.thy
changeset 81182 fc5066122e68
parent 81091 c007e6d9941d
--- a/src/CCL/Type.thy	Fri Oct 18 11:44:05 2024 +0200
+++ b/src/CCL/Type.thy	Fri Oct 18 14:20:09 2024 +0200
@@ -14,6 +14,8 @@
 
 syntax
   "_Subtype" :: "[idt, 'a set, o] \<Rightarrow> 'a set"  (\<open>(\<open>indent=1 notation=\<open>mixfix Subtype\<close>\<close>{_: _ ./ _})\<close>)
+syntax_consts
+  "_Subtype" == Subtype
 translations
   "{x: A. B}" == "CONST Subtype(A, \<lambda>x. B)"