File tree Expand file tree Collapse file tree 3 files changed +6
-7
lines changed
Expand file tree Collapse file tree 3 files changed +6
-7
lines changed Original file line number Diff line number Diff line change @@ -676,7 +676,7 @@ Proof.
676676 apply idpath.
677677Qed .
678678
679- Definition dpr_q_pbpairing_cwf_unique (hs : has_homsets CC)
679+ Definition dpr_q_pbpairing_cwf_unique
680680 {Γ} (A : C⟨Γ⟩)
681681 {Γ'} (f : Γ' --> Γ)
682682 {X} (h : X --> Γ ∙ A) (k : X --> Γ') (H : h ;; π A = k ;; f)
@@ -687,10 +687,10 @@ Proof.
687687 destruct t as [hk [e2 e1]].
688688 refine (@total2_paths_f _ _ (tpair _ hk (tpair _ e2 e1)) _
689689 (dpr_q_pbpairing_cwf_mapunique A f H hk e2 e1) _).
690- unshelve refine (total2_paths_f _ _); apply hs .
690+ unshelve refine (total2_paths_f _ _); apply homset_property .
691691Qed .
692692
693- Lemma is_pullback_reindx_cwf (hs : has_homsets CC) : ∏ (Γ : CC) (A : C⟨Γ⟩) (Γ' : CC)
693+ Lemma is_pullback_reindx_cwf : ∏ (Γ : CC) (A : C⟨Γ⟩) (Γ' : CC)
694694 (f : Γ' --> Γ),
695695 isPullback (dpr_q_cwf A f).
696696Proof .
@@ -699,7 +699,6 @@ Proof.
699699 intros e h k H.
700700 exists (dpr_q_pbpairing_cwf _ _ h k H).
701701 apply dpr_q_pbpairing_cwf_unique.
702- assumption.
703702Defined .
704703
705704End CwF_lemmas.
Original file line number Diff line number Diff line change @@ -97,10 +97,10 @@ Proof.
9797 + simpl. unfold dm_sub_struct_of_CwF.
9898 simpl.
9999 refine (pr1 (postcomp_pb_with_iso CC _ _ _ _ (q_cwf A f) _ _ f _
100- (is_pullback_reindx_cwf (homset_property _) _ _ _ _ ) _ _ _ _)).
100+ (is_pullback_reindx_cwf _ _ _ _ ) _ _ _ _)).
101101 sym. assumption.
102102 + eapply (pr2 ( postcomp_pb_with_iso CC _ _ _ _ (q_cwf A f) _ _ f _
103- (is_pullback_reindx_cwf (homset_property _) _ _ _ _ ) _ _ _ _ )).
103+ (is_pullback_reindx_cwf _ _ _ _ ) _ _ _ _ )).
104104 - simpl.
105105 apply hinhpr.
106106 unfold iso_to_dpr.
Original file line number Diff line number Diff line change 8484 exists (@q_cwf CC C).
8585 exists (@dpr_q_cwf CC C).
8686 intros; apply @is_symmetric_isPullback. { apply homs_sets. }
87- apply is_pullback_reindx_cwf. apply homs_sets.
87+ apply is_pullback_reindx_cwf.
8888Defined .
8989
9090(** * Splitness of the constructed TypeCat *)
You can’t perform that action at this time.
0 commit comments