Skip to content

Commit

Permalink
chore: remove remaining cdots that were not · (#12146)
Browse files Browse the repository at this point in the history
A simple replacement `. --> ·`.

See #12143 for the source of these replacements.
  • Loading branch information
adomani committed Apr 15, 2024
1 parent 4932e9d commit 8a7f842
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
Original file line number Diff line number Diff line change
Expand Up @@ -394,7 +394,7 @@ def colimitPresheafObjIsoComponentwiseLimit (F : J ⥤ PresheafedSpace.{_, _, v}
refine' (F.obj (unop X)).presheaf.mapIso (eqToIso _)
simp only [Functor.op_obj, unop_op, op_inj_iff, Opens.map_coe, SetLike.ext'_iff,
Set.preimage_preimage]
refine congr_arg (Set.preimage . U.1) (funext fun x => ?_)
refine congr_arg (Set.preimage · U.1) (funext fun x => ?_)
erw [← TopCat.comp_app]
congr
exact ι_preservesColimitsIso_inv (forget C) F (unop X)
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Ideal/Over.lean
Original file line number Diff line number Diff line change
Expand Up @@ -396,7 +396,7 @@ theorem exists_ideal_over_prime_of_isIntegral_of_isPrime
refine' _root_.trans _ (_root_.trans (congr_arg (comap (Ideal.Quotient.mk
(comap (algebraMap R S) I))) hQ') _)
· rw [comap_comap]
exact congr_arg (comap . Q') (RingHom.ext fun r => rfl)
exact congr_arg (comap · Q') (RingHom.ext fun r => rfl)
· refine' _root_.trans (comap_map_of_surjective _ Quotient.mk_surjective _) (sup_eq_left.2 _)
simpa [← RingHom.ker_eq_comap_bot] using hIP

Expand Down

0 comments on commit 8a7f842

Please sign in to comment.