Skip to content

Commit 7b8b39c

Browse files
Merge pull request #192 from rmatthes/beautifyisos
repair work to accommodate PR #1359 for UniMath
2 parents f3540fd + 0ea906f commit 7b8b39c

File tree

4 files changed

+8
-8
lines changed

4 files changed

+8
-8
lines changed

TypeTheory/ALV1/RelativeUniverses.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -862,7 +862,7 @@ Proof.
862862
rewrite functor_comp.
863863
repeat rewrite assoc. apply maponpaths_2.
864864
apply pathsinv0. rewrite <- assoc. rewrite <- assoc.
865-
apply (iso_inv_to_left D' _ _ _ (αpwiso Xf )).
865+
apply (iso_inv_to_left (C:=D') _ _ _ (αpwiso Xf )).
866866
cbn. unfold precomp_with. rewrite id_right.
867867
assert (XR := nat_trans_ax α').
868868
apply pathsinv0.

TypeTheory/Auxiliary/Auxiliary.v

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -1129,7 +1129,7 @@ Lemma commuting_square_transfer_iso {C : precategory}
11291129
-> p1' ;; f' = p2' ;; g'.
11301130
Proof.
11311131
intro H.
1132-
refine (pre_comp_with_iso_is_inj _ _ _ _ i_d _ _ _ _).
1132+
refine (pre_comp_with_iso_is_inj _ _ _ i_d _ _ _ _).
11331133
exact (pr2 i_d). (* TODO: access function [is_iso_from_iso]? *)
11341134
rewrite 2 assoc.
11351135
rewrite <- i_p1, <- i_p2.
@@ -1163,7 +1163,7 @@ Proof.
11631163
+ exact (h ;; iso_inv_from_iso i_b).
11641164
+ exact (k ;; iso_inv_from_iso i_c).
11651165
+ abstract (
1166-
apply (post_comp_with_iso_is_inj _ _ _ i_a (pr2 _));
1166+
apply (post_comp_with_iso_is_inj _ _ i_a (pr2 _));
11671167
(* TODO: access function for isos! *)
11681168
repeat rewrite <- assoc;
11691169
rewrite i_f, i_g;
@@ -1193,17 +1193,17 @@ Proof.
11931193
apply subtypePath.
11941194
intro; apply isapropdirprod; apply homset_property.
11951195
cbn.
1196-
apply (post_comp_with_iso_is_inj _ _ _ (iso_inv_from_iso i_d) (pr2 _)).
1196+
apply (post_comp_with_iso_is_inj _ _ (iso_inv_from_iso i_d) (pr2 _)).
11971197
eapply @pathscomp0.
11981198
2: { rewrite <- assoc. cbn. rewrite iso_inv_after_iso. eapply pathsinv0, id_right. }
11991199
apply PullbackArrowUnique; cbn.
1200-
+ apply (post_comp_with_iso_is_inj _ _ _ i_b (pr2 _)).
1200+
+ apply (post_comp_with_iso_is_inj _ _ i_b (pr2 _)).
12011201
repeat rewrite <- assoc.
12021202
rewrite i_p1, iso_after_iso_inv, id_right.
12031203
eapply @pathscomp0.
12041204
apply maponpaths. rewrite assoc, iso_after_iso_inv. apply id_left.
12051205
apply (pr1 (pr2 hk')).
1206-
+ apply (post_comp_with_iso_is_inj _ _ _ i_c (pr2 _)).
1206+
+ apply (post_comp_with_iso_is_inj _ _ i_c (pr2 _)).
12071207
repeat rewrite <- assoc.
12081208
rewrite i_p2, iso_after_iso_inv, id_right.
12091209
eapply @pathscomp0.

TypeTheory/Csystems/lCsystems.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -539,7 +539,7 @@ Proof.
539539
assert (e: f_star gt0 (ftf g2) = f_star (C0ax5a gt0 f) g1)
540540
by exact (! maponpaths (f_star gt0) pbeq @ ! C0ax7a gt0 f g1).
541541
apply (eq_par_arrow_cor_objirr (isaset_ob CC) _ _ (pnX 1) e).
542-
- apply (pre_comp_with_iso_is_inj _ _ _ _ (C0eiso gt0 (ftf g2))).
542+
- apply (pre_comp_with_iso_is_inj _ _ _ (C0eiso gt0 (ftf g2))).
543543
{ apply iso_is_iso. }
544544
apply pathsinv0.
545545
etrans.

TypeTheory/OtherDefs/TypeCat_to_CwF_Pitts.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -353,7 +353,7 @@ Proof.
353353
= (q_typecat (reind_typecat A (dpr_typecat A)) (a;; q_typecat A γ))
354354
;; (q_typecat A (dpr_typecat A))).
355355

356-
unshelve refine (pre_comp_with_iso_is_inj _ _ _ _ _ _ _ _ _).
356+
unshelve refine (pre_comp_with_iso_is_inj _ _ _ _ _ _ _ _).
357357
Focus 4.
358358
etrans. Focus 2. symmetry; apply assoc.
359359
etrans. Focus 2. apply (@q_q_typecat (((CC,,homs_sets),,pr1 C),,pr2 C)).

0 commit comments

Comments
 (0)