Skip to content

Commit

Permalink
Fix deprecation from MathComp 1.15
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed Jun 8, 2023
1 parent f555a76 commit 910634f
Show file tree
Hide file tree
Showing 3 changed files with 11 additions and 11 deletions.
2 changes: 1 addition & 1 deletion theories/acyclic.v
Original file line number Diff line number Diff line change
Expand Up @@ -52,7 +52,7 @@ Coercion equivalence_rel_trans : equivalence_rel >-> transitive.

Notation EquivalenceRel R Req := (EquivRel R Req Req Req).

#[export] Hint Resolve equiv_equivalence_rel.
#[export] Hint Resolve equiv_equivalence_rel : core.

Section EquivalencePartitionExtra.

Expand Down
8 changes: 4 additions & 4 deletions theories/extra.v
Original file line number Diff line number Diff line change
Expand Up @@ -261,17 +261,17 @@ Variable r : rel V.
Local Notation "x -[]-> y" :=
(connect r x y) (at level 10, format "x -[]-> y") .

Local Notation connect_to s := (connect (rel_of_simpl_rel (relto s r))).
Local Notation connect_to s := (connect (rel_of_simpl (relto s r))).

Local Notation "x -[ s ]-> y" := (connect_to s x y)
(at level 10, format "x -[ s ]-> y").

Local Notation "x =[]= y" := (symconnect r x y)
(at level 10, format "x =[]= y").

Local Notation symconnect_to a := (symconnect (rel_of_simpl_rel (relto a r))).
Local Notation symconnect_to a := (symconnect (rel_of_simpl (relto a r))).

Local Notation "x =[ a ]= y" := (symconnect (rel_of_simpl_rel (relto a r)) x y)
Local Notation "x =[ a ]= y" := (symconnect (rel_of_simpl (relto a r)) x y)
(at level 10, format "x =[ a ]= y").

Lemma connect_to1 (a : pred V) x y : y \in a -> r x y -> x -[a]-> y.
Expand Down Expand Up @@ -340,4 +340,4 @@ Qed.
Lemma setUDl (T : finType) (A B : {set T}) : A :|: B :\: A = A :|: B.
Proof. by apply/setP=> x; rewrite !inE; do !case: (_ \in _). Qed.

End extra_set.
End extra_set.
12 changes: 6 additions & 6 deletions theories/kosaraju.v
Original file line number Diff line number Diff line change
Expand Up @@ -20,17 +20,17 @@ Variable r : rel T.
Local Notation "x -[]-> y" :=
(connect r x y) (at level 10, format "x -[]-> y") .

Local Notation connect_to s := (connect (rel_of_simpl_rel (relto s r))).
Local Notation connect_to s := (connect (rel_of_simpl (relto s r))).

Local Notation "x -[ s ]-> y" := (connect_to s x y)
(at level 10, format "x -[ s ]-> y").

Local Notation "x =[]= y" := (symconnect r x y)
(at level 10, format "x =[]= y").

Local Notation symconnect_to a := (symconnect (rel_of_simpl_rel (relto a r))).
Local Notation symconnect_to a := (symconnect (rel_of_simpl (relto a r))).

Local Notation "x =[ a ]= y" := (symconnect (rel_of_simpl_rel (relto a r)) x y)
Local Notation "x =[ a ]= y" := (symconnect (rel_of_simpl (relto a r)) x y)
(at level 10, format "x =[ a ]= y").

Lemma connect_to_C1r x y z :
Expand Down Expand Up @@ -175,7 +175,7 @@ Section ConnectRelto.
Variable r : rel T.

Local Notation "x -[ s ]-> y" :=
(connect (rel_of_simpl_rel (relto s r)) x y)
(connect (rel_of_simpl (relto s r)) x y)
(at level 10, format "x -[ s ]-> y").

Local Notation "x -[]-> y" :=
Expand All @@ -184,7 +184,7 @@ Local Notation "x -[]-> y" :=
Local Notation "x =[]= y" := (symconnect r x y)
(at level 10, format "x =[]= y").

Local Notation "x =[ a ]= y" := (symconnect (rel_of_simpl_rel (relto a r)) x y)
Local Notation "x =[ a ]= y" := (symconnect (rel_of_simpl (relto a r)) x y)
(at level 10, format "x =[ a ]= y").

Local Notation "C[ x ]_( a , l )" := (can_to r x a l)
Expand Down Expand Up @@ -481,7 +481,7 @@ Definition pdfs := rpdfs #|T|.
Definition tseq := (foldl pdfs (setT, [::]) (enum T)).2.

Local Notation "x -[ l ]-> y" :=
(connect (rel_of_simpl_rel (relto l (grel g))) x y)
(connect (rel_of_simpl (relto l (grel g))) x y)
(at level 10, format "x -[ l ]-> y").
Local Notation "x -[]-> y" := (connect (grel g) x y)
(at level 10, format "x -[]-> y").
Expand Down

0 comments on commit 910634f

Please sign in to comment.