How to reduce a cofix expression?...
Read MoreCoq vector: shiftin, shiftout, and last...
Read MoreRocq: Transparent aliased definition (that instance solver sees though)...
Read MoreWhy are logical connectives and booleans separate in Coq?...
Read MoreWhat's the difference between Program Fixpoint and Function in Coq?...
Read MoreIs there any difference between "parameters" and "indices" in Coq theorems?...
Read MoreHow can I prove Proof Irrelevance from Propositional Extensionality in Coq?...
Read Morehow to prove 2 step induction of list in coq using fix tactic...
Read MoreWhat is the difference between Lemma and Theorem in Coq...
Read MoreCoq Error Syntax error: '.' expected after [gallina] (in [vernac_aux])...
Read MoreI'm having difficulty definining a property in Coq, not sure how to approach...
Read MoreCoq is reusing a term in Induction Hypothesis, instead of creating a fresh one...
Read MoreHow to prove theorems about mutual inductive types by using tactics in Coq?...
Read MoreEfficient Record Construction in Coq: Is Direct Proof Inclusion Possible?...
Read MoreAgda-like programming in Coq/Proof General?...
Read MorePigeonhole proof without decidable equality or excluded middle...
Read MoreWhy does Coq solve_in_Union tactic fail directly but works through assertion of identical goal?...
Read MoreHow can I prove excluded middle with the given hypothesis (forall P Q : Prop, (P -> Q) -> (~P ...
Read MoreUnfolding an opaque fixpoint in Coq...
Read MoreLtac for deterministic rewriting/sorting of operands...
Read MoreCan I use a tactics under `coqtop -nois`?...
Read MoreWhat is to be used in place of exfalso omega?...
Read MoreCasting a value from one fintype to another?...
Read MoreHow can we use the familiar notation of integer arithmetics in ssreflect?...
Read More