Skip to content

Commit

Permalink
chore: remove an erw (leanprover-community#16445)
Browse files Browse the repository at this point in the history
  • Loading branch information
FR-vdash-bot committed Sep 3, 2024
1 parent fa76f8b commit 8525fd6
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/FractionalIdeal/Operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -226,7 +226,7 @@ theorem canonicalEquiv_symm : (canonicalEquiv S P P').symm = canonicalEquiv S P'
exact ⟨fun ⟨y, mem, Eq⟩ => ⟨y, mem, Eq⟩, fun ⟨y, mem, Eq⟩ => ⟨y, mem, Eq⟩⟩

theorem canonicalEquiv_flip (I) : canonicalEquiv S P P' (canonicalEquiv S P' P I) = I := by
rw [← canonicalEquiv_symm]; erw [RingEquiv.apply_symm_apply]
rw [← canonicalEquiv_symm, RingEquiv.symm_apply_apply]

@[simp]
theorem canonicalEquiv_canonicalEquiv (P'' : Type*) [CommRing P''] [Algebra R P'']
Expand Down

0 comments on commit 8525fd6

Please sign in to comment.