File tree Expand file tree Collapse file tree 2 files changed +10
-2
lines changed Expand file tree Collapse file tree 2 files changed +10
-2
lines changed Original file line number Diff line number Diff line change @@ -362,6 +362,15 @@ lemma cancel_left {g₁ g₂ : A →ₐ[R] B} {f : B →ₐ[R] C} (hf : Function
362
362
end Semiring
363
363
end AlgHom
364
364
365
+ namespace AlgHomClass
366
+
367
+ @[simp]
368
+ lemma toRingHom_toAlgHom {R A B : Type *} [CommSemiring R] [Semiring A] [Semiring B] [Algebra R A]
369
+ [Algebra R B] {F : Type *} [FunLike F A B] [AlgHomClass F R A B] (f : F) :
370
+ RingHomClass.toRingHom (AlgHomClass.toAlgHom f) = RingHomClass.toRingHom f := rfl
371
+
372
+ end AlgHomClass
373
+
365
374
namespace RingHom
366
375
367
376
variable {R S : Type *}
Original file line number Diff line number Diff line change @@ -482,8 +482,7 @@ def _root_.Subalgebra.valA (p : Subalgebra R A) : p →A[R] A where
482
482
toAlgHom := p.val
483
483
484
484
@[simp, norm_cast]
485
- theorem _root_.Subalgebra.coe_valA (p : Subalgebra R A) :
486
- (p.valA : p →ₐ[R] A) = p.subtype :=
485
+ theorem _root_.Subalgebra.coe_valA (p : Subalgebra R A) : p.valA = p.subtype :=
487
486
rfl
488
487
489
488
@[simp]
You can’t perform that action at this time.
0 commit comments