summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4813.v
blob: 5f8ea74c1ac749592249514c7e3c8dd2e06e74ed (plain)
1
2
3
4
5
6
7
8
9
(* On the strength of "apply with" (see also #4782) *)

Record ProverT := { Facts : Type }.
Record ProverT_correct (P : ProverT) :=  { Valid : Facts P -> Prop ;
                                           Valid_weaken : Valid = Valid }.
Definition reflexivityValid (_ : unit) := True.
Definition reflexivityProver_correct : ProverT_correct {| Facts := unit |}.
Proof.
    eapply Build_ProverT_correct with (Valid := reflexivityValid).