Skip to content

Commit

Permalink
Wrap lines
Browse files Browse the repository at this point in the history
  • Loading branch information
Vierkantor committed Jan 17, 2024
1 parent 680197f commit 4145626
Show file tree
Hide file tree
Showing 7 changed files with 18 additions and 10 deletions.
4 changes: 3 additions & 1 deletion Mathlib/Analysis/Normed/Group/Hom.lean
Original file line number Diff line number Diff line change
Expand Up @@ -92,7 +92,9 @@ instance toAddMonoidHomClass : AddMonoidHomClass (NormedAddGroupHom V₁ V₂) V
map_add f := f.map_add'
map_zero f := (AddMonoidHom.mk' f.toFun f.map_add').map_zero

/-- Helper instance for when there are too many metavariables to apply `DFunLike.coeFun` directly. -/
/--
Helper instance for when there are too many metavariables to apply `DFunLike.coeFun` directly.
-/
instance coeFun : CoeFun (NormedAddGroupHom V₁ V₂) fun _ => V₁ → V₂ :=
⟨DFunLike.coe⟩

Expand Down
3 changes: 2 additions & 1 deletion Mathlib/LinearAlgebra/FinsuppVectorSpace.lean
Original file line number Diff line number Diff line change
Expand Up @@ -79,7 +79,8 @@ protected def basis {φ : ι → Type*} (b : ∀ i, Basis (φ i) R M) : Basis (
(b i).repr.symm (g.comapDomain _ (Set.injOn_of_injective sigma_mk_injective _))
support := g.support.image Sigma.fst
mem_support_toFun := fun i => by
rw [Ne.def, ← (b i).repr.injective.eq_iff, (b i).repr.apply_symm_apply, DFunLike.ext_iff]
rw [Ne.def, ← (b i).repr.injective.eq_iff, (b i).repr.apply_symm_apply,
DFunLike.ext_iff]
simp only [exists_prop, LinearEquiv.map_zero, comapDomain_apply, zero_apply,
exists_and_right, mem_support_iff, exists_eq_right, Sigma.exists, Finset.mem_image,
not_forall] }
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/RingTheory/Ideal/QuotientOperations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -600,7 +600,8 @@ def quotientEquivAlg (I : Ideal A) (J : Ideal B) (f : A ≃ₐ[R₁] B) (hIJ : J
{ quotientEquiv I J (f : A ≃+* B) hIJ with
commutes' := fun r => by
-- Porting note: Needed to add the below lemma because Equivs coerce weird
have : ∀ (e : RingEquiv (A ⧸ I) (B ⧸ J)), Equiv.toFun e.toEquiv = DFunLike.coe e := fun _ ↦ rfl
have : ∀ (e : RingEquiv (A ⧸ I) (B ⧸ J)), Equiv.toFun e.toEquiv = DFunLike.coe e :=
fun _ ↦ rfl
rw [this]
simp only [quotientEquiv_apply, RingHom.toFun_eq_coe, quotientMap_algebraMap,
RingEquiv.coe_toRingHom, AlgEquiv.coe_ringEquiv, AlgEquiv.commutes, Quotient.mk_algebraMap]}
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Topology/Algebra/Module/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -710,7 +710,8 @@ theorem one_apply (x : M₁) : (1 : M₁ →L[R₁] M₁) x = x :=
#align continuous_linear_map.one_apply ContinuousLinearMap.one_apply

instance [Nontrivial M₁] : Nontrivial (M₁ →L[R₁] M₁) :=
0, 1, fun e ↦ have ⟨x, hx⟩ := exists_ne (0 : M₁); hx (by simpa using DFunLike.congr_fun e.symm x)⟩
0, 1, fun e ↦
have ⟨x, hx⟩ := exists_ne (0 : M₁); hx (by simpa using DFunLike.congr_fun e.symm x)⟩

section Add

Expand Down
5 changes: 3 additions & 2 deletions Mathlib/Topology/Category/CompHaus/EffectiveEpi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -54,8 +54,9 @@ def struct {B X : CompHaus.{u}} (π : X ⟶ B) (hπ : Function.Surjective π) :
(by ext; exact hab)) a)
uniq e h g hm := by
suffices g = (QuotientMap.of_surjective_continuous hπ π.continuous).liftEquiv ⟨e,
fun a b hab ↦ DFunLike.congr_fun (h ⟨fun _ ↦ a, continuous_const⟩ ⟨fun _ ↦ b, continuous_const⟩
(by ext; exact hab)) a⟩ by assumption
fun a b hab ↦ DFunLike.congr_fun
(h ⟨fun _ ↦ a, continuous_const⟩ ⟨fun _ ↦ b, continuous_const⟩ (by ext; exact hab))
a⟩ by assumption
rw [← Equiv.symm_apply_eq (QuotientMap.of_surjective_continuous hπ π.continuous).liftEquiv]
ext
simp only [QuotientMap.liftEquiv_symm_apply_coe, ContinuousMap.comp_apply, ← hm]
Expand Down
5 changes: 3 additions & 2 deletions Mathlib/Topology/Category/Profinite/EffectiveEpi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -52,8 +52,9 @@ def struct {B X : Profinite.{u}} (π : X ⟶ B) (hπ : Function.Surjective π) :
(by ext; exact hab)) a)
uniq e h g hm := by
suffices g = (QuotientMap.of_surjective_continuous hπ π.continuous).liftEquiv ⟨e,
fun a b hab ↦ DFunLike.congr_fun (h ⟨fun _ ↦ a, continuous_const⟩ ⟨fun _ ↦ b, continuous_const⟩
(by ext; exact hab)) a⟩ by assumption
fun a b hab ↦ DFunLike.congr_fun
(h ⟨fun _ ↦ a, continuous_const⟩ ⟨fun _ ↦ b, continuous_const⟩ (by ext; exact hab))
a⟩ by assumption
rw [← Equiv.symm_apply_eq (QuotientMap.of_surjective_continuous hπ π.continuous).liftEquiv]
ext
simp only [QuotientMap.liftEquiv_symm_apply_coe, ContinuousMap.comp_apply, ← hm]
Expand Down
5 changes: 3 additions & 2 deletions Mathlib/Topology/Category/Stonean/EffectiveEpi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -51,8 +51,9 @@ def struct {B X : Stonean.{u}} (π : X ⟶ B) (hπ : Function.Surjective π) : E
(by ext; exact hab)) a)
uniq e h g hm := by
suffices g = (QuotientMap.of_surjective_continuous hπ π.continuous).liftEquiv ⟨e,
fun a b hab ↦ DFunLike.congr_fun (h ⟨fun _ ↦ a, continuous_const⟩ ⟨fun _ ↦ b, continuous_const⟩
(by ext; exact hab)) a⟩ by assumption
fun a b hab ↦ DFunLike.congr_fun
(h ⟨fun _ ↦ a, continuous_const⟩ ⟨fun _ ↦ b, continuous_const⟩ (by ext; exact hab))
a⟩ by assumption
rw [← Equiv.symm_apply_eq (QuotientMap.of_surjective_continuous hπ π.continuous).liftEquiv]
ext
simp only [QuotientMap.liftEquiv_symm_apply_coe, ContinuousMap.comp_apply, ← hm]
Expand Down

0 comments on commit 4145626

Please sign in to comment.