src/HOLCF/Ssum1.thy
author paulson
Wed, 21 Aug 1996 13:22:23 +0200
changeset 1933 8b24773de6db
parent 1479 21eb5e156d91
child 2640 ee4dfce170a0
permissions -rw-r--r--
Addition of message NS5

(*  Title:      HOLCF/ssum1.thy
    ID:         $Id$
    Author:     Franz Regensburger
    Copyright   1993  Technische Universitaet Muenchen

Partial ordering for the strict sum ++
*)

Ssum1 = Ssum0 +

consts

  less_ssum     :: "[('a ++ 'b),('a ++ 'b)] => bool"    

rules

  less_ssum_def "less_ssum s1 s2 == (@z.
         (! u x.s1=Isinl(u) & s2=Isinl(x) --> z = (u << x))
        &(! v y.s1=Isinr(v) & s2=Isinr(y) --> z = (v << y))
        &(! u y.s1=Isinl(u) & s2=Isinr(y) --> z = (u = UU))
        &(! v x.s1=Isinr(v) & s2=Isinl(x) --> z = (v = UU)))"

end