Skip to content

Commit

Permalink
Fix after merge
Browse files Browse the repository at this point in the history
  • Loading branch information
mattam82 committed Sep 21, 2020
1 parent 4186c44 commit 8d95960
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 7 deletions.
2 changes: 1 addition & 1 deletion pcuic/theories/PCUICInductiveInversion.v
Original file line number Diff line number Diff line change
Expand Up @@ -2643,7 +2643,7 @@ Proof.
exists x; intuition eauto.
now rewrite ConstraintSetFact.add_iff.
firstorder eauto.
subst. exists x0; firstorder.
subst. exists x0; firstorder auto with *.
Qed.

Lemma subst_instance_variance_cstrs l u i i' :
Expand Down
4 changes: 2 additions & 2 deletions pcuic/theories/PCUICSpine.v
Original file line number Diff line number Diff line change
Expand Up @@ -856,11 +856,11 @@ Proof.
rewrite Nat.add_0_r.
specialize (X (subst_context (skipn #|Γ0| s) 0 Γ0) ltac:(now autorewrite with len) _ _
(subst [t1] #|Γ0| T) cs subsl').
rewrite -{1}H0. apply X.
rewrite -{1}H1. apply X.
rewrite -subst_app_simpl'.
apply subslet_length in subsl'.
now autorewrite with len in subsl'.
rewrite -H0. now rewrite firstn_skipn.
rewrite -H1. now rewrite firstn_skipn.
Qed.

Lemma arity_spine_it_mkProd_or_LetIn_Sort {cf:checker_flags} Σ Γ ctx s args inst :
Expand Down
4 changes: 0 additions & 4 deletions safechecker/theories/PCUICSafeChecker.v
Original file line number Diff line number Diff line change
Expand Up @@ -100,14 +100,10 @@ Proof.
now rewrite IHt1.
Qed.

Derive NoConfusion for sort_family.
Derive EqDec for sort_family.

Definition mkApps_decompose_app t :
t = mkApps (fst (decompose_app t)) (snd (decompose_app t))
:= mkApps_decompose_app_rec t [].


Derive NoConfusion EqDec for sort_family.

Inductive type_error :=
Expand Down

0 comments on commit 8d95960

Please sign in to comment.