aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authorErik Martin-Dorel2019-02-25 02:05:40 +0100
committerErik Martin-Dorel2019-04-23 12:54:43 +0200
commit0a00a122a04ed9afdaccc2dae85e61d51d5d7a89 (patch)
tree0731ca7135cbb8cd66a6ea72b8ef707266e9a481 /plugins
parent540a581a42114d7cf19b0135d7ad3702fa7cdaca (diff)
[ssr] under: Move {beta_expand, unify_helper} in the module type (qualify them)
Diffstat (limited to 'plugins')
-rw-r--r--plugins/ssr/ssreflect.v42
1 files changed, 21 insertions, 21 deletions
diff --git a/plugins/ssr/ssreflect.v b/plugins/ssr/ssreflect.v
index 7e2c1c913f..f8d761b088 100644
--- a/plugins/ssr/ssreflect.v
+++ b/plugins/ssr/ssreflect.v
@@ -528,27 +528,6 @@ Parameter under_done :
forall (T : Type) (x : T), @Under T x x.
Notation "''Under[' x ]" := (@Under _ x _)
(at level 8, format "''Under[' x ]").
-End UNDER.
-
-Module Export Under : UNDER.
-Definition Under := @eq.
-Lemma Under_from_eq (T : Type) (x y : T) :
- @Under T x y -> x = y.
-Proof. by []. Qed.
-Definition Over := Under.
-Lemma over :
- forall (T : Type) (x : T) (y : T), @Under T x y = @Over T x y.
-Proof. by []. Qed.
-Lemma over_done :
- forall (T : Type) (x : T), @Over T x x.
-Proof. by []. Qed.
-Lemma under_done :
- forall (T : Type) (x : T), @Under T x x.
-Proof. by []. Qed.
-End Under.
-
-Register Under as plugins.ssreflect.Under.
-Register Under_from_eq as plugins.ssreflect.Under_from_eq.
Ltac beta_expand c e :=
match e with
@@ -571,6 +550,27 @@ Ltac unify_helper :=
| [ |- @Under _ ?c ?e ] =>
beta_expand c e
end.
+End UNDER.
+
+Module Export Under : UNDER.
+Definition Under := @eq.
+Lemma Under_from_eq (T : Type) (x y : T) :
+ @Under T x y -> x = y.
+Proof. by []. Qed.
+Definition Over := Under.
+Lemma over :
+ forall (T : Type) (x : T) (y : T), @Under T x y = @Over T x y.
+Proof. by []. Qed.
+Lemma over_done :
+ forall (T : Type) (x : T), @Over T x x.
+Proof. by []. Qed.
+Lemma under_done :
+ forall (T : Type) (x : T), @Under T x x.
+Proof. by []. Qed.
+End Under.
+
+Register Under as plugins.ssreflect.Under.
+Register Under_from_eq as plugins.ssreflect.Under_from_eq.
Ltac over :=
solve [ apply Under.under_done