Skip to content
Snippets Groups Projects
Commit df663290 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Test case for `TCSimpl`.

parent 903bfaa4
No related branches found
No related tags found
1 merge request!521Add `TCSimpl` type class.
"tc_simpl_test"
: string
1 goal
P : nat → Prop
y : nat
============================
P (S (S (S (S (S (S y))))))
From stdpp Require Import prelude. From stdpp Require Import strings.
Lemma tc_simpl_test_lemma (P : nat Prop) x y :
TCSimpl x y
P x P y.
Proof. by intros ->%TCSimpl_eq. Qed.
Check "tc_simpl_test".
Lemma tc_simpl_test (P : nat Prop) y : P (5 + S y).
Proof.
apply (tc_simpl_test_lemma _ _ _ _). (* would be nicer with ssr [apply:] *)
Show.
Abort.
(** Check that [@Reflexive Prop ?r] picks the instance setoid_rewrite needs. (** Check that [@Reflexive Prop ?r] picks the instance setoid_rewrite needs.
Really, we want to set [Hint Mode Reflexive] in a way that this fails, but Really, we want to set [Hint Mode Reflexive] in a way that this fails, but
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment