-
The new treatment of globs (introduced in #440 which fixes #102) leads to an unsoundness.
The theory below illustrates that.
(There are some admits, I can fill them in if they are required, but I …
-
I'm using `HSubst` in a case where the outer type doesn't have variables of its own (first-order logic; terms are a separate type, variables are bound by quantifiers in the props). I want to derive `H…
-
If I execute the following file to the end in CoqIDE (and vscoq), and I close the file, the coqproofworker that tried to check the (diverging) proof of the lemma asynchornous in the background doe…
-
For instance modifying the example in the doc to add Polymorphic:
~~~coq
Require Import Relation_Definitions Setoid.
Record Setoid : Type :=
{ car: Type;
eq: car -> car -> Prop;
refl…
-
Hi,
is this project still maintained. We like it very much and would hate to see it go abandoned.
We'd be glad to help!
-
```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…
-
thread for ideas and discussions for RL env. The standard/common way in ML is to use OpenAIs Gym (https://gym.openai.com/). Currently, I am unsure if that is what we want for our environment (e.g. cuz…
-
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
-
Hi!
I'm very interesting in your works. I would like to reproduce your results but I have a problem when I run vocabulary.py error :"rdkit.Chem.rdchem.KekulizeException: Can't kekulize mol. Unkekul…