diff options
Diffstat (limited to 'test-suite/output')
-rw-r--r-- | test-suite/output/UnivBinders.out | 12 | ||||
-rw-r--r-- | test-suite/output/UnivBinders.v | 3 | ||||
-rw-r--r-- | test-suite/output/inference.out | 2 | ||||
-rw-r--r-- | test-suite/output/inference.v | 6 |
4 files changed, 9 insertions, 14 deletions
diff --git a/test-suite/output/UnivBinders.out b/test-suite/output/UnivBinders.out index 668b4e578..6f41b2fcf 100644 --- a/test-suite/output/UnivBinders.out +++ b/test-suite/output/UnivBinders.out @@ -149,24 +149,24 @@ inmod@{u} -> Type@{v} (* u v |= *) Applied.infunct is universe polymorphic -axfoo@{i Top.41 Top.42} : Type@{Top.41} -> Type@{i} -(* i Top.41 Top.42 |= *) +axfoo@{i Top.44 Top.45} : Type@{Top.44} -> Type@{i} +(* i Top.44 Top.45 |= *) axfoo is universe polymorphic Argument scope is [type_scope] Expands to: Constant Top.axfoo -axbar@{i Top.41 Top.42} : Type@{Top.42} -> Type@{i} -(* i Top.41 Top.42 |= *) +axbar@{i Top.44 Top.45} : Type@{Top.45} -> Type@{i} +(* i Top.44 Top.45 |= *) axbar is universe polymorphic Argument scope is [type_scope] Expands to: Constant Top.axbar -axfoo' : Type@{Top.44} -> Type@{axbar'.i} +axfoo' : Type@{Top.47} -> Type@{axbar'.i} axfoo' is not universe polymorphic Argument scope is [type_scope] Expands to: Constant Top.axfoo' -axbar' : Type@{Top.44} -> Type@{axbar'.i} +axbar' : Type@{Top.47} -> Type@{axbar'.i} axbar' is not universe polymorphic Argument scope is [type_scope] diff --git a/test-suite/output/UnivBinders.v b/test-suite/output/UnivBinders.v index 266d94ad9..c6efc240a 100644 --- a/test-suite/output/UnivBinders.v +++ b/test-suite/output/UnivBinders.v @@ -44,6 +44,9 @@ Module mono. Monomorphic Definition monomono := Type@{MONOU}. Check monomono. + + Monomorphic Inductive monoind@{i} : Type@{i} := . + Monomorphic Record monorecord@{i} : Type@{i} := mkmonorecord {}. End mono. Check mono.monomono. (* qualified MONOU *) Import mono. diff --git a/test-suite/output/inference.out b/test-suite/output/inference.out index 5e9eff048..f7ffd1959 100644 --- a/test-suite/output/inference.out +++ b/test-suite/output/inference.out @@ -4,8 +4,6 @@ fun e : option L => match e with | None => None end : option L -> option L -fun (m n p : nat) (H : S m <= S n + p) => le_S_n m (n + p) H - : forall m n p : nat, S m <= S n + p -> m <= n + p fun n : nat => let y : T n := A n in ?t ?x : T n : forall n : nat, T n where diff --git a/test-suite/output/inference.v b/test-suite/output/inference.v index 73169dae6..57a4739e9 100644 --- a/test-suite/output/inference.v +++ b/test-suite/output/inference.v @@ -13,12 +13,6 @@ Definition P (e:option L) := Print P. -(* Check that plus is folded even if reduction is involved *) -Set Warnings Append "-deprecated-option". -Set Refolding Reduction. -Check (fun m n p (H : S m <= (S n) + p) => le_S_n _ _ H). - - (* Check that the heuristic to solve constraints is not artificially dependent on the presence of a let-in, and in particular that the second [_] below is not inferred to be n, as if obtained by |