aboutsummaryrefslogtreecommitdiff
path: root/test-suite/modules
diff options
context:
space:
mode:
authorJim Fehrle2020-05-28 15:25:14 -0700
committerJim Fehrle2020-05-30 11:24:24 -0700
commit044f76cf32080f0a56309544e5335e44f89725b4 (patch)
treec2fcb7bcf1d68591e1c34d786e621d54a5c1be61 /test-suite/modules
parenta102a80d886bafc75991a446d1c1ae4c04494666 (diff)
Remove info tactic, deprecated in 8.5
Diffstat (limited to 'test-suite/modules')
-rw-r--r--test-suite/modules/PO.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/test-suite/modules/PO.v b/test-suite/modules/PO.v
index 4c0ee1b5bd..767b3c1922 100644
--- a/test-suite/modules/PO.v
+++ b/test-suite/modules/PO.v
@@ -23,11 +23,11 @@ Module Pair (X: PO) (Y: PO) <: PO.
Hint Unfold le.
Lemma le_refl : forall p : T, le p p.
- info auto.
+ auto.
Qed.
Lemma le_trans : forall p1 p2 p3 : T, le p1 p2 -> le p2 p3 -> le p1 p3.
- unfold le; intuition; info eauto.
+ unfold le; intuition; eauto.
Qed.
Lemma le_antis : forall p1 p2 : T, le p1 p2 -> le p2 p1 -> p1 = p2.
@@ -39,9 +39,9 @@ Module Pair (X: PO) (Y: PO) <: PO.
enough (t0 = t2) as ->.
reflexivity.
- info auto.
+ auto.
- info auto.
+ auto.
Qed.
End Pair.
@@ -53,5 +53,5 @@ Require Nat.
Module NN := Pair Nat Nat.
Lemma zz_min : forall p : NN.T, NN.le (0, 0) p.
- info auto with arith.
+ auto with arith.
Qed.