@@ -11,7 +11,7 @@ Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
1111Require Import TypeTheory.Auxiliary.Auxiliary.
1212Require Import TypeTheory.ALV1.TypeCat.
1313
14- (* This should be upstreamed *)
14+ (* TODO: upstream? *)
1515Arguments nat_trans_ax {C C'} {F F'} a {x x'} f.
1616
1717Local Open Scope cat.
@@ -161,7 +161,7 @@ Section Terms.
161161 : reind_tm f a ;; q_typecat A f = f ;; a.
162162 Proof .
163163 simpl.
164- set (pb := make_Pullback _ _ _ _ _ _ _ ).
164+ set (pb := make_Pullback _ _).
165165 now rewrite (PullbackArrow_PullbackPr2 pb).
166166 Qed .
167167
@@ -230,9 +230,9 @@ Section Terms.
230230 = tm_transportb (reind_id_type_typecat _ _) a.
231231 Proof .
232232 apply subtypePath; [ intros x; apply homset_property|]; simpl.
233- set (pb := make_Pullback _ _ _ _ _ _ _ ).
233+ set (pb := make_Pullback _ _).
234234 (* Why is there a ' version of this lemma??? *)
235- apply pathsinv0, (PullbackArrowUnique' _ _ pb).
235+ apply pathsinv0, (PullbackArrowUnique' _ _ _ pb).
236236 - rewrite <-assoc.
237237 etrans; [eapply maponpaths, idtoiso_dpr_typecat|].
238238 exact (pr2 a).
@@ -257,10 +257,10 @@ Section Terms.
257257 (reind_tm g (reind_tm f a)).
258258 Proof .
259259 apply subtypePath; [ intros x; apply homset_property|]; simpl.
260- set (pb := make_Pullback _ _ _ _ _ _ _ ).
261- set (pb' := make_Pullback _ _ _ _ _ _ _ ).
262- set (pb'' := make_Pullback _ _ _ _ _ _ _ ).
263- apply pathsinv0, (PullbackArrowUnique' _ _ pb).
260+ set (pb := make_Pullback _ _).
261+ set (pb' := make_Pullback _ _).
262+ set (pb'' := make_Pullback _ _).
263+ apply pathsinv0, (PullbackArrowUnique' _ _ _ pb).
264264 - rewrite <- assoc.
265265 etrans; [eapply maponpaths, idtoiso_dpr_typecat|].
266266 apply (PullbackArrow_PullbackPr1 pb').
@@ -329,8 +329,8 @@ Section Terms.
329329 apply pathsinv0, PullbackArrowUnique.
330330 { apply (section_property (tm_transportb _ _)). }
331331 apply pathsinv0.
332- etrans. { refine (postCompWithPullbackArrow _ _ _
333- (make_Pullback _ _ _ _ _ _ _ ) _ _ _). }
332+ etrans. { refine (postCompWithPullbackArrow _ _ _ _
333+ (make_Pullback _ _) _ _ _). }
334334 apply pathsinv0, PullbackArrowUnique; cbn; refine (_ @ ! id_right _).
335335 - rewrite <- assoc.
336336 etrans. { apply maponpaths, dpr_q_typecat. }
@@ -378,7 +378,7 @@ Section Terms.
378378 + now induction e; rewrite <-assoc, id_left.
379379 + unfold map_into_Pb.
380380 set (pb := Auxiliary.Pbb _ _ _ _ _ _ _ _ _ _ _).
381- rewrite <-assoc, (postCompWithPullbackArrow _ _ _ pb).
381+ rewrite <-assoc, (postCompWithPullbackArrow _ _ _ _ pb).
382382 apply PullbackArrowUnique; cbn.
383383 - rewrite <-!assoc, dpr_q_typecat; induction e.
384384 now rewrite id_left, assoc, af, id_left, id_right.
@@ -505,4 +505,4 @@ Section Types_with_Terms.
505505 apply tm_transportf_irrelevant.
506506 Qed .
507507
508- End Types_with_Terms.
508+ End Types_with_Terms.
0 commit comments