Skip to content

Commit

Permalink
coe_fn_coe_base doesn't need to be removed from the simp set anymore
Browse files Browse the repository at this point in the history
  • Loading branch information
Vierkantor committed Mar 5, 2021
1 parent a4d5add commit 36ce6ed
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 6 deletions.
8 changes: 3 additions & 5 deletions src/analysis/calculus/iterated_deriv.lean
Expand Up @@ -135,7 +135,7 @@ lemma times_cont_diff_on_of_differentiable_on_deriv {n : with_top ℕ}
begin
apply times_cont_diff_on_of_differentiable_on,
simpa [iterated_fderiv_within_eq_equiv_comp,
continuous_linear_equiv.comp_differentiable_on_iff, -coe_fn_coe_base],
continuous_linear_equiv.comp_differentiable_on_iff],
end

/-- On a set with unique derivatives, a `C^n` function has derivatives up to `n` which are
Expand All @@ -144,8 +144,7 @@ lemma times_cont_diff_on.continuous_on_iterated_deriv_within {n : with_top ℕ}
(h : times_cont_diff_on 𝕜 n f s) (hmn : (m : with_top ℕ) ≤ n) (hs : unique_diff_on 𝕜 s) :
continuous_on (iterated_deriv_within m f s) s :=
begin
simp [iterated_deriv_within_eq_equiv_comp, continuous_linear_equiv.comp_continuous_on_iff,
-coe_fn_coe_base],
simp [iterated_deriv_within_eq_equiv_comp, continuous_linear_equiv.comp_continuous_on_iff],
exact h.continuous_on_iterated_fderiv_within hmn hs
end

Expand All @@ -155,8 +154,7 @@ lemma times_cont_diff_on.differentiable_on_iterated_deriv_within {n : with_top
(h : times_cont_diff_on 𝕜 n f s) (hmn : (m : with_top ℕ) < n) (hs : unique_diff_on 𝕜 s) :
differentiable_on 𝕜 (iterated_deriv_within m f s) s :=
begin
simp [iterated_deriv_within_eq_equiv_comp, continuous_linear_equiv.comp_differentiable_on_iff,
-coe_fn_coe_base],
simp [iterated_deriv_within_eq_equiv_comp, continuous_linear_equiv.comp_differentiable_on_iff],
exact h.differentiable_on_iterated_fderiv_within hmn hs
end

Expand Down
2 changes: 1 addition & 1 deletion src/set_theory/cofinality.lean
Expand Up @@ -78,7 +78,7 @@ begin
refine le_trans (min_le _ _) _,
{ exact ⟨f ⁻¹' S, λ a,
let ⟨b, bS, h⟩ := H (f a) in ⟨f.symm b, by simp [bS, ← f.map_rel_iff, h,
-coe_fn_coe_base, -coe_fn_coe_trans, principal_seg.coe_coe_fn', initial_seg.coe_coe_fn]⟩⟩ },
-coe_fn_coe_trans, principal_seg.coe_coe_fn', initial_seg.coe_coe_fn]⟩⟩ },
{ exact lift_mk_le.{u v (max u v)}.2
⟨⟨λ ⟨x, h⟩, ⟨f x, h⟩, λ ⟨x, h₁⟩ ⟨y, h₂⟩ h₃,
by congr; injection h₃ with h'; exact f.to_equiv.injective h'⟩⟩ }
Expand Down

0 comments on commit 36ce6ed

Please sign in to comment.