Skip to content

Commit

Permalink
chore: classify added dsimp only porting notes (#10753)
Browse files Browse the repository at this point in the history
Classifies by adding issue number (#10752) to porting notes claiming `added dsimp only`.
  • Loading branch information
pitmonticone committed Feb 20, 2024
1 parent c521802 commit ecce7d9
Show file tree
Hide file tree
Showing 3 changed files with 14 additions and 14 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Order/Interval.lean
Expand Up @@ -679,7 +679,7 @@ noncomputable instance completeLattice [@DecidableRel α (· ≤ ·)] :
lift s to NonemptyInterval α using ha
exact iInf₂_le_of_le s hs (le_iSup₂_of_le s hs s.fst_le_snd)⟩
le_sSup := fun s s ha => by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
split_ifs with h
· exact (h ha).le
cases s
Expand All @@ -693,7 +693,7 @@ noncomputable instance completeLattice [@DecidableRel α (· ≤ ·)] :
exact ha
· exact le_iSup₂_of_le _ ha le_rfl
sSup_le := fun s s ha => by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
split_ifs with h
· exact bot_le
obtain ⟨b, hs, hb⟩ := not_subset.1 h
Expand All @@ -713,7 +713,7 @@ noncomputable instance completeLattice [@DecidableRel α (· ≤ ·)] :
iSup₂_le fun s hs => le_iInf₂ <| h.2 hs⟩
else
sInf_le := fun s₁ s ha => by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
split_ifs with h
· lift s to NonemptyInterval α using ne_of_mem_of_not_mem ha h.1
-- Porting note: Lean failed to figure out the function `f` by itself,
Expand Down
20 changes: 10 additions & 10 deletions Mathlib/RingTheory/IsAdjoinRoot.lean
Expand Up @@ -215,17 +215,17 @@ where `S` is given by adjoining a root of `f` to `R`. -/
def lift (h : IsAdjoinRoot S f) : S →+* T where
toFun z := (h.repr z).eval₂ i x
map_zero' := by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [h.eval₂_repr_eq_eval₂_of_map_eq hx _ _ (map_zero _), eval₂_zero]
map_add' z w := by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [h.eval₂_repr_eq_eval₂_of_map_eq hx _ (h.repr z + h.repr w), eval₂_add]
· rw [map_add, map_repr, map_repr]
map_one' := by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [h.eval₂_repr_eq_eval₂_of_map_eq hx _ _ (map_one _), eval₂_one]
map_mul' z w := by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [h.eval₂_repr_eq_eval₂_of_map_eq hx _ (h.repr z * h.repr w), eval₂_mul]
· rw [map_mul, map_repr, map_repr]
#align is_adjoin_root.lift IsAdjoinRoot.lift
Expand Down Expand Up @@ -371,11 +371,11 @@ def modByMonicHom (h : IsAdjoinRootMonic S f) : S →ₗ[R] R[X] where
map_add' x y := by
conv_lhs =>
rw [← h.map_repr x, ← h.map_repr y, ← map_add]
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [h.modByMonic_repr_map, add_modByMonic]
map_smul' c x := by
rw [RingHom.id_apply, ← h.map_repr x, Algebra.smul_def, h.algebraMap_apply, ← map_mul]
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [h.modByMonic_repr_map, ← smul_eq_C_mul, smul_modByMonic, h.map_repr]
#align is_adjoin_root_monic.mod_by_monic_hom IsAdjoinRootMonic.modByMonicHom

Expand Down Expand Up @@ -435,24 +435,24 @@ def basis (h : IsAdjoinRootMonic S f) : Basis (Fin (natDegree f)) R S :=
ext i
simp only [h.modByMonicHom_map, Finsupp.comapDomain_apply, Polynomial.toFinsupp_apply]
rw [(Polynomial.modByMonic_eq_self_iff h.Monic).mpr, Polynomial.coeff]
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [Finsupp.mapDomain_apply Fin.val_injective]
rw [degree_eq_natDegree h.Monic.ne_zero, degree_lt_iff_coeff_zero]
intro m hm
rw [Polynomial.coeff]
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [Finsupp.mapDomain_notin_range]
rw [Set.mem_range, not_exists]
rintro i rfl
exact i.prop.not_le hm
map_add' := fun x y => by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [map_add, toFinsupp_add, Finsupp.comapDomain_add_of_injective Fin.val_injective]
-- Porting note: the original simp proof with the same lemmas does not work
-- See https://github.com/leanprover-community/mathlib4/issues/5026
-- simp only [map_add, Finsupp.comapDomain_add_of_injective Fin.val_injective, toFinsupp_add]
map_smul' := fun c x => by
dsimp only -- Porting note: added
dsimp only -- Porting note (#10752): added `dsimp only`
rw [map_smul, toFinsupp_smul, Finsupp.comapDomain_smul_of_injective Fin.val_injective,
RingHom.id_apply] }
-- Porting note: the original simp proof with the same lemmas does not work
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Gluing.lean
Expand Up @@ -390,7 +390,7 @@ def mk' (h : MkCore.{u}) : TopCat.GlueData where
V i := (Opens.toTopCat _).obj (h.V i.1 i.2)
f i j := (h.V i j).inclusion
f_id i := by
-- Porting note: added `dsimp only`
-- Porting note (#10752): added `dsimp only`
dsimp only
exact (h.V_id i).symm ▸ IsIso.of_iso (Opens.inclusionTopIso (h.U i))
f_open := fun i j : h.J => (h.V i j).openEmbedding
Expand Down

0 comments on commit ecce7d9

Please sign in to comment.