aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets/MSetGenTree.v
diff options
context:
space:
mode:
authorGravatar Pierre Boutillier <pierre.boutillier@pps.univ-paris-diderot.fr>2014-09-08 16:19:39 +0200
committerGravatar Pierre Boutillier <pierre.boutillier@ens-lyon.org>2014-10-01 23:24:36 +0200
commit183112fc6a5fbb7d1c6d60b9717cdb8aceda78ca (patch)
tree8ac0350e08c22893acbb3905e028aee18f86bb5b /theories/MSets/MSetGenTree.v
parentb9a6247ddc52082065b56f296c889c41167e0507 (diff)
Simpl less (so that cbn will not simpl too much)
Diffstat (limited to 'theories/MSets/MSetGenTree.v')
-rw-r--r--theories/MSets/MSetGenTree.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/MSets/MSetGenTree.v b/theories/MSets/MSetGenTree.v
index d1d9897fb..154c2384c 100644
--- a/theories/MSets/MSetGenTree.v
+++ b/theories/MSets/MSetGenTree.v
@@ -1019,7 +1019,7 @@ Lemma flatten_e_elements :
forall l x r c e,
elements l ++ flatten_e (More x r e) = elements (Node c l x r) ++ flatten_e e.
Proof.
- intros; simpl. now rewrite elements_node, app_ass.
+ intros. now rewrite elements_node, app_ass.
Qed.
Lemma cons_1 : forall s e,
@@ -1053,7 +1053,7 @@ Lemma compare_cont_Cmp : forall s1 cont e2 l,
(forall e, Cmp (cont e) l (flatten_e e)) ->
Cmp (compare_cont s1 cont e2) (elements s1 ++ l) (flatten_e e2).
Proof.
- induction s1 as [|c1 l1 Hl1 x1 r1 Hr1]; simpl; intros; auto.
+ induction s1 as [|c1 l1 Hl1 x1 r1 Hr1]; intros; auto.
rewrite elements_node, app_ass; simpl.
apply Hl1; auto. clear e2. intros [|x2 r2 e2].
simpl; auto.