src/HOL/Library/FuncSet.thy
changeset 14565 c6dc17aab88a
parent 13595 7e6cdcd113a2
child 14706 71590b7733b7
--- a/src/HOL/Library/FuncSet.thy	Wed Apr 14 13:28:46 2004 +0200
+++ b/src/HOL/Library/FuncSet.thy	Wed Apr 14 14:13:05 2004 +0200
@@ -30,6 +30,10 @@
   funcset :: "['a set, 'b set] => ('a => 'b) set"  (infixr "\<rightarrow>" 60) 
   "@lam" :: "[pttrn, 'a set, 'a => 'b] => ('a=>'b)"  ("(3\<lambda>_\<in>_./ _)" [0,0,3] 3)
 
+syntax (HTML output)
+  "@Pi" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set"  ("(3\<Pi> _\<in>_./ _)"   10)
+  "@lam" :: "[pttrn, 'a set, 'a => 'b] => ('a=>'b)"  ("(3\<lambda>_\<in>_./ _)" [0,0,3] 3)
+
 translations
   "PI x:A. B" => "Pi A (%x. B)"
   "A -> B"    => "Pi A (_K B)"