This repository was archived by the owner on Jul 24, 2024. It is now read-only.
File tree Expand file tree Collapse file tree 2 files changed +17
-5
lines changed Expand file tree Collapse file tree 2 files changed +17
-5
lines changed Original file line number Diff line number Diff line change @@ -263,17 +263,29 @@ section hom_map
263
263
264
264
variables {S : Type w} [comm_ring S]
265
265
266
- lemma ring_hom.map_det {M : matrix n n R} { f : R →+* S} :
266
+ lemma _root_. ring_hom.map_det ( f : R →+* S) (M : matrix n n R) :
267
267
f M.det = matrix.det (f.map_matrix M) :=
268
268
by simp [matrix.det_apply', f.map_sum, f.map_prod]
269
269
270
- lemma alg_hom.map_det [algebra R S] {T : Type z} [comm_ring T] [algebra R T]
271
- {M : matrix n n S} {f : S →ₐ[R] T} :
270
+ lemma _root_.ring_equiv.map_det (f : R ≃+* S) (M : matrix n n R) :
271
+ f M.det = matrix.det (f.map_matrix M) :=
272
+ f.to_ring_hom.map_det _
273
+
274
+ lemma _root_.alg_hom.map_det [algebra R S] {T : Type z} [comm_ring T] [algebra R T]
275
+ (f : S →ₐ[R] T) (M : matrix n n S) :
272
276
f M.det = matrix.det ((f : S →+* T).map_matrix M) :=
273
- by rw [← alg_hom.coe_to_ring_hom, ring_hom.map_det]
277
+ f.to_ring_hom.map_det _
278
+
279
+ lemma _root_.alg_equiv.map_det [algebra R S] {T : Type z} [comm_ring T] [algebra R T]
280
+ (f : S ≃ₐ[R] T) (M : matrix n n S) :
281
+ f M.det = matrix.det ((f : S →+* T).map_matrix M) :=
282
+ f.to_alg_hom.map_det _
274
283
275
284
end hom_map
276
285
286
+ @[simp] lemma det_conj_transpose [star_ring R] (M : matrix m m R) : det (Mᴴ) = star (det M) :=
287
+ ((star_ring_aut : ring_aut R).map_det _).symm.trans $ congr_arg star M.det_transpose
288
+
277
289
section det_zero
278
290
/-!
279
291
### `det_zero` section
Original file line number Diff line number Diff line change @@ -359,7 +359,7 @@ begin
359
359
vandermonde (λ i, e.symm i pb.gen),
360
360
calc algebra_map K (algebraic_closure _) (bilin_form.to_matrix pb.basis (trace_form K L)).det
361
361
= det ((algebra_map K _).map_matrix $
362
- bilin_form.to_matrix pb.basis (trace_form K L)) : ring_hom.map_det
362
+ bilin_form.to_matrix pb.basis (trace_form K L)) : ring_hom.map_det _ _
363
363
... = det (Mᵀ ⬝ M) : _
364
364
... = det M * det M : by rw [det_mul, det_transpose]
365
365
... ≠ 0 : mt mul_self_eq_zero.mp _,
You can’t perform that action at this time.
0 commit comments