Search code examples
How does the "intro ->" in Coq work on context?...


coq

Read More
Coq datatype - pair of pair with bracket...


typesfunctional-programmingcoqcoqide

Read More
apply ltac to subexpression of a goal...


coqltac

Read More
Defining functions inside proof scope...


coqcoq-tactic

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
Computational behaviour of Successor...


coq

Read More
Parametrizing a Module in Coq...


coqproof

Read More
Unifying types of identical meanings...


coq

Read More
Alternative tactic for `ssreflect`'s `move=>`...


coqssreflect

Read More
Implicit arguments propagation...


coq

Read More
proof of adding 1 to some number changes the parity in Coq...


coq

Read More
How to use symmetricity of an equality on Coq...


coq

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


coqproofdependent-type

Read More
Why unable to perform case analysis in rather simple case...


coqssreflect

Read More
Is this a correct application of 'exists' in Coq?...


coq

Read More
Coq: Cannot guess decreasing argument of fix...


coqcoqide

Read More
Is there any way to rewrite the function in "is_lim"?...


coqcoq-tactic

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


coqprooftheorem-proving

Read More
Cannot find a physical path bound to logical path matching suffix <> and prefix Coquelicot...


coqcoqide

Read More
Coq: Strong specification of haskell's Replicate function...


haskellcoqcoqidecoq-extraction

Read More
how to simplify basic arithmetic in more complex goals...


coqssreflect

Read More
Coq: Prove Inductive relation (vs Fixpoint)...


coqcoqide

Read More
Coq: Proof of list pair...


coqcoqide

Read More
Reduction in coq when the simpl or cbn tactics are not effective...


coqcoq-tactic

Read More
Destructing equality of dependent records in coq...


coqdependent-type

Read More
The type checker's behavior while pattern matching in Coq...


coq

Read More
Don't understand `destruct` tactic on hypothesis `~ (exists x : X, ~ P x)` in Coq...


coqcoq-tactic

Read More
What does "eq^~" mean in Coq?...


coq

Read More
Coq extraction to Haskell...


haskellcoq

Read More
BackNext