-
``` coq
Set Universe Polymorphism.
Inductive paths A (x : A) : forall _ : A, Type := idpath : paths A x x.
Notation "x = y" := (@paths _ x y) (at level 70, no associativity) : type_scope.
Axioms A B …
-
**What happens:**
In a module, Agda accepts the following record and function definition without complaints:
```
record _suchThat_ (b : Set) (φ : Set → Set) : Set where
field
prop : φ b…
-
Consider the following code:
```agda
open import Agda.Primitive using (lsuc; lzero)
module Main where
data Nat : Set where
zero : Nat
succ : Nat -> Nat
-- ----------------------------…
-
Add charge readout for machines(especially accumulators) and equipment grids(cars/tanks/locomotives) that show percentage(0-100).
An example of how this would be useful is when using electricity from…
-
Fu Peng noted (7/8/15) that formulae could be marked coinductive, instead of predicates, i.e. in the following program:
```
k1 : Eq a => Eq (P a)
k2 : Eq f (g a) => Eq (Cmp f g a)
k3 : Eq f (Fix (Cm…
-
#### Description of the problem
The following code worked fine in Coq 8.14, but no longer works in Coq 8.15:
```coq
From Coq Require Import String.
From Coq.ssr Require Export ssreflect.
…
-
How would the following scenario be done with StellarGraph - note that I am interested in step 3: Can the loaded model be trained with just the new nodes and not have to spend the time re-training the…
-
```coq
Require Import Coq.Init.Notations.
Require Import Coq.Init.Datatypes.
Inductive Wrapper (T : Type) :=
| Wrap : T -> Wrapper T
.
Inductive Unwrapper :=
| Empty : Unwrapper
| Un…
-
#### Description of the problem
I'd like to have hash maps and hash sets where where keys (for map) / values (for sets) are the following types:
- `ident`
- `int`
- `string`
- `inductive`
…
-
http://paste.atlauncher.com/view/e6e37dbf When I decided to only have Chromaticraft and Inductive installed so you could get a cleaner look at the error. I'm unsure of why this happens; Crashes at Ini…