Search code examples
Non-trivial Fixpoint on nested recursive types...


coqtheorem-proving

Read More
What is the difference between Lemma and Theorem in Coq...


coqtheorem-proving

Read More
Failed to solve constraints: (k ≤ 5) x (k * 2 ≡ 5). How could I make this work?...


agdatheorem-proving

Read More
How can I prove dependent function types equal in Agda?...


agdadependent-typetheorem-proving

Read More
Installing Z3 binding with haskell on mac...


haskellstackz3theorem-provingcabal-install

Read More
Programming in the Calculus of Inductive Constructions with Coq...


coqdependent-typetheorem-proving

Read More
What's the role of unification in Coq's core type system?...


coqdependent-typetype-systemstheorem-provingunification

Read More
(Z3Py) Using all_smt to generate all solutions of a model...


pythonz3smtz3pytheorem-proving

Read More
Proving Transitivity of Pointwise Relations on Lists in Coq...


coqtheorem-provingcoq-tactic

Read More
Proving extensional equality of two functions...


functional-programmingcoqtheorem-proving

Read More
Instantiate typeclass over type_synonym...


typesisabelletheorem-proving

Read More
Recursive function leads to simplifier loop in Isabelle...


recursionisabelletheorem-proving

Read More
Proving n + S n = S (n + n) without n + S m = S (n + m)...


logiccoqprooftheorem-proving

Read More
Why can't all existential binders be replaced by unique constants during skolemization?...


logicprooftheorem-provingtype-theory

Read More
Trace tauto, finish...


debuggingmaththeorem-provinglean

Read More
Implementation for decision procedure for the theory of the reals...


z3smttheorem-provingcvc4

Read More
definitions with fin types (lean)...


maththeorem-provinglean

Read More
How to prove A \/ False -> A in Coq?...


logiccoqtheorem-proving

Read More
Lean4: Proving that `(xs = ys) = (reverse xs = reverse ys)`...


logiccoqprooftheorem-provinglean

Read More
How to proceed in Isabelle when the goal has implications and existentials?...


isabelleprooftheorem-provingformal-verificationisar

Read More
Proving a Type is Uninhabited in Agda...


agdatheorem-provinginduction

Read More
Not able to make a simple proof in Dafny: if `0<=a<=1 & 0<=b<=1 & -1<=c<=1...


z3prooftheorem-provingdafny

Read More
An unexpected 'possible division by zero' when values are known to be positive...


divide-by-zerotheorem-provingdafny

Read More
Agda: Can't find std-lib when installing with Stack...


functional-programmingagdadependent-typetheorem-provingagda-mode

Read More
Proving a covariance inequality in Dafny, use contradiction?...


z3covariancetheorem-provingdafnyinduction

Read More
Cannot prove in Dafny that variance(x)>=0...


covarianceassertionprooftheorem-provingdafny

Read More
Cannot prove in Dafny that f(a,b)=f(b,a)...


z3theorem-provingdafnyterminationformal-verification

Read More
Dafny cannot prove that 'a^2<=b^2*c^2' implies 'a<=b*c' for reals greater than...


z3theorem-provingdafnysquare-root

Read More
Modular arithmetic proofs in agda...


mathproofagdatheorem-provingagda-stdlib

Read More
Does Z3 (and other solvers) always use terminating decision procedures when possible?...


arraysz3smttheorem-provingfirst-order-logic

Read More
BackNext