-
Hi~ @matenure
I want to change the some code to pytorch version, so I have some question about the use of inductive file and the transductive file. And if I have an inductive task for GCN, but the o…
-
https://aconite-ac.github.io/theorem_proving_in_lean4_ja/inductive_types.html#enumerated-types-%E5%88%97%E6%8C%99%E5%9E%8B
> We will use the match expression to define a function from Weekday to th…
-
On Coq 8.9, with coq-equations version 1.2 beta2,
```
From Equations Require Import Equations.
Require Import Vector.
Derive DependentElimination for t.
Anomaly "Uncaught exception Reductio…
-
### Prerequisites
* [X] Put an X between the brackets on this line if you have done all of the following:
* Check that your issue is not already [filed](https://github.com/leanprover/lean4/iss…
-
I wanted to experiment with the possibility of using template-coq as a tactic language to solve a "simple" problem with universes (which was the impetus for my initial question on slack). Here's the p…
-
Found live by @pigworker. The first mixed co-pattern and pattern matching
definition leads to a case tree too strict in `n` for `F (r zero n) (k , l) refl`
to make sense.
However, Agda is not con…
-
Hello Lean Developer,
I was writing universe-lifting function due to lack of cumulative universe
```
inductive liftU.{u v} (X: Type u) : Type (max v (u + 1)) :=
| inh : X → liftU X
```
I…
-
## Problem
There's a tension between two desires: to have seamlessly composable code gadgets and to have proper abstraction barriers.
Postulating a new name is a form of human communication, names…
-
The function `IndPredBelow.mkBelow` fails to generate `brecOn` for the following inductive predicate.
```lean
set_option trace.Meta.IndPredBelow true in
inductive TransClosure (r : α → α → Prop) : …
-
Yo!
So I'm slightly confused about the documentation regarding this feature:
"Limit switch socket 24V/5V/3.3V optional, ready for more other equipment, such as -inductive sensor, BL-Touch"
I'…