-
The following definition fails to be proven (or take any steps) with the prover:
```
module ITEMS-SYNTAX
imports DOMAINS-SYNTAX
syntax Item ::= "A"
syntax Items ::= List{Item, "|"}
e…
-
eg
~~~coq
Fixpoint edivn_rec d m q {struct m} :=
match Nat.sub m d with
| 0 => (q, m)
| S m' => edivn_rec d m' (S q)
end.
~~~
`Nat.sub m d` is smaller than `m` and so `m'` is strictly …
-
Unlike other binary relations over lists, `Data.List.Relation.Binary.Permutation.(Setoid/Propositional)` are implemented separately which results in an awful lot of proof duplication. It also means th…
-
At the moment we have:
```agda
_≤_ : Rel A _
x ≤ y = (x < y) ⊎ (x ≈ y)
```
and
```agda
data ReflClosure {A : Set a} (_∼_ : Rel A ℓ) : Rel A (a ⊔ ℓ) where
refl : Reflexive (ReflClosure …
-
Timmermans, Stefan and Iddo Tavory. 2012. [“Theory Construction in Qualitative Research: From Grounded Theory to Abductive Analysis.”](http://static1.squarespace.com/static/54282b13e4b0e88c57a39d51/t/…
-
The idea is to turn this:
```c#
Insert.IntoTable("TableName")
.Row(new { SomeColumn = "test1" })
.Row(new { SomeColumn = "test2" });
```
into this:
```c#
Insert.IntoTable("TableName")
.Rows(n…
-
This may be a known fact, but Agda allows definitions that occur in their own type:
```agda
A : Set
a : A
data D : A → Set where
d : D a
A = D a
a = d
```
The term `d` h…
-
See https://github.com/oscoin/oscoin/pull/407#discussion_r267220722
In a nutshell, #402 left out two things during chain selection:
- We didn't prune chains which were selected but that failed f…
-
The PlusCal translator could generate a `PCOK` from the set of possible pc values that is manually added as a conjunct in a user-provided `TypeOK`, and that is robust against algorithm changes:
```…
-
#### Description of the problem
A simple proof script that involves `n` constructor applications can lead to a proof term whose type-checking time is quadratic in `n`. This is illustrated by th…