Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a52ce83

Browse files
committed
feat(combinatorics/configuration): The order of a projective plane is at least 2 (#11550)
This PR proves that the order of a projective plane is strictly larger than 1.
1 parent 9150268 commit a52ce83

File tree

1 file changed

+23
-0
lines changed

1 file changed

+23
-0
lines changed

src/combinatorics/configuration.lean

Lines changed: 23 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -395,6 +395,29 @@ variables (P) {L}
395395
lemma point_count_eq [projective_plane P L] (l : L) : point_count P l = order P L + 1 :=
396396
(line_count_eq (dual P) l).trans (congr_arg (λ n, n + 1) (dual.order P L))
397397

398+
variables (P L)
399+
400+
lemma one_lt_order [projective_plane P L] : 1 < order P L :=
401+
begin
402+
obtain ⟨p₁, p₂, p₃, l₁, l₂, l₃, -, -, h₂₁, h₂₂, h₂₃, h₃₁, h₃₂, h₃₃⟩ := @exists_config P L _ _,
403+
classical,
404+
rw [←add_lt_add_iff_right, ←point_count_eq, point_count, nat.card_eq_fintype_card],
405+
simp_rw [fintype.two_lt_card_iff, ne, subtype.ext_iff],
406+
have h := mk_point_ax (λ h, h₂₁ ((congr_arg _ h).mpr h₂₂)),
407+
exact ⟨⟨mk_point _, h.2⟩, ⟨p₂, h₂₂⟩, ⟨p₃, h₃₂⟩,
408+
ne_of_mem_of_not_mem h.1 h₂₁, ne_of_mem_of_not_mem h.1 h₃₁, ne_of_mem_of_not_mem h₂₃ h₃₃⟩,
409+
end
410+
411+
variables {P} (L)
412+
413+
lemma two_lt_line_count [projective_plane P L] (p : P) : 2 < line_count L p :=
414+
by simpa only [line_count_eq L p, nat.succ_lt_succ_iff] using one_lt_order P L
415+
416+
variables (P) {L}
417+
418+
lemma two_lt_point_count [projective_plane P L] (l : L) : 2 < point_count P l :=
419+
by simpa only [point_count_eq P l, nat.succ_lt_succ_iff] using one_lt_order P L
420+
398421
end projective_plane
399422

400423
end configuration

0 commit comments

Comments
 (0)