Clean up trailing whitespaces and an unused definition.

This commit is contained in:
Dan Frumin 2017-08-09 18:05:58 +02:00
parent 31e08af1d1
commit 33808928db
15 changed files with 137 additions and 152 deletions

View File

@ -103,21 +103,6 @@ Section operations.
split ; apply p. split ; apply p.
Defined. Defined.
Definition map (A B : Type) (f : A -> B) : FSet A -> FSet B.
Proof.
hrecursion.
- apply .
- intro a.
apply {|f a|}.
- apply ().
- apply assoc.
- apply comm.
- apply nl.
- apply nr.
- intros.
apply idem.
Defined.
Local Ltac remove_transport Local Ltac remove_transport
:= intros ; apply path_forall ; intro Z ; rewrite transport_arrow := intros ; apply path_forall ; intro Z ; rewrite transport_arrow
; rewrite transport_const ; simpl. ; rewrite transport_const ; simpl.