* 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