aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/Reals/DiscrR.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Reals/DiscrR.v b/theories/Reals/DiscrR.v
index 4e917ddbf..b3982dab1 100644
--- a/theories/Reals/DiscrR.v
+++ b/theories/Reals/DiscrR.v
@@ -54,5 +54,6 @@ Qed.
Recursive Tactic Definition Sup0 :=
Match Context With
+ | [ |- ``0<1`` ] -> Apply Rlt_R0_R1
| [ |- ``0<?1`` ] -> Repeat (Apply Rmult_lt_pos Orelse Apply Rplus_lt_pos; Try Apply Rlt_R0_R1 Orelse Apply Rlt_R0_R2)
| [ |- ``?1>0`` ] -> Change ``0<?1``; Sup0. \ No newline at end of file