src/HOL/UNITY/PPROD.thy
changeset 80768 c7723cc15de8
parent 69597 ff784d5a5bfb
child 80914 d97fdabd9e2b
--- a/src/HOL/UNITY/PPROD.thy	Sun Aug 25 20:54:20 2024 +0200
+++ b/src/HOL/UNITY/PPROD.thy	Sun Aug 25 21:10:01 2024 +0200
@@ -16,6 +16,8 @@
 
 syntax
   "_PLam" :: "[pttrn, nat set, 'b set] => (nat => 'b) set"  ("(3plam _:_./ _)" 10)
+syntax_consts
+  "_PLam" == PLam
 translations
   "plam x : A. B" == "CONST PLam A (%x. B)"