diff options
| author | Jan-Oliver Kaiser | 2020-05-14 17:08:20 +0200 |
|---|---|---|
| committer | Pierre Roux | 2021-04-22 09:16:22 +0200 |
| commit | 2cbc36c6ae4ca22e000dbb045c865f54a454aca3 (patch) | |
| tree | 28cfb03cc4af70bcd86f7058571aa5a44da270b0 /test-suite/output/Warnings.v | |
| parent | 3442bfa0e7c7e5ba3ce7d62f16d221c2e6da03cf (diff) | |
Enable canonical `fun _ => _` projections.
Diffstat (limited to 'test-suite/output/Warnings.v')
| -rw-r--r-- | test-suite/output/Warnings.v | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/output/Warnings.v b/test-suite/output/Warnings.v index 7465442cab..ce92bcbbb2 100644 --- a/test-suite/output/Warnings.v +++ b/test-suite/output/Warnings.v @@ -1,5 +1,5 @@ (* Term in warning was not printed in the right environment at some time *) -Record A := { B:Type; b:B->B }. -Definition a B := {| B:=B; b:=fun x => x |}. +Record A := { B:Type; b:Prop }. +Definition a B := {| B:=B; b:=forall x, x > 0 |}. Canonical Structure a. |
