src/HOL/Library/Tools/lazy.hs
author desharna
Fri, 19 Sep 2025 14:01:41 +0200
changeset 83192 fba18bf9e670
parent 82379 3f875966c3e1
permissions -rw-r--r--
splitted vampire_smt in two versions: vampire_smt_dt natively handles datatypes and vampire_smt_nodt does not

{- Author: Pascal Stoop, ETH Zurich
   Author: Andreas Lochbihler, Digital Asset -}

module Lazy(Lazy, delay, force) where

newtype Lazy a = Lazy a
delay f = Lazy (f ())
force (Lazy x) = x