Theory Projective_Plane_Axioms
theory Projective_Plane_Axioms
imports Main
begin
text ‹
Contents:
\begin{itemize}
\item We introduce the types of points and lines and an incidence relation between them.
\item A set of axioms for the projective plane (the models of these axioms are
n-dimensional with $n\ge 2$).
\end{itemize}
›
section ‹The Axioms of the Projective Plane›
locale projective_plane =
fixes incid :: "'point ⇒ 'line ⇒ bool"
assumes ax1: "∃l. incid P l ∧ incid Q l"
assumes ax2: "∃P. incid P l ∧ incid P m"
assumes ax_uniqueness: "⟦incid P l; incid Q l; incid P m; incid Q m⟧ ⟹ P = Q ∨ l = m"
assumes ax3: "∃A B C D. distinct [A,B,C,D] ∧ (∀l.
(incid A l ∧ incid B l ⟶ ¬(incid C l) ∧ ¬(incid D l)) ∧
(incid A l ∧ incid C l ⟶ ¬(incid B l) ∧ ¬(incid D l)) ∧
(incid A l ∧ incid D l ⟶ ¬(incid B l) ∧ ¬(incid C l)) ∧
(incid B l ∧ incid C l ⟶ ¬(incid A l) ∧ ¬(incid D l)) ∧
(incid B l ∧ incid D l ⟶ ¬(incid A l) ∧ ¬(incid C l)) ∧
(incid C l ∧ incid D l ⟶ ¬(incid A l) ∧ ¬(incid B l)))"
end