mirror of https://github.com/nmvdw/HITs-Examples
Clean up trailing whitespaces and an unused definition.
This commit is contained in:
parent
31e08af1d1
commit
33808928db
|
@ -103,21 +103,6 @@ Section operations.
|
|||
split ; apply p.
|
||||
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
|
||||
:= intros ; apply path_forall ; intro Z ; rewrite transport_arrow
|
||||
; rewrite transport_const ; simpl.
|
||||
|
|
Loading…
Reference in New Issue