Search code examples
How to prove reverse nil is nil in Lean...


theorem-provingformal-verificationlean

Read More
Isabelle Code Generation and Linear Order...


isabelletheorem-proving

Read More
How to perform multiple exists-eliminations that all share a single multivariate universally-quantif...


theorem-provinglean

Read More
How to use `exists.elim` in Lean?...


theorem-provinglean

Read More
How can one prove (¬ ∀ x, p x) → (∃ x, ¬ p x) from first principles in LEAN?...


theorem-provinglean

Read More
Coq : Admit assert...


coqtheorem-proving

Read More
Isabelle/HOL restrict codomain...


isabelletheorem-proving

Read More
Why does `rewrite` of associativity fail in binomial theorem proof in LEAN?...


prooftheorem-provinglean

Read More
Simp does not use the provided lemma in Isabelle...


isabelletheorem-provingsimplification

Read More
undefined in Isabelle/HOL...


isabelletheorem-proving

Read More
How to prove two statements in propositional logic using LEAN?...


theorem-provinglean

Read More
Isabelle/HOL Question about Sets of Tuples...


isabelletheorem-proving

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


theorem-provinglean

Read More
Coq: type mismatch on dependent lists which could be solved by a proof...


listcoqdependent-typetheorem-proving

Read More
Induction issue...


theorem-provinglean

Read More
Coq: prove that if (A, B) = (C, D) then A = C /\ B = D...


coqtheorem-proving

Read More
How do you read the coq quantifier `forall P: Set -> Prop`?...


typescoqprooftheorem-proving

Read More
Proving the false case of an if and only if in Agda...


agdatheorem-proving

Read More
Simple refl-based proof problem in Lean (but not in Agda)...


agdatheorem-provinglean

Read More
Coq theorem proving: Simple fraction law in peano arithmetic...


coqtheorem-provingpeano-numbers

Read More
How does one properly simplify a coq goal with a previous lemma?...


coqtheorem-provingcoq-tactic

Read More
Well-founded recursion in Lean...


theorem-provinglean

Read More
ATS Proof: Why does this static if need greater than or equal to?...


if-statementtheorem-provingats

Read More
How can i prove that cons after uncons over coinductive list(a.k.a Stream) are identity, in Agda?...


agdatheorem-provingcoinduction

Read More
Basic Isabelle sequence limit proof...


isabelleprooftheorem-proving

Read More
Is this formalization of the empty set correct in Agda?...


logicagdatheorem-provingset-theory

Read More
Idris: Is there a way to reference an abstracted variable in an equality proof?...


idristheorem-proving

Read More
How to use a refutation to direct the type checker in Haskell?...


haskelltypesdependent-typetheorem-proving

Read More
In Coq, are there tactics for working with Rabs, Rineq?...


coqtheorem-provingcoq-tacticreal-number

Read More
What kind of functions preserve properties of closure?...


isabelletheorem-proving

Read More
BackNext