src/HOLCF/ex/Pattern_Match.thy
changeset 40026 8f8f18a88685
parent 39557 fe5722fce758
child 40322 707eb30e8a53
equal deleted inserted replaced
40025:876689e6bbdf 40026:8f8f18a88685
   356 
   356 
   357 subsection {* ML code for generating definitions *}
   357 subsection {* ML code for generating definitions *}
   358 
   358 
   359 ML {*
   359 ML {*
   360 local open HOLCF_Library in
   360 local open HOLCF_Library in
       
   361 
       
   362 infixr 6 ->>;
       
   363 infix 9 ` ;
   361 
   364 
   362 val beta_rules =
   365 val beta_rules =
   363   @{thms beta_cfun cont_id cont_const cont2cont_Rep_CFun cont2cont_LAM'} @
   366   @{thms beta_cfun cont_id cont_const cont2cont_Rep_CFun cont2cont_LAM'} @
   364   @{thms cont2cont_fst cont2cont_snd cont2cont_Pair};
   367   @{thms cont2cont_fst cont2cont_snd cont2cont_Pair};
   365 
   368