Skip to content

Commit

Permalink
chore: remove shadowed variable name (#17272)
Browse files Browse the repository at this point in the history
The variable name `H` was repeated.  The ambiguity could potentially be an issue for using `apply lemma_name (H := x)`.

Found while working on the unused variable command linter.
  • Loading branch information
adomani committed Sep 30, 2024
1 parent c07cbe1 commit 71a8921
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/RingTheory/IsTensorProduct.lean
Original file line number Diff line number Diff line change
Expand Up @@ -424,7 +424,7 @@ noncomputable def Algebra.pushoutDesc [H : Algebra.IsPushout R S R' S'] {A : Typ
rw [mul_add, map_add, map_add, mul_add, e₁, e₂]

@[simp]
theorem Algebra.pushoutDesc_left [H : Algebra.IsPushout R S R' S'] {A : Type*} [Semiring A]
theorem Algebra.pushoutDesc_left [Algebra.IsPushout R S R' S'] {A : Type*} [Semiring A]
[Algebra R A] (f : S →ₐ[R] A) (g : R' →ₐ[R] A) (H) (x : S) :
Algebra.pushoutDesc S' f g H (algebraMap S S' x) = f x := by
letI := Module.compHom A f.toRingHom
Expand All @@ -442,7 +442,7 @@ theorem Algebra.lift_algHom_comp_left [Algebra.IsPushout R S R' S'] {A : Type*}
AlgHom.ext fun x => (Algebra.pushoutDesc_left S' f g H x : _)

@[simp]
theorem Algebra.pushoutDesc_right [H : Algebra.IsPushout R S R' S'] {A : Type*} [Semiring A]
theorem Algebra.pushoutDesc_right [Algebra.IsPushout R S R' S'] {A : Type*} [Semiring A]
[Algebra R A] (f : S →ₐ[R] A) (g : R' →ₐ[R] A) (H) (x : R') :
Algebra.pushoutDesc S' f g H (algebraMap R' S' x) = g x :=
letI := Module.compHom A f.toRingHom
Expand Down

0 comments on commit 71a8921

Please sign in to comment.