How to prove that a functional is injective in Agda?

Consider for example the following code: open import Relation.Binary.PropositionalEquality record Foo (A : Set) : Set where constructor foo field foo-a : A map-foo : forall {A} -> (A -> A) -> Foo A -> Foo A map-foo f (foo a) = foo (f a) map-foo-injective : forall {A} {f g : A -> A}… Read More How to prove that a functional is injective in Agda?

Configuration file for command-line options

I’d like all modules in my Agda library to be compiled with the –prop command-line option. Is there some configuration file where I can put default options for my library? >Solution : You should be able to use the flags: field in the library’s .agda-lib. The test case for the feature is precisely –prop: https://github.com/agda/agda/blob/ebf922e06c3d1e86ae3cd4cc99cbe9ac8bc5648a/test/Succeed/default-flags/lib.agda-lib… Read More Configuration file for command-line options