Search code examples
how to prove 2 step induction of list in coq using fix tactic...


coqtheorem-provingcoq-tactic

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


coqtheorem-proving

Read More
Isabelle 2017 -- getting started...


isabelletheorem-proving

Read More
Coq is reusing a term in Induction Hypothesis, instead of creating a fresh one...


coqtheorem-provinginduction

Read More
Can we have an arbitrary big upper bound for the looping variable in Dafny?...


dafnytheorem-proving

Read More
How to prove mathematical induction formulae in LEAN theorem prover?...


theorem-provinglean

Read More
how to prove the correctness of a c program with coq...


ctheorem-proving

Read More
Wrong Typeclass Instance used in Coq Proof...


functional-programmingcoqtypeclassdependent-typetheorem-proving

Read More
How to define mutual inductive propositions in Lean?...


dependent-typetheorem-provingmutual-recursionlean

Read More
Non-trivial Fixpoint on nested recursive types...


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
BackNext