[Agda] Question about the meaning of 'abstract'
Andreas Abel
andreas.abel at ifi.lmu.de
Fri Nov 16 00:33:53 CET 2012
If you have an abstract definition
abstract
lhs = rhs
is it ok with the meaning of `abstract' that
lhs == rhs
holds propositionally outside the abstract block. Agda currently says
yes, but would you agree with Agda?
abstract
T : Set -> Set
T A = A
see-through : ∀ {A} → T A ≡ A
see-through = refl
opaque : ∀ {A} → T A ≡ A
opaque = see-through
Cheers,
Andreas
--
Andreas Abel <>< Du bist der geliebte Mensch.
Theoretical Computer Science, University of Munich
Oettingenstr. 67, D-80538 Munich, GERMANY
andreas.abel at ifi.lmu.de
http://www2.tcs.ifi.lmu.de/~abel/
More information about the Agda
mailing list