Skip to content
New issue

Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.

By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.

Already on GitHub? Sign in to your account

Porting note: was simp #10745

Open
pitmonticone opened this issue Feb 20, 2024 · 1 comment
Open

Porting note: was simp #10745

pitmonticone opened this issue Feb 20, 2024 · 1 comment
Labels
porting-notes Mathlib3 to Mathlib4 porting notes.

Comments

@pitmonticone
Copy link
Collaborator

Classifies porting notes claiming was simp.

Examples

theorem Function.Surjective.isEngelian {f : L →ₗ⁅R⁆ L₂} (hf : Function.Surjective f)
(h : LieAlgebra.IsEngelian.{u₁, u₂, u₄} R L) : LieAlgebra.IsEngelian.{u₁, u₃, u₄} R L₂ := by
intro M _i1 _i2 _i3 _i4 h'
letI : LieRingModule L M := LieRingModule.compLieHom M f
letI : LieModule R L M := compLieHom M f
have hnp : ∀ x, IsNilpotent (toEndomorphism R L M x) := fun x => h' (f x)
have surj_id : Function.Surjective (LinearMap.id : M →ₗ[R] M) := Function.surjective_id
haveI : LieModule.IsNilpotent R L M := h M hnp
apply hf.lieModuleIsNilpotent surj_id
-- Porting note: was `simp`
intros; simp only [LinearMap.id_coe, id_eq]; rfl
#align function.surjective.is_engelian Function.Surjective.isEngelian

@[isROrC_simps] -- porting note: was `simp`
theorem conj_inv (x : K) : conj x⁻¹ = (conj x)⁻¹ :=
star_inv' _
#align is_R_or_C.conj_inv IsROrC.conj_inv

-- @[simp] -- Porting note: simp can prove this
theorem quotientInfEquivSupQuotient_symm_apply_eq_zero_iff {p p' : Submodule R M} {x : ↥(p ⊔ p')} :
(quotientInfEquivSupQuotient p p').symm (Submodule.Quotient.mk x) = 0 ↔ (x : M) ∈ p' :=
(LinearEquiv.symm_apply_eq _).trans <| by
-- Porting note: Was `simp`.
rw [_root_.map_zero, Quotient.mk_eq_zero, mem_comap, Submodule.coeSubtype]
#align linear_map.quotient_inf_equiv_sup_quotient_symm_apply_eq_zero_iff LinearMap.quotientInfEquivSupQuotient_symm_apply_eq_zero_iff

-- Porting note: was `simp`. LHS is not normal form.
-- @[simp, norm_cast]
@[norm_cast]
theorem natCast_pow {m n : ℕ} : (↑(m ^ n) : Cardinal) = (↑m : Cardinal) ^ (↑n : Cardinal) := by
induction n <;> simp [pow_succ', power_add, *, Pow.pow]
#align cardinal.nat_cast_pow Cardinal.natCast_pow

@pitmonticone pitmonticone added the porting-notes Mathlib3 to Mathlib4 porting notes. label Feb 20, 2024
mathlib-bors bot pushed a commit that referenced this issue Feb 20, 2024
Classifies by adding issue number (#10745) to porting notes claiming `was simp`.
mathlib-bors bot pushed a commit that referenced this issue Feb 21, 2024
Classifies by adding issue number (#10745) to porting note claiming anything semantically equivalent to `was simp`. 

Related merged PR: #10746.
mathlib-bors bot pushed a commit that referenced this issue Feb 21, 2024
Classifies by adding issue number (#10745) to porting note claiming anything semantically equivalent to `was simp`. 

Related merged PR: #10746.
thorimur pushed a commit that referenced this issue Feb 24, 2024
Classifies by adding issue number (#10745) to porting notes claiming `was simp`.
thorimur pushed a commit that referenced this issue Feb 24, 2024
Classifies by adding issue number (#10745) to porting note claiming anything semantically equivalent to `was simp`. 

Related merged PR: #10746.
thorimur pushed a commit that referenced this issue Feb 26, 2024
Classifies by adding issue number (#10745) to porting notes claiming `was simp`.
thorimur pushed a commit that referenced this issue Feb 26, 2024
Classifies by adding issue number (#10745) to porting note claiming anything semantically equivalent to `was simp`. 

Related merged PR: #10746.
riccardobrasca pushed a commit that referenced this issue Mar 1, 2024
Classifies by adding issue number (#10745) to porting notes claiming `was simp`.
riccardobrasca pushed a commit that referenced this issue Mar 1, 2024
Classifies by adding issue number (#10745) to porting note claiming anything semantically equivalent to `was simp`. 

Related merged PR: #10746.
dagurtomas pushed a commit that referenced this issue Mar 22, 2024
Classifies by adding issue number (#10745) to porting notes claiming `was simp`.
dagurtomas pushed a commit that referenced this issue Mar 22, 2024
Classifies by adding issue number (#10745) to porting note claiming anything semantically equivalent to `was simp`. 

Related merged PR: #10746.
@grunweg
Copy link
Collaborator

grunweg commented Apr 14, 2024

Some of these are resolved in #12128.

Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment
Labels
porting-notes Mathlib3 to Mathlib4 porting notes.
Projects
None yet
Development

No branches or pull requests

2 participants