Search code examples
Prove that f(n) = Θ(g(n)) iff g(n) = Θ(f(n))...

algorithmprooftheorem-provingbig-o

Read More
How to prove the data are generated or calculated by TEE (e.g., Intel SGX)?...

proofteesgxenclave

Read More
Using loop invariants to prove correctness of a simple algorithm...

algorithmloopsproofloop-invariant

Read More
Why Coq doesn't allow inversion, destruct, etc. when the goal is a Type?...

coqproofinversion

Read More
How to prove r → (∃ x : α, r) in Lean...

logicprooftheorem-provinglean

Read More
Cases tactic in Lean does not create hypothesis...

prooflean

Read More
Dafny GCD lemma Proof...

proofdafnyproof-of-correctness

Read More
Lean 4 'unknown identifier Proof'...

prooftheorem-provinglean

Read More
TLA+ model checker fails to generate states...

prooftla+

Read More
Convert a Bits8 to a `Subset Nat (`LT` 256)`...

proofidrisdependent-type

Read More
Proving correctness in formal logic...

proofformal-methodspost-conditionshoare-logicproof-of-correctness

Read More
Proving equivalence of two rev_append implementations...

coqproofformal-verification

Read More
Can I safely assume that isomorphic types are equal?...

coqproofagdadependent-typetheorem-proving

Read More
How do I prove an existential goal that asks for a certain function in Coq?...

coqproof

Read More
Parametrizing a Module in Coq...

coqproof

Read More
How to write a 'safe' head in coq?...

coqproofdependent-type

Read More
Produce a function in Coq which outputs every witness to an existence-uniqueness axiom...

coqprooftheorem-proving

Read More
Using big-O to prove N^2 is O(2^N)...

big-oproof

Read More
Using Hoare-Rules to show PRECONDITION implies POSTCONDITION in a simple program (just 2 assignments...

proofproof-of-correctnesshoare-logic

Read More
Proving basic properties of recursive "less than" definition for naturals in Isabelle...

isabelleproofisar

Read More
Agda not eliminating clause in goal despite pattern matching on it...

typesproofagdatheorem-proving

Read More
Coq ssreflect sum of sums...

coqproofcoq-tacticssreflect

Read More
Apply function in goal in lean proof...

prooftheorem-provinglean

Read More
Could you help me design an algorithm and prove for this problem please?...

algorithmgreedyproof

Read More
Idris "did not change type" for rewrite with exact same type...

proofidris

Read More
Cauchy-Schwartz Inequality in Coq?...

coqproofcoq-tacticformal-verificationssreflect

Read More
Coq - adding choice function to context...

mathcoqproof

Read More
How to prove this invariant?...

adaproofinvariantsproof-of-correctnessspark-ada

Read More
arrange numbers to form largest number - proof of algorithm...

algorithmproof

Read More
Big theta notation in substitution proofs for recurrences...

algorithmsubstitutionrecurrenceproofclrs

Read More
BackNext