-
Here is the code snippet:
``` C
/*@
lemma void insync_head_matches(list alist)
requires alist == nil;
ensures fst(head(alist)) == 1;
{
}
@*/
```
The master-version of VeriFast fails on t…
necto updated
8 years ago
-
### Proposal
In a language that compiles pattern matching down to recursor theroems, it seems natural to be able to define custom recursors and have pattern matching and induction work just as befo…
-
Hello authors, we have reproduced your code. We loaded the classifier of ImageNette, and the accuracy could reach 0.99, but we trained from scratch without loading any weights, and the result was only…
-
As primitive integers, floats, and arrays are added to coq, their behavior is specified using axioms. It would be cool if there was a proof that these axioms are consistent, constructing an isomorphic…
-
A problematic consequence is that it triggers anomaly when unquoting.
```coq
From Coq Require Import Strings.String.
From MetaCoq.Template Require Import All.
Set Primitive Projections.
(* G…
-
Browsing [the documentation](https://leanprover-community.github.io/mathlib4_docs/Lean/Expr.html#Lean.Expr) I was a bit confused why some paragraphs are randomly indendet, e.g. “The [bvar](https://lea…
-
With the following code:
```
Inductive paths {A : Type} (a : A) : A -> Type :=
idpath : paths a a.
Scheme paths_ind := Induction for paths Sort Type.
```
I get the following error message:
``…
-
Example:
```
type t =
| Foo
| Bar
| Foobar of t * t
let rec just_id = function
| Foo -> Foo
| Bar -> Bar
| Foobar (t0, t1) -> Foobar (just_id t0, just_id t1)
```
Produced `cmm…
riaqn updated
8 months ago
-
The problem is described in the comments of the following code:
```fstar
// Two monads, with returns and binds
assume val m1: Type0 -> Type0
assume val m2: Type0 -> Type0
assume val return1: …
TWal updated
4 months ago
-
### Proposal
I think structures should work in mutual blocks. #2587 reports an error message related to this feature, and everyone commented in the issue expected this to work (I expect this to ful…