Search code examples
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
proof L = {a^n b^m | n>=m} is irregular language...

proofpumping-lemma

Read More
Modular arithmetic proofs in agda...

mathproofagdatheorem-provingagda-stdlib

Read More
Proof that "if m <= n then max(m, n) = n" in Coq...

coqproof

Read More
How does Dafny support induction if Z3 does not?...

z3proofdafnyformal-verificationinduction

Read More
How to prove time complexity of bubble sort using dafny?...

time-complexitybubble-sortproofdafny

Read More
Using any/all with proof or examples...

python-3.xpython-3.8proofany

Read More
Coq: Implementation of splitstring and proof that nothing gets deleted...

coqproofinduction

Read More
Making sure that the function I am using returns the correct kind of values in haskell. (i.e does no...

haskellproofproof-of-correctness

Read More
dafny sequence to multiset...

proofdafnymultiset

Read More
Can you check for duplicates by taking the sum of the array and then the product of the array?...

algorithmduplicatesproof

Read More
Lawvere's fixed point theorem in agda...

proofagdatheorem-provingcategory-theory

Read More
Dafny proof by contradiction with quantifiers...

proofdafnyset-theory

Read More
Proofs of simple arithmetic expressions...

coqproof

Read More
Proof of having k edge-disjoint paths there and back...

algorithmgraphgraph-theoryproofmax-flow

Read More
How to do an inductive proof...

coqproofinduction

Read More
How to prove insert_BST in Coq...

logiccoqproofcoq-tacticproof-of-correctness

Read More
Creating Coq tactic: how to use a newly generated name?...

coqproofcoq-tactic

Read More
How do you lookup the definition or implementation of Coq proof tactics?...

mathcoqproof

Read More
Why can't programs be proven?...

maththeoryproofaxiomformal-verification

Read More
How to prove that another definition of permutation is the same as the Default Permutation Library f...

permutationcoqproofinduction

Read More
Coq - Rewriting a FMap Within a Relation...

programming-languagescoqproof

Read More
Find subset with elements that are furthest apart from eachother...

algorithmproof

Read More
BackNext