src/Cube/Lomega.thy
author paulson
Fri, 21 Nov 2003 11:15:40 +0100
changeset 14265 95b42e69436c
parent 4583 6d9be46ea566
permissions -rw-r--r--
HOL: installation of Ring_and_Field as the basis for Naturals and Reals


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