The Hahn-Banach theorem for real vectorspaces (Isabelle/Isar)
(by Gertrud Bauer, TU Munich);
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