Search code examples
How to have a proposition of comparing two 'int' types in Coq?...


logiccoqcompcert

Read More
Need finding the right tactic over Int.lt...


coqcompcert

Read More
How to express "there exists a unique X" in Coq?...


coq

Read More
Step by step simplification in coq?...


coq

Read More
'else' in definitions - Coq...


coq

Read More
Coq nat type check on match...


typescoq

Read More
What is the downside of using functional extensionality in COQ...


coq

Read More
Find the definition and notations like ++ in Coq...


coq

Read More
Coq: Insufficient Justification error...


coq

Read More
Where did lt_index go?...


coq

Read More
How can a coq Set or Type be a proposition...


typessetcoqboolean-expressionfirst-order-logic

Read More
Coq: apply transitivity with substitution...


relationcoqtransitivity

Read More
What's the square bracket syntax [ |- Set] in Coq?...


coq

Read More
How to express subset relation in Coq?...


coqset-theory

Read More
Coq type error when matching with type family...


coq

Read More
Print existing setoids and morphisms in Coq...


coqrewriting

Read More
In Coq: inversion of existential quantifier with multiple variables, with one command?...


existscoqinversion

Read More
Unfolding nested definitions in Coq...


typeclasscoq

Read More
multiple successes in Coq branching and backtracking?...


coqcoq-tactic

Read More
what's the correct usage for Coq "local application of tactics"?...


coqcoq-tactic

Read More
Coq inversion tactic that works on the goal?...


coqcoq-tactic

Read More
What's the difference between revert and generalize tactics in Coq?...


coqcoq-tactic

Read More
Coq: a single notation for multiple constructors...


constructorcoq

Read More
Where is the Extensionality of predicates axiom Coq...


coq

Read More
Coq: Unknown interpretation for negative integer expressions...


coq

Read More
example for introduction pattern (p1 & ... & pn) does not work...


coq

Read More
How to apply Fixpoint definitions within proofs in Coq?...


coq

Read More
`No more subgoals, but there are non-instantiated existential variables` in Coq proof language?...


coq

Read More
Is one being penalized by using 'same_relation' (and possibly other library definitions)?...


coq

Read More
Best way to handle (sub) types of the form `{ x : nat | x >= 13 /\ x <= 19 }`?...


coq

Read More
BackNext