(* Title: Imperative_HOL_Time/Heap_Time_Monad.thy Author: Maximilian P. L. Haslbeck & Bohua Zhan, TU Muenchen *) section ‹A monad with a polymorphic heap and time and primitive reasoning infrastructure› text ‹This theory is an adapted version of ‹Imperative_HOL/Heap_Monad›, where the heap is extended by time bookkeeping.› theory Heap_Time_Monad imports "HOL-Imperative_HOL.Heap" "HOL-Library.Monad_Syntax" begin subsection ‹The monad› subsubsection ‹Monad construction› text ‹Monadic heap actions either produce values and transform the heap, or fail›