-
eg with `Inductive Foo := foo : Type -> Foo.` it doesn't matter whether it's declared template or not, so why warn?
See also https://github.com/coq/coq/pull/8488#issuecomment-450424437
-
### Prerequisite
- [X] I have searched [Issues](https://github.com/open-mmlab/mmgeneration/issues) and [Discussions](https://github.com/open-mmlab/mmgeneration/discussions) but cannot get the expec…
-
**What version of Racket are you using?**
Racket v8.12 [cs]
**What program did you run?**
At the command-line REPL:
```racket
Welcome to Racket v8.12 [cs].
> (define v1* add1)
> (define…
-
https://github.com/cornellhyperloop/electrical/blob/master/State_Estimation/src/statemachine.cpp
-
Hi,
I tried to do some training on coq, but when i define this :
`Inductive nat : Type :=
| O : nat
| S : nat -> nat.
Check (S (S (S (S O)))).`
i don't get 4 as printed... Also when i try thi…
-
### Prerequisites
* [X] Check that your issue is not already filed:
https://github.com/leanprover/lean4/issues
* [X] Reduce the issue to a minimal, self-contained, reproducible test case.
…
-
Reproduction:
1. Open foo.v, which is not formatted, e.g.
```
Inductive day : Type :=
| monday
| tuesday
| wednesday
| thursday
| friday
| saturday
| sunday.
```
2. Press…
-
I don't think the following code should be accepted:
```agda
open import Agda.Builtin.Size
record Sized-type (i : Size) : Set₁ where
inductive
field
force : Size< i → Set
open Sized…
-
#### Description of the problem
```coq
Inductive t (A : Type) : unit -> Type := tc : A -> t A tt.
Lemma k A (H: t A tt) : True.
symmetry in H.
(* Anomaly "in retyping: Not an arity." *)
```
…
-
Inequalities:
* Have a set of inductive inequality definitions (http://www.reddit.com/r/Idris/comments/6ya7jg/unification_problems_associated_with_totality/), and bijections to the witness-style ones…