src/Cube/Lomega.thy
author wenzelm
Mon, 04 Oct 1999 21:48:23 +0200
changeset 7707 1f4b67fdfdae
parent 4583 6d9be46ea566
permissions -rw-r--r--
simprocs now in IntArith;


Lomega = Base +

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

end