src/Cube/L2.thy
author nipkow
Wed, 24 Jun 1998 13:59:45 +0200
changeset 5077 71043526295f
parent 4583 6d9be46ea566
permissions -rw-r--r--
* HOL/List: new function list_update written xs[i:=v] that updates the i-th list position. May also be iterated as in xs[i:=a,j:=b,...].


L2 = Base +

rules
  pi_bs         "[| A:[]; !!x. x:A ==> B(x):* |] ==> Prod(A,B):*"
  lam_bs        "[| A:[]; !!x. x:A ==> f(x):B(x); !!x. x:A ==> B(x):* |]
                   ==> Abs(A,f) : Prod(A,B)"

end