diff -r 65a546c2b8ed -r 7ef6ba42914b sum.thy --- a/sum.thy Mon Jan 24 16:03:03 1994 +0100 +++ b/sum.thy Wed Jan 26 17:53:27 1994 +0100 @@ -17,7 +17,7 @@ Abs_Sum :: "(['a,'b,bool] => bool) => 'a+'b" Inl :: "'a => 'a+'b" Inr :: "'b => 'a+'b" - case :: "['a+'b, 'a=>'c,'b=>'c] =>'c" + sum_case :: "['a+'b, 'a=>'c,'b=>'c] =>'c" rules Inl_Rep_def "Inl_Rep == (%a. %x y p. x=a & p)" Inr_Rep_def "Inr_Rep == (%b. %x y p. y=b & ~p)" @@ -29,6 +29,6 @@ (*defining the abstract constants*) Inl_def "Inl == (%a. Abs_Sum(Inl_Rep(a)))" Inr_def "Inr == (%b. Abs_Sum(Inr_Rep(b)))" - case_def "case == (%p f g. @z. (!x. p=Inl(x) --> z=f(x))\ -\ & (!y. p=Inr(y) --> z=g(y)))" + sum_case_def "sum_case == (%p f g. @z. (!x. p=Inl(x) --> z=f(x))\ +\ & (!y. p=Inr(y) --> z=g(y)))" end