Theory Higher_Projective_Space_Axioms
theory Higher_Projective_Space_Axioms
imports Main
begin
text ‹
Contents:
▪ We introduce the types of 'point and 'line and an incidence relation between them.
▪ A set of axioms for higher projective spaces, i.e. we allow models of dimension ‹>› 3.
›
section ‹The axioms for Higher Projective Geometry›
lemma distinct4_def:
"distinct [A,B,C,D] = ((A ≠ B) ∧ (A ≠ C) ∧ (A ≠ D) ∧ (B ≠ C) ∧ (B ≠ D) ∧ (C ≠ D))"
by auto
lemma distinct3_def:
"distinct [A,B,C] = ((A ≠ B) ∧ (A ≠ C) ∧ (B ≠ C))"
by auto
locale higher_projective_space =
fixes incid :: "'point ⇒ 'line ⇒ bool"
assumes ax1_existence: "∃l. (incid P l) ∧ (incid M l)"
assumes ax1_uniqueness: "(incid P k) ⟶ (incid M k) ⟶ (incid P l) ⟶ (incid M l) ⟶ (P = M) ∨ (k = l)"
assumes ax2: "distinct [A,B,C,D] ⟶ (incid A lAB ∧ incid B lAB)
⟶ (incid C lCD ∧ incid D lCD) ⟶ (incid A lAC ∧ incid C lAC) ⟶
(incid B lBD ∧ incid D lBD) ⟶ (∃I.(incid I lAB ∧ incid I lCD)) ⟶
(∃J.(incid J lAC ∧ incid J lBD))"
assumes ax3: "∃A B C. distinct [A,B,C] ∧ (incid A l) ∧ (incid B l) ∧ (incid C l)"
assumes ax4: "∃l m.∀P. ¬(incid P l ∧ incid P m)"
end