Skip to content

Commit bad9e36

Browse files
committed
feat: add Basis.flag_le_ker_dual (#11265)
From sphere-eversion; I adapted the proof to mathlib's definition and golfed it a bit. This adds a new import; as this file is not imported anywhere, this seems fine.
1 parent 16cc6aa commit bad9e36

File tree

2 files changed

+9
-0
lines changed

2 files changed

+9
-0
lines changed

Mathlib/Data/Fin/Basic.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1082,6 +1082,9 @@ theorem coe_eq_castSucc {a : Fin n} : (a : Fin (n + 1)) = castSucc a := by
10821082
exact val_cast_of_lt (Nat.lt.step a.is_lt)
10831083
#align fin.coe_eq_cast_succ Fin.coe_eq_castSucc
10841084

1085+
theorem coe_succ_lt_iff_lt {n : ℕ} {j k : Fin n} : (j : Fin <| n + 1) < k ↔ j < k := by
1086+
simp only [coe_eq_castSucc]; rfl
1087+
10851088
#align fin.coe_succ_eq_succ Fin.coeSucc_eq_succ
10861089

10871090
#align fin.lt_succ Fin.lt_succ

Mathlib/LinearAlgebra/Basis/Flag.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yury Kudryashov, Patrick Massot
55
-/
66
import Mathlib.LinearAlgebra.Basis
7+
import Mathlib.LinearAlgebra.Dual
78
import Mathlib.Data.Fin.FlagRange
89

910
/-!
@@ -79,6 +80,11 @@ theorem flag_le_ker_coord (b : Basis (Fin n) R M) {k : Fin (n + 1)} {l : Fin n}
7980
nontriviality R
8081
exact b.flag_le_ker_coord_iff.2 h
8182

83+
theorem flag_le_ker_dual (b : Basis (Fin n) R M) (k : Fin n) :
84+
b.flag k.castSucc ≤ LinearMap.ker (b.dualBasis k) := by
85+
nontriviality R
86+
rw [coe_dualBasis, b.flag_le_ker_coord_iff]
87+
8288
end CommRing
8389

8490
section DivisionRing

0 commit comments

Comments
 (0)