Skip to content

Commit

Permalink
Adapt w.r.t. coq/coq#18895.
Browse files Browse the repository at this point in the history
  • Loading branch information
ppedrot authored and andres-erbsen committed Apr 11, 2024
1 parent 2a0a2c3 commit 208894a
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/RatUtil.v
Original file line number Diff line number Diff line change
Expand Up @@ -5,11 +5,11 @@ Create HintDb rat discriminated.
Create HintDb ratsimpl discriminated.

#[global]
Hint Immediate (@reflexivity Rat eqRat _) : rat.
Hint Extern 1 => simple eapply (@reflexivity Rat eqRat _) : rat.
#[global]
Hint Immediate (@reflexivity Rat leRat _) : rat.
Hint Extern 1 => simple eapply (@reflexivity Rat leRat _) : rat.
#[global]
Hint Immediate (rat0_le_all) : rat.
Hint Immediate rat0_le_all : rat.

Lemma maxRat_same r : maxRat r r = r.
Proof. intros; cbv [maxRat]; destruct (bleRat r r) eqn:?; trivial. Qed.
Expand Down

0 comments on commit 208894a

Please sign in to comment.