diff -r e1f6cd9f682e -r 5ef75ff3baeb src/HOLCF/Porder.thy --- a/src/HOLCF/Porder.thy Thu Mar 24 13:25:12 1994 +0100 +++ b/src/HOLCF/Porder.thy Thu Mar 24 13:36:34 1994 +0100 @@ -3,25 +3,13 @@ Author: Franz Regensburger Copyright 1993 Technische Universitaet Muenchen -Definition of class porder (partial order) - -The prototype theory for this class is void.thy +Conservative extension of theory Porder0 by constant definitions *) -Porder = Void + - -(* Introduction of new class. The witness is type void. *) - -classes po < term +Porder = Porder0 + -(* default type is still term ! *) -(* void is the prototype in po *) - -arities void :: po - -consts "<<" :: "['a,'a::po] => bool" (infixl 55) - +consts "<|" :: "['a set,'a::po] => bool" (infixl 55) "<<|" :: "['a set,'a::po] => bool" (infixl 55) lub :: "'a set => 'a::po" @@ -32,21 +20,6 @@ rules -(* class axioms: justification is theory Void *) - -refl_less "x << x" - (* witness refl_less_void *) - -antisym_less "[|x< x = y" - (* witness antisym_less_void *) - -trans_less "[|x< x<bool = less_void" - (* class definitions *) is_ub "S <| x == ! y.y:S --> y< (x< C(i) = C(j)"