Skip to content

Commit 8afa771

Browse files
committed
Make all of All_Forall universe polymorphic
Turns out All isn't enough.
1 parent f820715 commit 8afa771

File tree

1 file changed

+5
-2
lines changed

1 file changed

+5
-2
lines changed

utils/theories/All_Forall.v

Lines changed: 5 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -3,12 +3,16 @@ From MetaCoq.Utils Require Import MCPrelude MCReflect MCList MCRelations MCProd
33
From Equations Require Import Equations.
44
Import ListNotations.
55

6+
Local Set Universe Polymorphism.
7+
Local Set Polymorphic Inductive Cumulativity.
8+
Local Unset Universe Minimization ToSet.
9+
610
Derive Signature for Forall Forall2.
711

812
(** Combinators *)
913

1014
(** 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 :=
1216
All_nil : All P []
1317
| All_cons : forall (x : A) (l : list A),
1418
P x -> All P l -> All P (x :: l).
@@ -3563,7 +3567,6 @@ Proof.
35633567
all: now apply In_All; constructor => //.
35643568
Qed.
35653569

3566-
Local Set Universe Polymorphism.
35673570
Lemma All_eta3 {A B C P} ls
35683571
: @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.
35693572
Proof.

0 commit comments

Comments
 (0)