From 2d449a9db34d1cfaff3b698cfc5b435e00100461 Mon Sep 17 00:00:00 2001 From: Jason Gross Date: Tue, 5 Jul 2016 16:01:04 -0700 Subject: Move option_map notation up This way, it's not eaten by a section --- theories/FSets/FMapFacts.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/FSets') diff --git a/theories/FSets/FMapFacts.v b/theories/FSets/FMapFacts.v index 741ee69d3..67bb56448 100644 --- a/theories/FSets/FMapFacts.v +++ b/theories/FSets/FMapFacts.v @@ -24,6 +24,8 @@ Hint Extern 1 (Equivalence _) => constructor; congruence. Module WFacts_fun (E:DecidableType)(Import M:WSfun E). +Notation option_map := option_map (compat "8.4"). + Notation eq_dec := E.eq_dec. Definition eqb x y := if eq_dec x y then true else false. @@ -437,8 +439,6 @@ intros; do 2 rewrite mem_find_b; rewrite remove_o; unfold eqb. destruct (eq_dec x y); auto. Qed. -Notation option_map := option_map (compat "8.4"). - Lemma map_o : forall m x (f:elt->elt'), find x (map f m) = option_map f (find x m). Proof. -- cgit v1.2.3