Skip to content

Commit 407b21a

Browse files
committed
Type Former over SplTCwF done.
1 parent b14923c commit 407b21a

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

TypeTheory/Initiality/SplitTypeCat_General.v

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -165,6 +165,8 @@ Section Terms.
165165
now rewrite (PullbackArrow_PullbackPr2 pb).
166166
Qed.
167167

168+
About q_q_typecat.
169+
168170
(** A concrete construction of “transport” of terms, by composing with [comp_ext_compare]. *)
169171
Definition tm_transportf {C : typecat} {Γ} {A A' : C Γ} (e : A = A')
170172
: tm A ≃ tm A'.
@@ -300,7 +302,8 @@ Section Terms.
300302
+ eapply (map_into_Pb _ _ _ _ _ (reind_pb_typecat A _) _ _ (idpath (identity _ ;; _))).
301303
+ apply Pb_map_commutes_1.
302304
Defined.
303-
305+
About reind_comp_typecat.
306+
About q_q_typecat.
304307
(* TODO: upstream; consider whether this should be primitive instead of [q_q_typecat]. *)
305308
Definition q_q_typecat' {C : split_typecat}
306309
: ∏ Γ (A : C Γ) Γ' (f : Γ' --> Γ) Γ'' (g : Γ'' --> Γ'),

0 commit comments

Comments
 (0)