Skip to content

Commit 9499961

Browse files
authored
Merge pull request #1045 from MetaCoq/coq-8.17-warnings
Fix remaining warnings, minor fixups
2 parents 1468636 + 9332f05 commit 9499961

File tree

10 files changed

+13
-16
lines changed

10 files changed

+13
-16
lines changed

common/theories/EnvironmentTyping.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -1012,12 +1012,12 @@ Module EnvTyping (T : Term) (E : EnvironmentSig T) (TU : TermUtils T E).
10121012

10131013
Notation lift_sorting_size csize ssize := (lift_sorting_size_gen csize ssize 1).
10141014
Notation typing_sort_size typing_size := (fun t s (tu: typing_sort _ t s) => typing_size t (tSort s) tu).
1015-
Notation lift_typing_size typing_size := (lift_sorting_size_gen typing_size (typing_sort_size typing_size) 0).
1015+
Notation lift_typing_size typing_size := (lift_sorting_size_gen typing_size%function (typing_sort_size typing_size%function) 0).
10161016
Notation typing_sort_size1 typing_size := (fun Γ t s (tu: typing_sort1 _ Γ t s) => typing_size Γ t (tSort s) tu).
10171017
Notation on_def_type_sorting_size ssize := (on_def_type_size_gen ssize 1).
10181018
Notation on_def_type_size typing_size := (on_def_type_size_gen (typing_sort_size1 typing_size) 0).
10191019
Notation on_def_body_sorting_size csize ssize := (on_def_body_size_gen csize ssize 1).
1020-
Notation on_def_body_size typing_size := (on_def_body_size_gen typing_size (typing_sort_size1 typing_size) 0).
1020+
Notation on_def_body_size typing_size := (on_def_body_size_gen typing_size%function (typing_sort_size1 typing_size%function) 0).
10211021
(* Will probably not pass the guard checker if in a list, must be unrolled like in on_def_* *)
10221022

10231023
Lemma lift_sorting_size_impl {checking sorting Qc Qs j} csize ssize :

erasure/theories/EEtaExpandedFix.v

+1
Original file line numberDiff line numberDiff line change
@@ -176,6 +176,7 @@ Inductive expanded_global_declarations : forall (Σ : global_declarations), Prop
176176
| expanded_global_nil : expanded_global_declarations []
177177
| expanded_global_cons decl Σ : expanded_global_declarations Σ ->
178178
expanded_decl Σ decl.2 -> expanded_global_declarations (decl :: Σ).
179+
Derive Signature for expanded_global_declarations.
179180

180181
Definition expanded_global_env := expanded_global_declarations.
181182

erasure/theories/Typed/OptimizeCorrectness.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -19,6 +19,7 @@ From MetaCoq.Utils Require Import MCList.
1919
From MetaCoq.Utils Require Import MCPrelude.
2020
From MetaCoq.Utils Require Import utils.
2121
From MetaCoq.Utils Require Import All_Forall.
22+
Require ssreflect.
2223

2324
Import ExAst.
2425
Import Kernames.
@@ -2639,8 +2640,7 @@ Proof.
26392640
eapply IHl in hn; tea. now rewrite Nat.add_succ_r in hn.
26402641
Qed.
26412642

2642-
2643-
Require Import ssreflect.
2643+
Import ssreflect.
26442644

26452645
Lemma forallbi_Alli {A} (f : nat -> A -> bool) n l :
26462646
Alli f n l <~> forallbi f n l.

pcuic/theories/PCUICEtaExpand.v

+2
Original file line numberDiff line numberDiff line change
@@ -705,6 +705,8 @@ Module Red1Apps.
705705

706706
where " Σ ;;; Γ |- t ⇝ u " := (red1 Σ Γ t u).
707707

708+
Derive Signature for red1.
709+
708710
Lemma red1_ind_all :
709711
forall (Σ : global_env) (P : context -> term -> term -> Type),
710712

pcuic/theories/PCUICNormal.v

-5
Original file line numberDiff line numberDiff line change
@@ -317,8 +317,6 @@ Proof.
317317
- inv whn; solve_discr; easy.
318318
Qed.
319319

320-
Set Firstorder Solver auto with core.
321-
322320
Definition whnf_whne_dec flags Σ Γ t :
323321
({∥whnf flags Σ Γ t∥} + {~∥whnf flags Σ Γ t∥}) *
324322
({∥whne flags Σ Γ t∥} + {~∥whne flags Σ Γ t∥}).
@@ -1936,6 +1934,3 @@ Section Normal.
19361934
Qed.
19371935

19381936
End Normal.
1939-
1940-
1941-

pcuic/theories/PCUICReduction.v

+2
Original file line numberDiff line numberDiff line change
@@ -153,6 +153,8 @@ Inductive red1 (Σ : global_env) (Γ : context) : term -> term -> Type :=
153153

154154
where " Σ ;;; Γ |- t ⇝ u " := (red1 Σ Γ t u).
155155

156+
Derive Signature for red1.
157+
156158
Definition red1_ctx Σ := (OnOne2_local_env (fun Δ => on_one_decl (fun t t' => red1 Σ Δ t t'))).
157159
Definition red1_ctx_rel Σ Γ := (OnOne2_local_env (fun Δ => on_one_decl (fun t t' => red1 Σ (Γ ,,, Δ) t t'))).
158160

safechecker/demo.v safechecker-plugin/demo.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
(* Distributed under the terms of the MIT license. *)
2-
Require Import MetaCoq.SafeChecker.Loader.
2+
Require Import MetaCoq.SafeCheckerPlugin.Loader.
33

44
MetaCoq SafeCheck (3 + 9).
55

safechecker/theories/Loader.v

-4
This file was deleted.

safechecker/theories/PCUICSafeConversion.v

+1-2
Original file line numberDiff line numberDiff line change
@@ -6045,8 +6045,6 @@ Qed.
60456045
_isconv Fallback Γ t1 π1 h1 t2 π2 h2 aux :=
60466046
λ { | leq | hx | r1 | r2 | hd := _isconv_fallback Γ leq t1 π1 h1 t2 π2 h2 r1 r2 hd hx aux }.
60476047

6048-
Derive Signature for dlexmod.
6049-
60506048
Lemma welltyped_R_zipc Σ (wfΣ : abstract_env_ext_rel X Σ) Γ :
60516049
forall x y : pack Γ, welltyped Σ Γ (zipc (tm1 x) (stk1 x)) -> R Γ y x -> welltyped Σ Γ (zipc (tm1 y) (stk1 y)).
60526050
Proof using Type.
@@ -6055,6 +6053,7 @@ Qed.
60556053
pose proof (hΣ := hΣ _ wfΣ). cbn.
60566054
sq.
60576055
destruct x, y; cbn in *.
6056+
red in HR. cbn in HR. red in HR. cbn in HR.
60586057
depind HR.
60596058
- cbn in *. specialize_Σ wfΣ.
60606059
eapply cored'_postpone in H as [u' [cor eq]].

utils/theories/wGraph.v

+2
Original file line numberDiff line numberDiff line change
@@ -6,6 +6,8 @@ From Equations Require Import Equations.
66

77
Local Open Scope Z_scope.
88

9+
Ltac Tauto.intuition_solver ::= auto with *.
10+
911
Lemma fold_max_In n m l (H : fold_left Z.max l n = m)
1012
: n = m \/ In m l.
1113
Proof.

0 commit comments

Comments
 (0)