view src/MetaDataSegment.agda @ 9:2652bc4fc17f

set src code numbers
author soto@cr.ie.u-ryukyu.ac.jp
date Tue, 15 Sep 2020 02:14:28 +0900
parents 73127e0ab57c
children
line wrap: on
line source

module subtype {l : Level} (Context : Set l) where

record DataSegment {ll : Level} (A : Set ll) : Set (l ⊔ ll) where
  field
    get : Context -> A
    set : Context -> A -> Context