summaryrefslogtreecommitdiff
path: root/backends/IsabelleHOL/Primitives.thy
blob: a0cc40bd1374dde7affc2850692de963daf1e476 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
theory Primitives imports
 Main
 "HOL-Library.Monad_Syntax"
begin


datatype u32 = u32 nat
datatype 'a result = Ok 'a | Err
fun u32_lt :: "u32 \<Rightarrow> u32 \<Rightarrow> bool" where
  "u32_lt (u32 a) (u32 b) = (a < b)"

definition bind :: "'a result \<Rightarrow> ('a \<Rightarrow> 'b result) \<Rightarrow> 'b result" where
 "bind m f \<equiv> (case m of Err \<Rightarrow> Err | Ok a \<Rightarrow> f a)"

adhoc_overloading Monad_Syntax.bind bind

declare bind_def[simp]

end