Search code examples
Theorem and Proof Environment in Beamer...


latexproofbeamerquartotheorem

Read More
How to instruct `auto` to simplify the goal during proof search?...


coqproof

Read More
Is is possible to rename a coq term?...


coqproofcoq-tactic

Read More
How to extract a variable from an exist clause...


proofdafny

Read More
Proof by reductio ad absurdum in Isabelle...


isabelleproof

Read More
Does sequencing an infinite list of IO actions by definition result in a never-ending action? Or is ...


haskellfunctional-programminglanguage-lawyerproofio-monad

Read More
Proof that the halting problem is NP-hard?...


theoryproofhalting-problemnp

Read More
How would I prove that b = c if (andb b c = orb b c) in coq?...


coqproofproof-of-correctness

Read More
Sledgehammer output with vampire...


isabelleproof

Read More
Agda Recursion on Proof...


proofagdaagda-mode

Read More
Agda Unresolved Metas...


proofagda

Read More
Proof of dynamic programming solution for Leetcode 818: Racecar...


algorithmdynamic-programmingproofcorrectnessproof-of-correctness

Read More
What is the proof of of (N–1) + (N–2) + (N–3) + ... + 1= N*(N–1)/2...


formulaproof

Read More
Coq simpl / unfold only once. (Replace part of goal with the result of one iteration of a function.)...


coqproofcoq-tacticinduction

Read More
Counterexample for first-order logic assertion...


logicprooffirst-order-logic

Read More
How can we prove by induction that binary search is correct?...


algorithmsearchbinary-searchproof

Read More
Is there a way for Coq to recall it already proved a property for the same element in the same proof...


automationcoqproof

Read More
How would you write ∀ y ∈ R+, ∃ z ∈ R, e^z = y in pseudocode?...


algorithmmathcomputer-scienceproof

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
Is there a proof that runST is indeed pure?...


haskellsemanticsproofst-monad

Read More
Is it possible to disambiguate instances with an intermediate step?...


haskelltypeclassproof

Read More
Prove (p → ¬ q) → ¬ (p ∧ q) in Lean4...


logicdiscrete-mathematicsprooflean

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


logiccoqprooftheorem-provinglean

Read More
Dafny existence statement cause slowness?...


proofdafnyfinite-group-theory

Read More
How to understand the time complexity of Kademlia node operation...


algorithmtime-complexityproofdhtkademlia

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


isabelleprooftheorem-provingformal-verificationisar

Read More
Finding 0 - (Python Testing) random.uniform(0,1) Double Precision Floating Point...


pythonrandomieee-754proof

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
Cannot prove in Dafny that variance(x)>=0...


covarianceassertionprooftheorem-provingdafny

Read More
BackNext