Skip to content

Commit 2479a7f

Browse files
Merge pull request #238 from Skantz/initlogic
#235: Remove dependency on Coq.Init.Logic
2 parents b2aa8ef + 6b975be commit 2479a7f

File tree

3 files changed

+7
-20
lines changed

3 files changed

+7
-20
lines changed

TypeTheory/CwF_TypeCat/CwF_SplitTypeCat_Equiv_Cats.v

+1
Original file line numberDiff line numberDiff line change
@@ -16,6 +16,7 @@ Require Import UniMath.CategoryTheory.DisplayedCats.Isos.
1616
Require Import UniMath.CategoryTheory.DisplayedCats.Fiber.
1717
Require Import UniMath.CategoryTheory.DisplayedCats.Constructions.
1818
Require Import UniMath.CategoryTheory.DisplayedCats.Equivalences.
19+
Require Import UniMath.CategoryTheory.DisplayedCats.Examples.Sigma.
1920

2021
Require Import TypeTheory.Auxiliary.Auxiliary.
2122
Require Import TypeTheory.Auxiliary.CategoryTheory.

TypeTheory/Initiality/Interpretation.v

+4-12
Original file line numberDiff line numberDiff line change
@@ -1,14 +1,6 @@
11
(** This file defines the interpretation function, from the syntax of our toy type theory into any split type-cat with suitable structure. *)
22

33

4-
(** * TODO NOTE: This file depends on Coq.Init.Logic.
5-
Removing the following line causes the error:
6-
7-
File "./TypeTheory/TypeTheory/Initiality/Interpretation.v", line 366, characters 4-5:
8-
Error: [Focus] Wrong bullet -: Current bullet + is not finished.
9-
*)
10-
Require Import Coq.Init.Logic.
11-
124
Require Import UniMath.MoreFoundations.All.
135
Require Import UniMath.CategoryTheory.Core.Prelude.
146

@@ -362,7 +354,7 @@ Section Partial_Interpretation.
362354
apply funextfun; intros i. apply maponpaths_2.
363355
eapply pathscomp0. 2: { apply partial_interpretation_rename_ty. }
364356
apply maponpaths_2, funextfun.
365-
refine (dB_Sn_rect _ _ _); auto.
357+
refine (dB_Sn_rect _ _ _); reflexivity.
366358
- (* term expressions *)
367359
destruct e as [ m i | m A B b | m A B t a ].
368360
+ (* [var_expr i] *)
@@ -373,7 +365,7 @@ Section Partial_Interpretation.
373365
apply funextfun; intros A_interp.
374366
assert (e_EA : (extend_environment (E ∘ f) A_interp
375367
= extend_environment E A_interp ∘ fmap_dB_S f)).
376-
{ apply funextfun. refine (dB_Sn_rect _ _ _); auto. }
368+
{ apply funextfun. refine (dB_Sn_rect _ _ _); reflexivity. }
377369
apply maponpaths_12.
378370
{ eapply pathscomp0. 2: { apply partial_interpretation_rename_ty. }
379371
apply maponpaths_2, e_EA. }
@@ -386,7 +378,7 @@ Section Partial_Interpretation.
386378
apply funextfun; intros A_interp.
387379
assert (e_EA : (extend_environment (E ∘ f) A_interp
388380
= extend_environment E A_interp ∘ fmap_dB_S f)).
389-
{ apply funextfun. refine (dB_Sn_rect _ _ _); auto. }
381+
{ apply funextfun. refine (dB_Sn_rect _ _ _); reflexivity. }
390382
apply maponpaths_12.
391383
{ eapply pathscomp0. 2: { apply partial_interpretation_rename_ty. }
392384
apply maponpaths_2, e_EA. }
@@ -514,7 +506,7 @@ a little more work to state. *)
514506
apply make_leq_partial'; cbn; intros [f_def b_def].
515507
use tpair.
516508
- refine (dB_Sn_rect _ _ _); assumption.
517-
- apply funextfun. refine (dB_Sn_rect _ _ _); auto.
509+
- apply funextfun. refine (dB_Sn_rect _ _ _); reflexivity.
518510
Defined.
519511

520512
Definition partial_interpretation_tm_as_raw_context_map

TypeTheory/TypeCat/General.v

+2-8
Original file line numberDiff line numberDiff line change
@@ -5,13 +5,6 @@ Note: much of this essentially duplicates material given already in the [CwF_Spl
55
66
Probably much of this really should belong in a different package. *)
77

8-
(** * TODO NOTE: This file depends on Coq.Init.Logic.
9-
Removing the following line causes the error:
10-
11-
File "./TypeTheory/TypeTheory/TypeCat/General.v", line 365, characters 6-115:
12-
Error: not found in table: core.eq.type
13-
*)
14-
Require Import Coq.Init.Logic.
158

169
Require Import UniMath.MoreFoundations.All.
1710
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
@@ -362,7 +355,8 @@ Section Terms.
362355
rewrite !maponpathscomp0, !idtoiso_concat_pr, <-!assoc.
363356
etrans; [ do 2 eapply maponpaths; rewrite assoc;
364357
apply (!q_comp_typecat A (dpr_typecat A) a)|].
365-
now rewrite af, id_left, q_id_typecat,
358+
destruct e, (!af).
359+
now rewrite id_left, q_id_typecat,
366360
<- idtoiso_concat_pr, <-maponpathscomp0, pathsinv0l.
367361
Qed.
368362

0 commit comments

Comments
 (0)