src/HOL/HOLCF/Cfun.thy
changeset 45695 b108b3d7c49e
parent 45606 b1e1508643b1
child 49759 ecf1d5d87e5e
equal deleted inserted replaced
45694:4a8743618257 45695:b108b3d7c49e
    11 
    11 
    12 default_sort cpo
    12 default_sort cpo
    13 
    13 
    14 subsection {* Definition of continuous function type *}
    14 subsection {* Definition of continuous function type *}
    15 
    15 
    16 cpodef ('a, 'b) cfun (infixr "->" 0) = "{f::'a => 'b. cont f}"
    16 definition "cfun = {f::'a => 'b. cont f}"
    17 by (auto intro: cont_const adm_cont)
    17 
       
    18 cpodef (open) ('a, 'b) cfun (infixr "->" 0) = "cfun :: ('a => 'b) set"
       
    19   unfolding cfun_def by (auto intro: cont_const adm_cont)
    18 
    20 
    19 type_notation (xsymbols)
    21 type_notation (xsymbols)
    20   cfun  ("(_ \<rightarrow>/ _)" [1, 0] 0)
    22   cfun  ("(_ \<rightarrow>/ _)" [1, 0] 0)
    21 
    23 
    22 notation
    24 notation