Datasets:

Modalities:
Text
Languages:
English
Libraries:
Datasets
License:
File size: 316 Bytes
4365a98
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
 
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
(* Author: Lars Hupel, TU München *)

subsection \<open>State monad\<close>

theory Applicative_State
imports
  Applicative
  "HOL-Library.State_Monad"
begin

applicative state for
  pure: State_Monad.return
  ap: State_Monad.ap
unfolding State_Monad.return_def State_Monad.ap_def
by (auto split: prod.splits)

end