Abstract
This entry provides a package for registering applicative functors and two proof methods for lifting of equations over applicative functors. The first method normalises applicative expressions according to the laws of applicative functors. This way, equations whose two sides contain the same list of variables can be lifted to every applicative functor.
To lift larger classes of equations, the second method exploits a number of additional properties (e.g., commutativity of effects) provided the properties have been declared for the concrete applicative functor at hand upon registration.
We declare several types from the Isabelle library as applicative functors and illustrate the use of the methods with two examples: the lifting of the arithmetic type class hierarchy to streams and the verification of a relabelling function on binary trees. We also formalise and verify the normalisation algorithm used by the first proof method.
License
History
- June 10, 2016
- implemented automatic derivation of lifted combinator reductions;
support arbitrary lifted relations using relators;
improved compatibility with locale interpretation
(revision ec336f354f37)
- March 3, 2016
- added formalisation of lifting with combinators
Topics
Session Applicative_Lifting
- Applicative
- Applicative_Environment
- Applicative_Option
- Applicative_Sum
- Applicative_Set
- Applicative_List
- Applicative_DNEList
- Applicative_Monoid
- Applicative_Filter
- Applicative_State
- Applicative_Stream
- Applicative_Open_State
- Applicative_PMF
- Applicative_Probability_List
- Applicative_Star
- Applicative_Vector
- Applicative_Functor
- Applicative_Environment_Algebra
- Stream_Algebra
- Tree_Relabelling
- Applicative_Examples
- Joinable
- Beta_Eta
- Combinators
- Idiomatic_Terms
- Abstract_AF
- Applicative_Test