src/HOLCF/Cfun1.thy
changeset 430 89e1986125fe
parent 243 c22b85994e17
child 1168 74be52691d62
equal deleted inserted replaced
429:888bbb4119f8 430:89e1986125fe
    16 
    16 
    17 arities "->" :: (pcpo,pcpo)term		(* No properties for ->'s range *)
    17 arities "->" :: (pcpo,pcpo)term		(* No properties for ->'s range *)
    18 
    18 
    19 consts  
    19 consts  
    20 	Cfun	:: "('a => 'b)set"
    20 	Cfun	:: "('a => 'b)set"
    21 	fapp	:: "('a -> 'b)=>('a => 'b)"	("(_[_])" [11,0] 1000)
    21 	fapp	:: "('a -> 'b)=>('a => 'b)"	("(_[_])" [1000,0] 1000)
    22 						(* usually Rep_Cfun *)
    22 						(* usually Rep_Cfun *)
    23 						(* application      *)
    23 						(* application      *)
    24 
    24 
    25 	fabs	:: "('a => 'b)=>('a -> 'b)"	(binder "LAM " 10)
    25 	fabs	:: "('a => 'b)=>('a -> 'b)"	(binder "LAM " 10)
    26 						(* usually Abs_Cfun *)
    26 						(* usually Abs_Cfun *)