src/HOL/UNITY/PPROD.thy
changeset 35054 a5db9779b026
parent 32960 69916a850301
child 35416 d8d7d1b785af
--- a/src/HOL/UNITY/PPROD.thy	Mon Feb 08 21:26:52 2010 +0100
+++ b/src/HOL/UNITY/PPROD.thy	Mon Feb 08 21:28:27 2010 +0100
@@ -11,17 +11,14 @@
 theory PPROD imports Lift_prog begin
 
 constdefs
-
   PLam  :: "[nat set, nat => ('b * ((nat=>'b) * 'c)) program]
             => ((nat=>'b) * 'c) program"
     "PLam I F == \<Squnion>i \<in> I. lift i (F i)"
 
 syntax
-  "@PLam" :: "[pttrn, nat set, 'b set] => (nat => 'b) set"
-              ("(3plam _:_./ _)" 10)
-
+  "_PLam" :: "[pttrn, nat set, 'b set] => (nat => 'b) set"  ("(3plam _:_./ _)" 10)
 translations
-  "plam x : A. B"   == "PLam A (%x. B)"
+  "plam x : A. B" == "CONST PLam A (%x. B)"
 
 
 (*** Basic properties ***)