diff options
author | Helmut Grohne <grohne@cs.uni-bonn.de> | 2014-02-17 10:30:43 +0100 |
---|---|---|
committer | Helmut Grohne <grohne@cs.uni-bonn.de> | 2014-02-17 10:30:43 +0100 |
commit | 248dc87e7c282a56bcc13fc28701a572288bc3ec (patch) | |
tree | ed2cfd816af4eac83063041d92441d364b4ab639 /Bidir.agda | |
parent | f4e7869c1d203fcf406b01e34d6276adf49fb79a (diff) | |
download | bidiragda-248dc87e7c282a56bcc13fc28701a572288bc3ec.tar.gz |
avoid useless repetition
Diffstat (limited to 'Bidir.agda')
-rw-r--r-- | Bidir.agda | 2 |
1 files changed, 1 insertions, 1 deletions
@@ -248,4 +248,4 @@ theorem-2 G n s v u p | h′ , ph′ | h , ph = drop-just (begin⟨ MaybeSetoid g′ = delete-many (get s′) g t = enumeratel n h↦h′ = flip union (reshape g′ n) - h′↦r = flip mapMV (enumeratel n) ∘ flip lookupM + h′↦r = flip mapMV t ∘ flip lookupM |