1
0
mirror of https://github.com/nmvdw/HITs-Examples synced 2025-12-13 22:03:51 +01:00

Some cleaning in notation

This commit is contained in:
Niels
2017-08-07 16:49:46 +02:00
parent 1bab2206a3
commit 1e373364b2
9 changed files with 136 additions and 137 deletions

View File

@@ -11,7 +11,7 @@ Section Length.
Opaque isIn_b.
Definition length (x: FSetC A) : nat.
Definition length (x : FSetC A) : nat.
Proof.
simple refine (FSetC_ind A _ _ _ _ _ _ x ); simpl.
- exact 0.
@@ -31,7 +31,7 @@ Section Length.
Definition length_FSet (x: FSet A) := length (FSet_to_FSetC x).
Lemma length_singleton: forall (a: A), length_FSet (L a) = 1.
Lemma length_singleton: forall (a: A), length_FSet ({|a|}) = 1.
Proof.
intro a.
cbn. reflexivity.