changeset 48 | 21291189b51e |
parent 0 | 7949f97df77a |
--- a/ex/simult.thy Thu Feb 24 14:45:57 1994 +0100 +++ b/ex/simult.thy Wed Mar 02 12:26:55 1994 +0100 @@ -50,7 +50,7 @@ "z: Part(TF(range(Leaf)),In1) ==> Rep_Forest(Abs_Forest(z)) = z" (*the concrete constants*) - TCONS_def "TCONS(M,N) == In0(M . N)" + TCONS_def "TCONS(M,N) == In0(M $ N)" FNIL_def "FNIL == In1(NIL)" FCONS_def "FCONS(M,N) == In1(CONS(M,N))" (*the abstract constants*)