-
#### Description of the problem
Hello,
I am quite confused by a case where a generalized rewrite fails. I might naturally be missing something, but I suspect that it is a bug/incomplete feature.…
YaZko updated
3 years ago
-
LH accepts this program:
```haskell
{-@ LIQUID "--higherorder" @-}
{-@ LIQUID "--totality" @-}
{-@ LIQUID "--exactdc" @-}
module Eq where
import Language.Haskell.Liquid.Proof…
-
Hi everyone,
I am opening this issue to collect comments - if any - about ZSA Swaps in order to advance the discussion on the topic and gather feedback from the community on the work done.
As yo…
-
Note: the issue was created automatically with bugzilla2github tool
Original bug ID: BZ#4042
From: @JasonGross
Reported version: 8.5
CC: coq-bugs-redist@lists.gforge.inria.fr
-
```
From mathcomp Require Import all_ssreflect all_algebra.
Import GRing.Theory.
Let test_ssrpat (n : nat) (R : ringType) (f1 f2 g : nat -> R) :
(\big[+%R/0%R]_(i < n) ((f1 i + f2 i) * g i) …
gares updated
4 years ago
-
Note: the issue was created automatically with bugzilla2github tool
Original bug ID: BZ#5301
From: @jhjourdan
Reported version: 8.6
CC: @RalfJung
-
As reported by @skaftetryne on [freemint-discuss](https://sourceforge.net/p/freemint/mailman/freemint-discuss/thread/1706364992.k2t4psfan4g4kksg%40epost.online.no/#msg58729557):
I'm usually running…
-
#### Description of the problem
The snippet below shows that Ltac1 can catch the "No head constant to reduce" exception from `red` but Ltac2 doesn't seem to be able to do the same. The only com…
-
```coq
Parameters F G: Prop.
Axiom F2G: F -> G.
Goal F -> exists n: nat, n * n = 0.
Proof.
intros HF.
eapply ex_ind.
intros x Hx.
unshelve eexists.
```
After this, the first go…
-
The program
```
> module Num
> import Data.Fin
> import Data.Vect
> import Data.VectType
> import Syntax.PreorderReasoning
> %default total
> multSV : (Num t) => t -> Vect m t -> Vect m t
> multSV…