-
Currently, when one extracts a client from an API definition, she gets a tree of functions running inside `ClientM` monad:
```
type MyAPI = "foo" :> Capture "x" Int :> Get '[JSON] Foo
: "…
-
TTKMorseSmaleComplex returns a 1-Separatrices object (output port 1). It has the fields
SeparatrixFunctionMaximum, SeparatrixFunctionMinimum, SeparatrixFunctionDifference
which suppose to reflect th…
-
While writing a compiler from Haskell Core to LLVM ([veggies](https://github.com/nomeata/veggies)) I noticed that it is very tedious to have to explicitly state the type of everything in the LLVM AST.…
-
Component: **algebra**
Keywords: **sd87**
Author: **Julian Rüth, Travis Scrimshaw**
Branch/Commit: **[`5a3e684`](https://github.com/sagemath/sagetrac-mirror/commit/5a3e684d060c68da916471acc34ef…
-
I tried to encode `ComposeLinkUTest::test_execute_2()` in scheme, to see what happens. I believe the intended encoding is this:
```
(define f1 (Project (Number 0)))
(define f2 (Lambda
(Vari…
linas updated
6 years ago
-
Hi, I reinvented the wheel before I found your library. But when I wanted to create the actual vectors at compile time I was stuck with no way to make them in a general way. Until I was able to make a…
-
I end up basically having to have one line per action due to the combination of the long function name and the type application plus the parameters themselves. IMO a name like `action` would be great.
-
| | |
|--------------------|----|
| Bugzilla Link | [PR34485](https://bugs.llvm.org/show_bug.cgi?id=34485) |
| Status | RESOLVED FIXED |
| Importance | P…
-
```
[1 of 3] Compiling Data.Vector.Generic.Sized ( src/Data/Vector/Generic/Sized.hs, .stack-work/dist/x86_64-osx/Cabal-1.22.5.0/build/Data/Vector/Generic/Sized.o )
/private/var/folders/…
-
When checking
```lean
inductive some_dep_type : bool → Type
| lala : Π b, some_dep_type b
def some_function (b : bool) (p : some_dep_type b) : unit := ()
lemma some_function_congruence :
…
timjb updated
7 years ago