Skip to content

Commit

Permalink
Merge PR #18910: Set some basic rewriting primitives in Type opaque f…
Browse files Browse the repository at this point in the history
…or TC search.

Reviewed-by: SkySkimmer
Ack-by: olaure01
Co-authored-by: SkySkimmer <SkySkimmer@users.noreply.github.com>
  • Loading branch information
coqbot-app[bot] and SkySkimmer committed Apr 19, 2024
2 parents ebea542 + 73c46f4 commit d1da9f7
Show file tree
Hide file tree
Showing 3 changed files with 8 additions and 5 deletions.
Original file line number Diff line number Diff line change
@@ -0,0 +1,5 @@
- **Changed:**
``Coq.CRelationClasses.arrow``, ``Coq.CRelationClasses.iffT`` and
``Coq.CRelationClasses.flip`` are now :cmd:`Typeclasses Opaque`
(`#18910 <https://github.com/coq/coq/pull/18910>`_,
by Pierre-Marie Pédrot).
6 changes: 1 addition & 5 deletions test-suite/bugs/bug_7675_3.v
Original file line number Diff line number Diff line change
Expand Up @@ -58,19 +58,15 @@ Ltac test S b1 b2 b3 b4 :=
unfold arrow, Basics.arrow; now rewrite <- HR | clear Ht ].

Goal True.
test Ri true true true true.
Proof.
test Ra true true true true.
test Rb false false false false.
test RBi true true true true.
test RBa true true true true.
test RBb false false false false.
test RTi true true true true.
test RTa true true true true.
test RTb false false false false.
test RRBi true true true true.
test RRBa true true true true.
test RRBb false false false false.
test RRTi true true true true.
test RRTa true true true true.
test RRTb false false false false.
apply I.
Expand Down
2 changes: 2 additions & 0 deletions theories/Classes/CRelationClasses.v
Original file line number Diff line number Diff line change
Expand Up @@ -33,6 +33,8 @@ Definition flip {A B C : Type} (f : A -> B -> C) := fun x y => f y x.

Definition iffT (A B : Type) := ((A -> B) * (B -> A))%type.

Global Typeclasses Opaque flip arrow iffT.

(** We allow to unfold the [crelation] definition while doing morphism search. *)

Section Defs.
Expand Down

0 comments on commit d1da9f7

Please sign in to comment.