src/Cube/L2.thy
author wenzelm
Thu, 18 Aug 2005 11:17:47 +0200
changeset 17112 736f4b7841a8
parent 4583 6d9be46ea566
permissions -rw-r--r--
moved after method.ML; moved FINDGOAL/HEADGOAL to method.ML; moved type method to method.ML; prepare attributes here; tuned various interfaces (cf. isar_thy.ML); tuned;


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