aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/micromega/Env.v
diff options
context:
space:
mode:
authorGravatar fkirchne <fkirchne@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-05-28 16:40:21 +0000
committerGravatar fkirchne <fkirchne@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-05-28 16:40:21 +0000
commit4fc5ff31b342253f889db23a3b46482a4c7fa1ca (patch)
tree5f617a4a1f48dec952b0ca5674bb719b063b60ba /plugins/micromega/Env.v
parentf9261830d886bf08599921d42539d8651437303f (diff)
A little bit of cleanup, and some annotations.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13036 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/micromega/Env.v')
-rw-r--r--plugins/micromega/Env.v14
1 files changed, 4 insertions, 10 deletions
diff --git a/plugins/micromega/Env.v b/plugins/micromega/Env.v
index 231004bca..119093818 100644
--- a/plugins/micromega/Env.v
+++ b/plugins/micromega/Env.v
@@ -17,27 +17,21 @@ Require Import Coq.Arith.Max.
Require Import List.
Set Implicit Arguments.
-(* I have addded a Leaf constructor to the varmap data structure (/plugins/ring/Quote.v)
- -- this is harmless and spares a lot of Empty.
- This means smaller proof-terms.
- BTW, by dropping the polymorphism, I get small (yet noticeable) speed-up.
-*)
-
Section S.
Variable D :Type.
Definition Env := positive -> D.
- Definition jump (j:positive) (e:Env) := fun x => e (Pplus x j).
+ Definition jump (j:positive) (e:Env) := fun x => e (Pplus x j).
- Definition nth (n:positive) (e : Env ) := e n.
+ Definition nth (n:positive) (e : Env ) := e n.
- Definition hd (x:D) (e: Env) := nth xH e.
+ Definition hd (x:D) (e: Env) := nth xH e.
Definition tail (e: Env) := jump xH e.
- Lemma psucc : forall p, (match p with
+ Lemma psucc : forall p, (match p with
| xI y' => xO (Psucc y')
| xO y' => xI y'
| 1%positive => 2%positive