Skip to content

Commit

Permalink
chore(Profinite/Extend): golf and remove unnecessary have statements (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
dagurtomas committed Oct 23, 2024
1 parent 3b90821 commit 9248301
Showing 1 changed file with 2 additions and 8 deletions.
10 changes: 2 additions & 8 deletions Mathlib/Topology/Category/Profinite/Extend.lean
Original file line number Diff line number Diff line change
Expand Up @@ -126,12 +126,7 @@ def cone (S : Profinite) :
pt := G.obj S
π := {
app := fun i ↦ G.map i.hom
naturality := fun _ _ f ↦ (by
have := f.w
simp only [const_obj_obj, StructuredArrow.left_eq_id, const_obj_map, Category.id_comp,
StructuredArrow.w] at this
simp only [const_obj_obj, comp_obj, StructuredArrow.proj_obj, const_obj_map, Category.id_comp,
Functor.comp_map, StructuredArrow.proj_map, ← map_comp, StructuredArrow.w]) }
naturality := fun _ _ f ↦ (by simp [← map_comp]) }

example : G.mapCone c = (cone G c.pt).whisker (functor c) := rfl

Expand Down Expand Up @@ -166,8 +161,7 @@ def cocone (S : Profinite) :
have := f.w
simp only [op_obj, const_obj_obj, op_map, CostructuredArrow.right_eq_id, const_obj_map,
Category.comp_id] at this
simp only [comp_obj, CostructuredArrow.proj_obj, op_obj, const_obj_obj, Functor.comp_map,
CostructuredArrow.proj_map, op_map, ← map_comp, this, const_obj_map, Category.comp_id]) }
simp [← map_comp, this]) }

example : G.mapCocone c.op = (cocone G c.pt).whisker (functorOp c) := rfl

Expand Down

0 comments on commit 9248301

Please sign in to comment.