Skip to content

Commit

Permalink
chore(combinatorics/configuration): don't use classical.some in a pro…
Browse files Browse the repository at this point in the history
…of (#12515)
  • Loading branch information
Ruben-VandeVelde committed Mar 8, 2022
1 parent ffa6e6d commit dc093e9
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/combinatorics/configuration.lean
Expand Up @@ -425,7 +425,7 @@ variables (P) (L)

lemma card_points [projective_plane P L] : fintype.card P = order P L ^ 2 + order P L + 1 :=
begin
let p : P := (classical.some (@exists_config P L _ _)),
obtain ⟨p, -⟩ := @exists_config P L _ _,
let ϕ : {q // q ≠ p} ≃ Σ (l : {l : L // p ∈ l}), {q // q ∈ l.1 ∧ q ≠ p} :=
{ to_fun := λ q, ⟨⟨mk_line q.2, (mk_line_ax q.2).2⟩, q, (mk_line_ax q.2).1, q.2⟩,
inv_fun := λ lq, ⟨lq.2, lq.2.2.2⟩,
Expand Down

0 comments on commit dc093e9

Please sign in to comment.