Skip to content

Commit

Permalink
chore(ring_theory/polynomial/quotient): remove spurious restrict_scal…
Browse files Browse the repository at this point in the history
…ars (#18916)

Verifying that the `restrict_scalars` here is spurious. This proof is timing out badly in mathlib4.

If someone would like to merge this, please do so, but please then handle updating the SHA in mathlib4 as well. :-)



Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed May 3, 2023
1 parent 645b6de commit 61d8b82
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/ring_theory/polynomial/quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,7 @@ variables {R : Type*} [comm_ring R]
isomorphism of $R$-algebras $R[X] / \langle X - x \rangle \cong R$. -/
noncomputable def quotient_span_X_sub_C_alg_equiv (x : R) :
(R[X] ⧸ ideal.span ({X - C x} : set R[X])) ≃ₐ[R] R :=
(alg_equiv.restrict_scalars R $ ideal.quotient_equiv_alg_of_eq R
(ideal.quotient_equiv_alg_of_eq R
(by exact ker_eval_ring_hom x : ring_hom.ker (aeval x).to_ring_hom = _)).symm.trans $
ideal.quotient_ker_alg_equiv_of_right_inverse $ λ _, eval_C

Expand Down

0 comments on commit 61d8b82

Please sign in to comment.