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

Commit 8910f6d

Browse files
feat(ring_theory/discriminant): remove an assumption (#11359)
We remove a `nonempty` assumption.
1 parent fd51bda commit 8910f6d

File tree

1 file changed

+10
-7
lines changed

1 file changed

+10
-7
lines changed

src/ring_theory/discriminant.lean

Lines changed: 10 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -108,15 +108,18 @@ variables [module.finite K L] [is_separable K L] [is_alg_closed E]
108108
variables (b : ι → L) (pb : power_basis K L)
109109

110110
/-- Over a field, if `b` is linear independent, then `algebra.discr K b ≠ 0`. -/
111-
lemma discr_not_zero_of_linear_independent [nonempty ι]
111+
lemma discr_not_zero_of_linear_independent
112112
(hcard : fintype.card ι = finrank K L) (hli : linear_independent K b) : discr K b ≠ 0 :=
113113
begin
114-
classical,
115-
have := span_eq_top_of_linear_independent_of_card_eq_finrank hli hcard,
116-
rw [discr_def, trace_matrix_def],
117-
simp_rw [← basis.mk_apply hli this],
118-
rw [← trace_matrix_def, trace_matrix_of_basis, ← bilin_form.nondegenerate_iff_det_ne_zero],
119-
exact trace_form_nondegenerate _ _
114+
by_cases h : nonempty ι,
115+
{ classical,
116+
have := span_eq_top_of_linear_independent_of_card_eq_finrank hli hcard,
117+
rw [discr_def, trace_matrix_def],
118+
simp_rw [← basis.mk_apply hli this],
119+
rw [← trace_matrix_def, trace_matrix_of_basis, ← bilin_form.nondegenerate_iff_det_ne_zero],
120+
exact trace_form_nondegenerate _ _ },
121+
letI := not_nonempty_iff.1 h,
122+
simp [discr],
120123
end
121124

122125
/-- If `L/K` is a field extension and `b : ι → L`, then `discr K b` is the square of the

0 commit comments

Comments
 (0)