File tree Expand file tree Collapse file tree 1 file changed +5
-2
lines changed Expand file tree Collapse file tree 1 file changed +5
-2
lines changed Original file line number Diff line number Diff line change @@ -3,12 +3,16 @@ From MetaCoq.Utils Require Import MCPrelude MCReflect MCList MCRelations MCProd
3
3
From Equations Require Import Equations.
4
4
Import ListNotations.
5
5
6
+ Local Set Universe Polymorphism.
7
+ Local Set Polymorphic Inductive Cumulativity.
8
+ Local Unset Universe Minimization ToSet.
9
+
6
10
Derive Signature for Forall Forall2.
7
11
8
12
(** Combinators *)
9
13
10
14
(** Forall combinators in Type to allow building them by recursion *)
11
- Polymorphic Cumulative Inductive All {A} (P : A -> Type ) : list A -> Type :=
15
+ Inductive All {A} (P : A -> Type ) : list A -> Type :=
12
16
All_nil : All P []
13
17
| All_cons : forall (x : A) (l : list A),
14
18
P x -> All P l -> All P (x :: l).
@@ -3563,7 +3567,6 @@ Proof.
3563
3567
all: now apply In_All; constructor => //.
3564
3568
Qed .
3565
3569
3566
- Local Set Universe Polymorphism.
3567
3570
Lemma All_eta3 {A B C P} ls
3568
3571
: @All (A * B * C)%type (fun '(a, b, c) => P a b c) ls <~> All (fun abc => P abc.1.1 abc.1.2 abc.2) ls.
3569
3572
Proof .
You can’t perform that action at this time.
0 commit comments