src/HOL/Product_Type.thy
changeset 18702 7dc7dcd63224
parent 18518 3b1dfa53e64f
child 18706 1e7562c7afe6
equal deleted inserted replaced
18701:98e6a0a011f3 18702:7dc7dcd63224
   772 *}
   772 *}
   773 attach (test) {*
   773 attach (test) {*
   774 fun gen_id_42 aG bG i = (aG i, bG i);
   774 fun gen_id_42 aG bG i = (aG i, bG i);
   775 *}
   775 *}
   776 
   776 
   777 consts_code
   777 code_alias
   778   "Pair"    ("(_,/ _)")
   778   "*" "Product_Type.*"
   779   "fst"     ("fst")
   779   "Pair" "Product_Type.Pair"
   780   "snd"     ("snd")
   780   "fst" "Product_Type.fst"
       
   781   "snd" "Product_Type.snd"
       
   782 
       
   783 code_primconst fst
       
   784 ml {*
       
   785 fun fst (x, y) = x;
       
   786 *}
       
   787 
       
   788 code_primconst snd
       
   789 ml {*
       
   790 fun snd (x, y) = y;
       
   791 *}
       
   792 
       
   793 code_syntax_tyco
       
   794   *
       
   795     ml (infix 2 "*")
       
   796     haskell (atom "(__,/ __)")
       
   797 
       
   798 code_syntax_const
       
   799   fst
       
   800     haskell (atom "fst")
       
   801   snd
       
   802     haskell (atom "snd")
   781 
   803 
   782 ML {*
   804 ML {*
   783 
   805 
   784 signature PRODUCT_TYPE_CODEGEN =
   806 signature PRODUCT_TYPE_CODEGEN =
   785 sig
   807 sig