You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Not sure it is very critical, but there seems to be an issue with template polymorphisms ending in Prop:
Inductive K A := C : A -> K A.
Definition L := K True.
From elpi.apps RequireImport derive.std.
Elpi derive.param1 K.
Elpi derive.param1 True.
Fail Elpi derive.param1 L.
(* param1: constant does not have the right type: Unable to unify "K True -> Type" with "L -> Prop"(universe inconsistency: Cannot enforce is_K.u1 <= Prop). *)
Deriving manually however works, so I suspect the generated is_K not to be declared as template polymorphic:
Inductive K A := C : A -> K A.
Definition L := K True.
From elpi.apps RequireImport derive.std.
Unset Uniform InductiveParameters.
Elpi derive.param1 True.
Inductive is_K (A : Type) (PA : A -> Type) : K A -> Type :=
is_C : forall a : A, PA a -> is_K A PA (C A a).
Definition is_L : L -> Prop := is_K True is_True.
The text was updated successfully, but these errors were encountered:
Not sure it is very critical, but there seems to be an issue with template polymorphisms ending in Prop:
Deriving manually however works, so I suspect the generated
is_K
not to be declared as template polymorphic:The text was updated successfully, but these errors were encountered: