Skip to content

Commit 55aad58

Browse files
Minor proof simplification
1 parent 50a379c commit 55aad58

File tree

2 files changed

+5
-6
lines changed

2 files changed

+5
-6
lines changed

TypeTheory/Initiality/SplitTypeCat_General.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -497,7 +497,7 @@ Section Types_with_Terms.
497497
+ eapply pathscomp0. { apply pathsinv0, reind_comp_typecat. }
498498
eapply pathscomp0. 2: { apply reind_id_type_typecat. }
499499
apply maponpaths, section_property.
500-
+ use (@maponpaths _ _ (section_pr1 _) (tm_transportf _ _) _ _).
500+
+ use (@maponpaths _ _ _ (tm_transportf _ _) _ _).
501501
refine (_ @ reind_tm_var_typecat' a).
502502
apply tm_transportf_irrelevant.
503503
Qed.

TypeTheory/OtherDefs/CwF_1.v

Lines changed: 4 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -15,9 +15,9 @@
1515
This file is very similar to [TypeTheory.OtherDefs.CwF_Pitts]; the main difference is that here the functor of types is bundled into an actual functor, whereas in [CwF_Pitts], it is split up componentwise.
1616
*)
1717

18+
Require Import UniMath.Foundations.Sets.
1819
Require Import UniMath.CategoryTheory.Core.Functors.
1920
Require Import UniMath.CategoryTheory.opp_precat.
20-
Require Import UniMath.Foundations.Sets.
2121
Require Import UniMath.CategoryTheory.limits.pullbacks.
2222
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
2323
Require Import TypeTheory.Auxiliary.Auxiliary.
@@ -521,7 +521,7 @@ Proof.
521521
apply pathsinv0.
522522
rew_trans_@.
523523
etrans. apply maponpaths, transportf_rtype_mapeq.
524-
rew_trans_@.
524+
rew_trans_@.
525525
(* TODO: try simplyfying with [term_typeeq_transport_lemma] *)
526526
refine (@maponpaths _ _ (fun e => transportf _ e _) _ (idpath _) _).
527527
apply cwf_types_isaset.
@@ -636,7 +636,6 @@ Proof.
636636
apply dpr_q_pbpairing_commutes.
637637
Defined.
638638

639-
640639
Definition dpr_q_pbpairing_cwf_mapunique
641640
{Γ} (A : C⟨Γ⟩)
642641
{Γ'} (f : Γ' --> Γ)
@@ -652,8 +651,8 @@ Proof.
652651
apply (pairing_mapeq _ _ e1 _).
653652
simpl. apply maponpaths.
654653
eapply pathscomp0.
655-
apply maponpaths, maponpaths.
656-
apply (@maponpaths (C ⟨ Γ' ∙ (A[[f]]) ⊢ A[[f]][[π (A[[f]])]] ⟩) _ (fun t => t ⟦hk⟧)).
654+
apply maponpaths, maponpaths.
655+
eapply (maponpaths (fun t => t ⟦hk⟧)).
657656
apply rterm_univ.
658657
eapply pathscomp0.
659658
apply maponpaths, maponpaths.

0 commit comments

Comments
 (0)