Skip to content

Commit

Permalink
Adapt to coq/coq#18705
Browse files Browse the repository at this point in the history
  • Loading branch information
proux01 committed Feb 24, 2024
1 parent 3c925f7 commit 36cd2b9
Show file tree
Hide file tree
Showing 334 changed files with 1,010 additions and 1,010 deletions.
14 changes: 7 additions & 7 deletions UniMath/Algebra/Apartness.v
Expand Up @@ -28,11 +28,11 @@ Qed.

Definition aprel (X : UU) := ∑ ap : hrel X, isaprel ap.
Definition aprel_pr1 {X : UU} (ap : aprel X) : hrel X := pr1 ap.
Coercion aprel_pr1 : aprel >-> hrel.
#[reversible] Coercion aprel_pr1 : aprel >-> hrel.

Definition apSet := ∑ X : hSet, aprel X.
Definition apSet_pr1 (X : apSet) : hSet := pr1 X.
Coercion apSet_pr1 : apSet >-> hSet.
#[reversible] Coercion apSet_pr1 : apSet >-> hSet.
Arguments apSet_pr1 X: simpl never.
Definition apSet_pr2 (X : apSet) : aprel X := pr2 X.
Declare Scope ap_scope.
Expand Down Expand Up @@ -71,11 +71,11 @@ Definition istightap {X : UU} (ap : hrel X) :=

Definition tightap (X : UU) := ∑ ap : hrel X, istightap ap.
Definition tightap_aprel {X : UU} (ap : tightap X) : aprel X := pr1 ap ,, (pr1 (pr2 ap)).
Coercion tightap_aprel : tightap >-> aprel.
#[reversible] Coercion tightap_aprel : tightap >-> aprel.

Definition tightapSet := ∑ X : hSet, tightap X.
Definition tightapSet_apSet (X : tightapSet) : apSet := pr1 X ,, (tightap_aprel (pr2 X)).
Coercion tightapSet_apSet : tightapSet >-> apSet.
#[reversible] Coercion tightapSet_apSet : tightapSet >-> apSet.

Definition tightapSet_rel (X : tightapSet) : hrel X := (pr1 (pr2 X)).
Declare Scope tap_scope.
Expand Down Expand Up @@ -180,18 +180,18 @@ Qed.

Definition apbinop (X : tightapSet) := ∑ op : binop X, isapbinop op.
Definition apbinop_pr1 {X : tightapSet} (op : apbinop X) : binop X := pr1 op.
Coercion apbinop_pr1 : apbinop >-> binop.
#[reversible] Coercion apbinop_pr1 : apbinop >-> binop.

Definition apsetwithbinop := ∑ X : tightapSet, apbinop X.
Definition apsetwithbinop_pr1 (X : apsetwithbinop) : tightapSet := pr1 X.
Coercion apsetwithbinop_pr1 : apsetwithbinop >-> tightapSet.
#[reversible] Coercion apsetwithbinop_pr1 : apsetwithbinop >-> tightapSet.
Definition apsetwithbinop_setwithbinop : apsetwithbinop -> setwithbinop :=
λ X : apsetwithbinop, (apSet_pr1 (apsetwithbinop_pr1 X)),, (pr1 (pr2 X)).
Definition op {X : apsetwithbinop} : binop X := op (X := apsetwithbinop_setwithbinop X).

Definition apsetwith2binop := ∑ X : tightapSet, apbinop X × apbinop X.
Definition apsetwith2binop_pr1 (X : apsetwith2binop) : tightapSet := pr1 X.
Coercion apsetwith2binop_pr1 : apsetwith2binop >-> tightapSet.
#[reversible] Coercion apsetwith2binop_pr1 : apsetwith2binop >-> tightapSet.
Definition apsetwith2binop_setwith2binop : apsetwith2binop -> setwith2binop :=
λ X : apsetwith2binop,
apSet_pr1 (apsetwith2binop_pr1 X),, pr1 (pr1 (pr2 X)),, pr1 (pr2 (pr2 X)).
Expand Down
60 changes: 30 additions & 30 deletions UniMath/Algebra/BinaryOperations.v
Expand Up @@ -425,7 +425,7 @@ Definition make_isgrop {X : UU} {opp : binop X} (is1 : ismonoidop opp) (is2 : in
isgrop opp := tpair (λ is : ismonoidop opp, invstruct opp is) is1 is2.

Definition pr1isgrop (X : UU) (opp : binop X) : isgrop opp -> ismonoidop opp := @pr1 _ _.
Coercion pr1isgrop : isgrop >-> ismonoidop.
#[reversible] Coercion pr1isgrop : isgrop >-> ismonoidop.

Definition grinv_is {X : UU} {opp : binop X} (is : isgrop opp) : X -> X := pr1 (pr2 is).

Expand Down Expand Up @@ -611,7 +611,7 @@ Definition make_isabmonoidop {X : UU} {opp : binop X} (H1 : ismonoidop opp) (H2

Definition pr1isabmonoidop (X : UU) (opp : binop X) : isabmonoidop opp -> ismonoidop opp :=
@pr1 _ _.
Coercion pr1isabmonoidop : isabmonoidop >-> ismonoidop.
#[reversible] Coercion pr1isabmonoidop : isabmonoidop >-> ismonoidop.

Definition commax_is {X : UU} {opp : binop X} (is : isabmonoidop opp) : iscomm opp := pr2 is.

Expand Down Expand Up @@ -722,11 +722,11 @@ Definition make_isabgrop {X : UU} {opp : binop X} (H1 : isgrop opp) (H2 : iscomm
isabgrop opp := make_dirprod H1 H2.

Definition pr1isabgrop (X : UU) (opp : binop X) : isabgrop opp -> isgrop opp := @pr1 _ _.
Coercion pr1isabgrop : isabgrop >-> isgrop.
#[reversible] Coercion pr1isabgrop : isabgrop >-> isgrop.

Definition isabgroptoisabmonoidop (X : UU) (opp : binop X) : isabgrop opp -> isabmonoidop opp :=
λ is : _, make_dirprod (pr1 (pr1 is)) (pr2 is).
Coercion isabgroptoisabmonoidop : isabgrop >-> isabmonoidop.
#[reversible] Coercion isabgroptoisabmonoidop : isabgrop >-> isabmonoidop.

Lemma isapropisabgrop {X : hSet} (opp : binop X) : isaprop (isabgrop opp).
Proof.
Expand Down Expand Up @@ -1015,7 +1015,7 @@ Proof.
+ simpl. apply (ringmultx0_is).
- apply (ringdistraxs_is is).
Defined.
Coercion isringopstoisrigops : isringops >-> isrigops.
#[reversible] Coercion isringopstoisrigops : isringops >-> isrigops.

(** *)

Expand All @@ -1024,7 +1024,7 @@ Definition iscommrigops {X : UU} (opp1 opp2 : binop X) : UU :=

Definition pr1iscommrigops (X : UU) (opp1 opp2 : binop X) :
iscommrigops opp1 opp2 -> isrigops opp1 opp2 := @pr1 _ _.
Coercion pr1iscommrigops : iscommrigops >-> isrigops.
#[reversible] Coercion pr1iscommrigops : iscommrigops >-> isrigops.

Definition rigiscommop2_is {X : UU} {opp1 opp2 : binop X} (is : iscommrigops opp1 opp2) :
iscomm opp2 := pr2 is.
Expand All @@ -1043,7 +1043,7 @@ Definition iscommringops {X : UU} (opp1 opp2 : binop X) : UU :=

Definition pr1iscommringops (X : UU) (opp1 opp2 : binop X) :
iscommringops opp1 opp2 -> isringops opp1 opp2 := @pr1 _ _.
Coercion pr1iscommringops : iscommringops >-> isringops.
#[reversible] Coercion pr1iscommringops : iscommringops >-> isringops.

Definition ringiscommop2_is {X : UU} {opp1 opp2 : binop X} (is : iscommringops opp1 opp2) :
iscomm opp2 := pr2 is.
Expand All @@ -1058,7 +1058,7 @@ Defined.
Definition iscommringopstoiscommrigops (X : UU) (opp1 opp2 : binop X)
(is : iscommringops opp1 opp2) : iscommrigops opp1 opp2 :=
make_dirprod (isringopstoisrigops _ _ _ (pr1 is)) (pr2 is).
Coercion iscommringopstoiscommrigops : iscommringops >-> iscommrigops.
#[reversible] Coercion iscommringopstoiscommrigops : iscommringops >-> iscommrigops.

(** **** Transfer properties of binary operations relative to weak equivalences *)

Expand Down Expand Up @@ -1532,7 +1532,7 @@ Definition make_setwithbinop (X : hSet) (opp : binop X) : setwithbinop :=
tpair (λ X : hSet, binop X) X opp.

Definition pr1setwithbinop : setwithbinop -> hSet := @pr1 _ (λ X : hSet, binop X).
Coercion pr1setwithbinop : setwithbinop >-> hSet.
#[reversible] Coercion pr1setwithbinop : setwithbinop >-> hSet.

Definition op {X : setwithbinop} : binop X := pr2 X.

Expand Down Expand Up @@ -1590,7 +1590,7 @@ Definition make_binopfun {X Y : setwithbinop} (f : X -> Y) (is : isbinopfun f) :
tpair _ f is.

Definition pr1binopfun (X Y : setwithbinop) : binopfun X Y -> (X -> Y) := @pr1 _ _.
Coercion pr1binopfun : binopfun >-> Funclass.
#[reversible] Coercion pr1binopfun : binopfun >-> Funclass.

Definition binopfunisbinopfun {X Y : setwithbinop} (f : binopfun X Y) : isbinopfun f := pr2 f.

Expand Down Expand Up @@ -1623,11 +1623,11 @@ Definition make_binopmono {X Y : setwithbinop} (f : incl X Y) (is : isbinopfun f
binopmono X Y := tpair _ f is.

Definition pr1binopmono (X Y : setwithbinop) : binopmono X Y -> incl X Y := @pr1 _ _.
Coercion pr1binopmono : binopmono >-> incl.
#[reversible] Coercion pr1binopmono : binopmono >-> incl.

Definition binopincltobinopfun (X Y : setwithbinop) :
binopmono X Y -> binopfun X Y := λ f, make_binopfun (pr1 (pr1 f)) (pr2 f).
Coercion binopincltobinopfun : binopmono >-> binopfun.
#[reversible] Coercion binopincltobinopfun : binopmono >-> binopfun.

Definition binopmonocomp {X Y Z : setwithbinop} (f : binopmono X Y) (g : binopmono Y Z) :
binopmono X Z := make_binopmono (inclcomp (pr1 f) (pr1 g)) (isbinopfuncomp f g).
Expand All @@ -1638,7 +1638,7 @@ Definition make_binopiso {X Y : setwithbinop} (f : X ≃ Y) (is : isbinopfun f)
binopiso X Y := tpair _ f is.

Definition pr1binopiso (X Y : setwithbinop) : binopiso X Y -> X ≃ Y := @pr1 _ _.
Coercion pr1binopiso : binopiso >-> weq.
#[reversible] Coercion pr1binopiso : binopiso >-> weq.

Lemma isasetbinopiso (X Y : setwithbinop) : isaset (binopiso X Y).
Proof.
Expand All @@ -1652,7 +1652,7 @@ Opaque isasetbinopiso.

Definition binopisotobinopmono (X Y : setwithbinop) :
binopiso X Y -> binopmono X Y := λ f, make_binopmono (weqtoincl (pr1 f)) (pr2 f).
Coercion binopisotobinopmono : binopiso >-> binopmono.
#[reversible] Coercion binopisotobinopmono : binopiso >-> binopmono.

Definition binopisocomp {X Y Z : setwithbinop} (f : binopiso X Y) (g : binopiso Y Z) :
binopiso X Z := make_binopiso (weqcomp (pr1 f) (pr1 g)) (isbinopfuncomp f g).
Expand Down Expand Up @@ -1983,7 +1983,7 @@ Definition subsetswithbinopconstr {X : setwithbinop} :

Definition pr1subsetswithbinop (X : setwithbinop) : subsetswithbinop X -> hsubtype X :=
@pr1 _ (λ A : hsubtype X, issubsetwithbinop (@op X) A).
Coercion pr1subsetswithbinop : subsetswithbinop >-> hsubtype.
#[reversible] Coercion pr1subsetswithbinop : subsetswithbinop >-> hsubtype.

Definition pr2subsetswithbinop {X : setwithbinop} (Y : subsetswithbinop X) :
issubsetwithbinop (@op X) (pr1subsetswithbinop X Y) := pr2 Y.
Expand All @@ -2002,7 +2002,7 @@ Proof.
(A -> A -> A)).
simpl. unfold binop. apply subopp.
Defined.
Coercion carrierofasubsetwithbinop : subsetswithbinop >-> setwithbinop.
#[reversible] Coercion carrierofasubsetwithbinop : subsetswithbinop >-> setwithbinop.


(** **** Relations compatible with a binary operation and quotient objects *)
Expand Down Expand Up @@ -2071,7 +2071,7 @@ Definition make_binophrel {X : setwithbinop} :

Definition pr1binophrel (X : setwithbinop) : binophrel X -> hrel X :=
@pr1 _ (λ R : hrel X, isbinophrel R).
Coercion pr1binophrel : binophrel >-> hrel.
#[reversible] Coercion pr1binophrel : binophrel >-> hrel.

Definition binophrel_resp_left {X : setwithbinop} (R : binophrel X)
{a b : X} (c : X) (r : R a b) : R (op c a) (op c b) :=
Expand All @@ -2088,7 +2088,7 @@ Definition make_binoppo {X : setwithbinop} :
tpair (λ R : po X, isbinophrel R).

Definition pr1binoppo (X : setwithbinop) : binoppo X -> po X := @pr1 _ (λ R : po X, isbinophrel R).
Coercion pr1binoppo : binoppo >-> po.
#[reversible] Coercion pr1binoppo : binoppo >-> po.

Definition binopeqrel (X : setwithbinop) : UU := total2 (λ R : eqrel X, isbinophrel R).

Expand All @@ -2098,7 +2098,7 @@ Definition make_binopeqrel {X : setwithbinop} :

Definition pr1binopeqrel (X : setwithbinop) : binopeqrel X -> eqrel X :=
@pr1 _ (λ R : eqrel X, isbinophrel R).
Coercion pr1binopeqrel : binopeqrel >-> eqrel.
#[reversible] Coercion pr1binopeqrel : binopeqrel >-> eqrel.

Definition binopeqrel_resp_left {X : setwithbinop} (R : binopeqrel X)
{a b : X} (c : X) (r : R a b) : R (op c a) (op c b) :=
Expand Down Expand Up @@ -2439,7 +2439,7 @@ Definition make_setwith2binop (X : hSet) (opps : (binop X) × (binop X)) :

Definition pr1setwith2binop : setwith2binop -> hSet :=
@pr1 _ (λ X : hSet, (binop X) × (binop X)).
Coercion pr1setwith2binop : setwith2binop >-> hSet.
#[reversible] Coercion pr1setwith2binop : setwith2binop >-> hSet.

Definition op1 {X : setwith2binop} : binop X := pr1 (pr2 X).

Expand Down Expand Up @@ -2490,7 +2490,7 @@ Definition make_twobinopfun {X Y : setwith2binop} (f : X -> Y) (is : istwobinopf
twobinopfun X Y := tpair _ f is.

Definition pr1twobinopfun (X Y : setwith2binop) : twobinopfun X Y -> (X -> Y) := @pr1 _ _.
Coercion pr1twobinopfun : twobinopfun >-> Funclass.
#[reversible] Coercion pr1twobinopfun : twobinopfun >-> Funclass.

Definition binop1fun {X Y : setwith2binop} (f : twobinopfun X Y) :
binopfun (setwithbinop1 X) (setwithbinop1 Y) :=
Expand Down Expand Up @@ -2542,11 +2542,11 @@ Definition make_twobinopmono {X Y : setwith2binop} (f : incl X Y) (is : istwobin
twobinopmono X Y := tpair _ f is.

Definition pr1twobinopmono (X Y : setwith2binop) : twobinopmono X Y -> incl X Y := @pr1 _ _.
Coercion pr1twobinopmono : twobinopmono >-> incl.
#[reversible] Coercion pr1twobinopmono : twobinopmono >-> incl.

Definition twobinopincltotwobinopfun (X Y : setwith2binop) :
twobinopmono X Y -> twobinopfun X Y := λ f, make_twobinopfun (pr1 (pr1 f)) (pr2 f).
Coercion twobinopincltotwobinopfun : twobinopmono >-> twobinopfun.
#[reversible] Coercion twobinopincltotwobinopfun : twobinopmono >-> twobinopfun.

Definition binop1mono {X Y : setwith2binop} (f : twobinopmono X Y) :
binopmono (setwithbinop1 X) (setwithbinop1 Y) :=
Expand All @@ -2565,11 +2565,11 @@ Definition make_twobinopiso {X Y : setwith2binop} (f : X ≃ Y) (is : istwobinop
twobinopiso X Y := tpair _ f is.

Definition pr1twobinopiso (X Y : setwith2binop) : twobinopiso X Y -> X ≃ Y := @pr1 _ _.
Coercion pr1twobinopiso : twobinopiso >-> weq.
#[reversible] Coercion pr1twobinopiso : twobinopiso >-> weq.

Definition twobinopisototwobinopmono (X Y : setwith2binop) :
twobinopiso X Y -> twobinopmono X Y := λ f, make_twobinopmono (weqtoincl (pr1 f)) (pr2 f).
Coercion twobinopisototwobinopmono : twobinopiso >-> twobinopmono.
#[reversible] Coercion twobinopisototwobinopmono : twobinopiso >-> twobinopmono.

Definition twobinopisototwobinopfun {X Y : setwith2binop} (f : twobinopiso X Y) :
twobinopfun X Y := make_twobinopfun f (pr2 f).
Expand Down Expand Up @@ -2820,7 +2820,7 @@ Definition subsetswith2binopconstr {X : setwith2binop} :

Definition pr1subsetswith2binop (X : setwith2binop) : subsetswith2binop X -> hsubtype X :=
@pr1 _ (λ A : hsubtype X, issubsetwith2binop A).
Coercion pr1subsetswith2binop : subsetswith2binop >-> hsubtype.
#[reversible] Coercion pr1subsetswith2binop : subsetswith2binop >-> hsubtype.

Definition totalsubsetwith2binop (X : setwith2binop) : subsetswith2binop X.
Proof.
Expand All @@ -2840,7 +2840,7 @@ Proof.
(pr2 (pr2 A) a a')) : (A -> A -> A)).
simpl. apply (make_dirprod subopp1 subopp2).
Defined.
Coercion carrierofsubsetwith2binop : subsetswith2binop >-> setwith2binop.
#[reversible] Coercion carrierofsubsetwith2binop : subsetswith2binop >-> setwith2binop.


(** **** Quotient objects *)
Expand Down Expand Up @@ -2872,7 +2872,7 @@ Definition make_twobinophrel {X : setwith2binop} :

Definition pr1twobinophrel (X : setwith2binop) : twobinophrel X -> hrel X :=
@pr1 _ (λ R : hrel X, is2binophrel R).
Coercion pr1twobinophrel : twobinophrel >-> hrel.
#[reversible] Coercion pr1twobinophrel : twobinophrel >-> hrel.

Definition twobinoppo (X : setwith2binop) : UU := total2 (λ R : po X, is2binophrel R).

Expand All @@ -2882,7 +2882,7 @@ Definition make_twobinoppo {X : setwith2binop} :

Definition pr1twobinoppo (X : setwith2binop) : twobinoppo X -> po X :=
@pr1 _ (λ R : po X, is2binophrel R).
Coercion pr1twobinoppo : twobinoppo >-> po.
#[reversible] Coercion pr1twobinoppo : twobinoppo >-> po.

Definition twobinopeqrel (X : setwith2binop) : UU := total2 (λ R : eqrel X, is2binophrel R).

Expand All @@ -2892,7 +2892,7 @@ Definition make_twobinopeqrel {X : setwith2binop} :

Definition pr1twobinopeqrel (X : setwith2binop) : twobinopeqrel X -> eqrel X :=
@pr1 _ (λ R : eqrel X, is2binophrel R).
Coercion pr1twobinopeqrel : twobinopeqrel >-> eqrel.
#[reversible] Coercion pr1twobinopeqrel : twobinopeqrel >-> eqrel.

Definition setwith2binopquot {X : setwith2binop} (R : twobinopeqrel X) : setwith2binop.
Proof.
Expand Down
10 changes: 5 additions & 5 deletions UniMath/Algebra/ConstructiveStructures.v
Expand Up @@ -24,7 +24,7 @@ Definition ConstructiveDivisionRig :=
× isapbinop (X := (pr1 (pr1 X)) ,, R) BinaryOperations.op2
× isConstrDivRig X R.
Definition ConstructiveDivisionRig_rig : ConstructiveDivisionRig -> rig := pr1.
Coercion ConstructiveDivisionRig_rig : ConstructiveDivisionRig >-> rig.
#[reversible] Coercion ConstructiveDivisionRig_rig : ConstructiveDivisionRig >-> rig.
Definition ConstructiveDivisionRig_apsetwith2binop : ConstructiveDivisionRig -> apsetwith2binop.
Proof.
intros X.
Expand Down Expand Up @@ -231,13 +231,13 @@ Definition ConstructiveCommutativeDivisionRig :=
× isConstrDivRig X R.
Definition ConstructiveCommutativeDivisionRig_commrig :
ConstructiveCommutativeDivisionRig -> commrig := pr1.
Coercion ConstructiveCommutativeDivisionRig_commrig :
#[reversible] Coercion ConstructiveCommutativeDivisionRig_commrig :
ConstructiveCommutativeDivisionRig >-> commrig.

Definition ConstructiveCommutativeDivisionRig_ConstructiveDivisionRig :
ConstructiveCommutativeDivisionRig -> ConstructiveDivisionRig :=
λ X, (pr1 (pr1 X),,pr1 (pr2 (pr1 X))) ,, (pr2 X).
Coercion ConstructiveCommutativeDivisionRig_ConstructiveDivisionRig :
#[reversible] Coercion ConstructiveCommutativeDivisionRig_ConstructiveDivisionRig :
ConstructiveCommutativeDivisionRig >-> ConstructiveDivisionRig.

Definition CCDRap {X : ConstructiveCommutativeDivisionRig} : hrel X := λ x y : X, CDRap (X := ConstructiveCommutativeDivisionRig_ConstructiveDivisionRig X) x y.
Expand Down Expand Up @@ -432,12 +432,12 @@ Definition ConstructiveField :=
× isConstrDivRig X R.
Definition ConstructiveField_commring :
ConstructiveField -> commring := pr1.
Coercion ConstructiveField_commring :
#[reversible] Coercion ConstructiveField_commring :
ConstructiveField >-> commring.
Definition ConstructiveField_ConstructiveCommutativeDivisionRig :
ConstructiveField -> ConstructiveCommutativeDivisionRig :=
λ X, (commringtocommrig (pr1 X)) ,, (pr2 X).
Coercion ConstructiveField_ConstructiveCommutativeDivisionRig :
#[reversible] Coercion ConstructiveField_ConstructiveCommutativeDivisionRig :
ConstructiveField >-> ConstructiveCommutativeDivisionRig.

Definition CFap {X : ConstructiveField} : hrel X := λ x y : X, CCDRap (X := ConstructiveField_ConstructiveCommutativeDivisionRig X) x y.
Expand Down
4 changes: 2 additions & 2 deletions UniMath/Algebra/DivisionRig.v
Expand Up @@ -69,7 +69,7 @@ Definition isDivRig_isrdistr {X : rig} (is : isDivRig X) : isrdistr (isDivRig_pl
Definition DivRig : UU :=
∑ (X : rig), isDivRig X.
Definition pr1DivRig (F : DivRig) : hSet := pr1 F.
Coercion pr1DivRig : DivRig >-> hSet.
#[reversible] Coercion pr1DivRig : DivRig >-> hSet.

Definition zeroDivRig {F : DivRig} : F := isDivRig_zero (pr2 F).
Definition oneDivRig {F : DivRig} : F := isDivRig_one (pr2 F).
Expand Down Expand Up @@ -143,7 +143,7 @@ End DivRig_pty.
Definition CommDivRig : UU :=
∑ (X : commrig), isDivRig X.
Definition CommDivRig_DivRig (F : CommDivRig) : DivRig := commrigtorig (pr1 F) ,, pr2 F.
Coercion CommDivRig_DivRig : CommDivRig >-> DivRig.
#[reversible] Coercion CommDivRig_DivRig : CommDivRig >-> DivRig.

Section CommDivRig_pty.

Expand Down
4 changes: 2 additions & 2 deletions UniMath/Algebra/Domains_and_Fields.v
Expand Up @@ -324,7 +324,7 @@ Opaque isapropisintdom.
Definition intdom : UU := total2 (λ X : commring, isintdom X).

Definition pr1intdom : intdom -> commring := @pr1 _ _.
Coercion pr1intdom : intdom >-> commring.
#[reversible] Coercion pr1intdom : intdom >-> commring.

Definition nonzeroax (X : intdom) : neg (@paths X 1 0) := pr1 (pr2 X).

Expand Down Expand Up @@ -530,7 +530,7 @@ Proof.
apply (hinhpr (ii2 e2)).
- intro e12. apply (hinhpr (ii1 e0)).
Defined.
Coercion fldtointdom : fld >-> intdom.
#[reversible] Coercion fldtointdom : fld >-> intdom.

Definition fldchoice {X : fld} (x : X) : (multinvpair X x) ⨿ (x = 0) := pr2 (pr2 X) x.

Expand Down
4 changes: 2 additions & 2 deletions UniMath/Algebra/GaussianElimination/Auxiliary.v
Expand Up @@ -501,13 +501,13 @@ End Dual.

Section Rings_and_Fields.

Coercion multlinvpair_of_multinvpair {R : rig} (x : R)
#[reversible] Coercion multlinvpair_of_multinvpair {R : rig} (x : R)
: @multinvpair R x -> @multlinvpair R x.
Proof.
intros [y [xy yx]]. esplit; eauto.
Defined.

Coercion multrinvpair_of_multinvpair {R : rig} (x : R)
#[reversible] Coercion multrinvpair_of_multinvpair {R : rig} (x : R)
: @multinvpair R x -> @multrinvpair R x.
Proof.
intros [y [xy yx]]. esplit; eauto.
Expand Down

0 comments on commit 36cd2b9

Please sign in to comment.