Skip to content

Commit

Permalink
Merge pull request #78 from JasonGross/fix-for-more-rapply-10760
Browse files Browse the repository at this point in the history
Fix for a new rapply tactic
  • Loading branch information
spitters authored Oct 16, 2023
2 parents fbb6ebe + 975c458 commit 83822de
Show file tree
Hide file tree
Showing 3 changed files with 9 additions and 9 deletions.
2 changes: 1 addition & 1 deletion implementations/nonneg_semiring_elements.v
Original file line number Diff line number Diff line change
Expand Up @@ -62,7 +62,7 @@ Proof. split. trivial. apply _. Qed.

(* Misc *)
Global Instance NonNeg_trivial_apart `{!TrivialApart R} : TrivialApart (R⁺).
Proof. intros x y. now rapply trivial_apart. Qed.
Proof. intros x y. now Tactics.rapply trivial_apart. Qed.

Global Instance NonNeg_equiv_dec `{∀ x y : R, Decision (x = y)} : ∀ x y: R⁺, Decision (x = y)
:= λ x y, decide_rel (=) ('x : R) ('y : R).
Expand Down
8 changes: 4 additions & 4 deletions implementations/semiring_pairs.v
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,7 @@ Global Instance SRpair_equiv : Equiv (SRpair SR) | 4 := λ x y, pos x + neg y =
Global Instance SRpair_apart `{Apart SR} : Apart (SRpair SR) := λ x y, pos x + neg y ≶ pos y + neg x.

Global Instance SRpair_trivial_apart `{!TrivialApart SR} : TrivialApart (SRpair SR).
Proof. intros x y. now rapply trivial_apart. Qed.
Proof. intros x y. now Tactics.rapply trivial_apart. Qed.

Instance: Setoid (SRpair SR).
Proof.
Expand Down Expand Up @@ -256,7 +256,7 @@ Section with_full_pseudo_semiring_order.
setoid_replace (zp + yn + xn) with (zp + xn + yn) by ring.
setoid_replace (yp + zn + xn) with (zn + (yp + xn)) by ring.
eassumption.
intros [??] [??]. now rapply tight_apart.
intros [??] [??]. now Tactics.rapply tight_apart.
Qed.

Instance: FullPseudoOrder SRpair_le SRpair_lt.
Expand All @@ -273,8 +273,8 @@ Section with_full_pseudo_semiring_order.
setoid_replace (zp + yn + xn) with (zp + xn + yn) by ring.
setoid_replace (yp + zn + xn) with (zn + (yp + xn)) by ring.
eassumption.
intros [??] [??]. now rapply apart_iff_total_lt.
intros [??] [??]. now rapply le_iff_not_lt_flip.
intros [??] [??]. now Tactics.rapply apart_iff_total_lt.
intros [??] [??]. now Tactics.rapply le_iff_not_lt_flip.
Qed.

Instance: ∀ z : SRpair SR, StrongSetoid_Morphism (z *.).
Expand Down
8 changes: 4 additions & 4 deletions theory/ring_congruence.v
Original file line number Diff line number Diff line change
Expand Up @@ -50,16 +50,16 @@ Section quotient_ring.
Qed.

Instance: Proper ((=) ==> (=) ==> (=)) quotient_plus.
Proof. intros [?] [?] E1 [?] [?] E2. now rapply ring_congr_plus. Qed.
Proof. intros [?] [?] E1 [?] [?] E2. now Tactics.rapply ring_congr_plus. Qed.

Instance: Proper ((=) ==> (=) ==> (=)) quotient_mult.
Proof. intros [?] [?] E1 [?] [?] E2. now rapply ring_congr_mult. Qed.
Proof. intros [?] [?] E1 [?] [?] E2. now Tactics.rapply ring_congr_mult. Qed.

Instance: Proper ((=) ==> (=)) quotient_negate.
Proof. intros [?] [?] E. now rapply ring_congr_negate. Qed.
Proof. intros [?] [?] E. now Tactics.rapply ring_congr_negate. Qed.

Global Instance: Setoid_Morphism quotient_inject.
Proof. split; try apply _. intros ?? E. now rapply ring_congr_subrelation. Qed.
Proof. split; try apply _. intros ?? E. now Tactics.rapply ring_congr_subrelation. Qed.

Global Instance: Ring (Quotient A R).
Proof.
Expand Down

0 comments on commit 83822de

Please sign in to comment.