Theory AxTriangleInequality
section ‹ AxTriangleInequality ›
text ‹ This theory declares the Triangle Inequality as an axiom.›
theory AxTriangleInequality
imports Norms
begin
text ‹ Although AxTriangleInequality can be proven rather than asserted we have
left it as an axiom to illustrate the flexibility of using Isabelle for mathematical
physics: well-known mathematical results can be asserted, leaving the researcher free
to concentrate on the physics. We can return later to prove the mathematical results
when time permits. ›
class AxTriangleInequality = Norms +
assumes AxTriangleInequality: "∀ p q . axTriangleInequality p q"
begin
end
end