src/Cube/LP.thy
author paulson
Wed, 03 Mar 1999 10:32:35 +0100
changeset 6297 5b9fbdfe22b7
parent 4583 6d9be46ea566
permissions -rw-r--r--
new theory of extending the state space


LP = Base +

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

end