Search code examples
Dependent Pair Types...


typescoqlogical-foundations

Read More
How can I prove excluded middle with the given hypothesis (forall P Q : Prop, (P -> Q) -> (~P ...


coqlogical-foundations

Read More
Understanding nat_ind2 in Logical Foundations...


coqlogical-foundationsproof-assistant

Read More
How do I apply (S n' <=? m) = true to S n' <= m?...


coqlogical-foundations

Read More
Software Foundations (lf): proving leb_plus_exists and plus_leb_exists...


coqlogical-foundations

Read More
Software Foundations Basics - Theorem lower_grade_lowers need to prove implication Eq = Lt -> Eq ...


coqcoq-tacticlogical-foundations

Read More
Software Foundations Basics Exercise - How do I access letter from grade?...


coqlogical-foundations

Read More
Cannot focus on a remaining unfocused goal in Coq...


coqlogical-foundations

Read More
Check cnat. and got Type return...


coqlogical-foundations

Read More
Proving MStar' in Logical Foundations (IndProp.v)...


coqlogical-foundations

Read More
How can I prove `add_le_cases` (`forall n m p q, n + m <= p + q -> n <= p \/ m <= q`)...


coqlogical-foundations

Read More
Mix-up of bool and Datatypes.bool after Require Import coq libraries...


coqlogical-foundations

Read More
Coq proving nonsensical inductive property implication?...


coqcoq-tacticlogical-foundations

Read More
How does the grading script of the LF series work for manually graded exercises?...


coqlogical-foundations

Read More
Quick Chick eqBoolArrowA_correct theorem...


coqlogical-foundations

Read More
Coq: unary to binary convertion...


coqlogical-foundations

Read More
Instance of Ord typeclass for option...


coqtypeclasslogical-foundations

Read More
IndProp: prove that Prop is not provable...


coqlogical-foundations

Read More
Mix-up of bool and Datatypes.bool after Require Import Omega...


coqlogical-foundations

Read More
Coq: help to formalize an informal proof...


coqlogical-foundations

Read More
How to apply a lemma to 2 hypothesis...


coqlogical-foundations

Read More
coq Basics: bin_to_nat function...


coqlogical-foundations

Read More
Rel: le_antisymmetric comprehension...


coqlogical-foundations

Read More
Rev.v le_antisymmetric...


coqlogical-foundations

Read More
Software Foundations: apply ... with ... tactic...


coqlogical-foundations

Read More
Software Foundations: proving leb_complete and leb_correct...


coqlogical-foundations

Read More
Logic: auxilliry lemma for tr_rev_correct...


coqlogical-foundations

Read More
Tactics: stuck in eqb_trans...


coqlogical-foundations

Read More
Proving that a reversible list is a palindrome in Coq...


coqpalindrometheorem-provinglogical-foundations

Read More
How to set implicit parameters for constructor...


coqlogical-foundations

Read More
BackNext