src/HOL/Product_Type.thy
changeset 72739 e7c2848b78e8
parent 72581 de581f98a3a1
child 75669 43f5dfb7fa35
equal deleted inserted replaced
72738:a4d7da18ac5c 72739:e7c2848b78e8
   811 
   811 
   812 end
   812 end
   813 
   813 
   814 code_printing
   814 code_printing
   815   constant scomp \<rightharpoonup> (Eval) infixl 3 "#->"
   815   constant scomp \<rightharpoonup> (Eval) infixl 3 "#->"
   816 
       
   817 no_notation fcomp (infixl "\<circ>>" 60)
       
   818 no_notation scomp (infixl "\<circ>\<rightarrow>" 60)
       
   819 
   816 
   820 text \<open>
   817 text \<open>
   821   \<^term>\<open>map_prod\<close> --- action of the product functor upon functions.
   818   \<^term>\<open>map_prod\<close> --- action of the product functor upon functions.
   822 \<close>
   819 \<close>
   823 
   820