src/HOLCF/Sprod.thy
changeset 36452 d37c6eed8117
parent 35900 aa5dfb03eb1e
child 39973 c62b4ff97bfc
equal deleted inserted replaced
36451:ddc965e172c4 36452:d37c6eed8117
     6 
     6 
     7 theory Sprod
     7 theory Sprod
     8 imports Bifinite
     8 imports Bifinite
     9 begin
     9 begin
    10 
    10 
    11 defaultsort pcpo
    11 default_sort pcpo
    12 
    12 
    13 subsection {* Definition of strict product type *}
    13 subsection {* Definition of strict product type *}
    14 
    14 
    15 pcpodef (Sprod)  ('a, 'b) sprod (infixr "**" 20) =
    15 pcpodef (Sprod)  ('a, 'b) sprod (infixr "**" 20) =
    16         "{p::'a \<times> 'b. p = \<bottom> \<or> (fst p \<noteq> \<bottom> \<and> snd p \<noteq> \<bottom>)}"
    16         "{p::'a \<times> 'b. p = \<bottom> \<or> (fst p \<noteq> \<bottom> \<and> snd p \<noteq> \<bottom>)}"