-
Hi, thanks for making this tool! I'm just getting started with it.
I have a file called proved_theorem.v which has:
Theorem trial: forall n: nat, 1 + n = S n.
Proof.
intros.
eauto.
Qed.
…
-
In MMJ2, whenever applying a theorem leaves unresolved substitutions, like when applying `~addcan2ad` in the example below, [work variables](http://mmj2-doc.tirix.org/doc/WorkVariables.html) such as `…
tirix updated
2 years ago
-
Hi,
If a Lemma type is too long and wrote on multiple lines, the type is cut in the Outline buffer :
Here is the lemma in my file :
```
Lemma get_app_l {A} (l l':list A)(n:nat) : n < length…
-
This makes a problem so it is possible to dupe with every single item of the items in Extra Utililities.
It has been tested with QED, A generator, Transfer node.
The process to reproduce it:
1. Open…
-
This program:
```haskell
{-@ LIQUID "--higherorder" @-}
{-@ LIQUID "--exactdc" @-}
module Bug where
import Language.Haskell.Liquid.ProofCombinators
data U1 p = U1
data M…
-
#### Description of the problem
I am completely stumped by this code:
```coq
From Coq Require Import String ZArith Relations.
Global Open Scope Z.
Inductive expr :=
| Var (x : string…
-
Note: the issue was created automatically with bugzilla2github tool
Original bug ID: BZ#5748
From: @gares
Reported version: 8.7+beta1
-
```coq
Monomorphic Universe hyp.
Definition hyps_universes : M@{hyp} (mlist Hyp@{Set}) := M.hyps.
Goal Type@{hyp} -> mlist Hyp@{Set}.
MProof.
intros T.
Set Printing All.
Set Printing …
Janno updated
3 years ago
-
```
During the demo, this sequence of commands is fairly common:
> let test : Set
> root
> next
After 'root', we expect to be deep *down* in the ProofState, so we would think
that 'prev' is the …
-
EDIT: the original definition acts as a self-redefinition, ie importing it erases any past redefinitions.
I find the following behavior puzzling:
```coq
Module M.
Ltac foo := fail.
End M.
…