Source code on Github
{-# OPTIONS --safe --without-K #-}
module Class.HasHsType.Core where

open import Meta.Prelude

record HasHsType (A : Set ) : Set₁ where
  field HsType : Set

module _ (A : Set ) where
  mkHsType : Set  HasHsType A
  mkHsType Hs .HasHsType.HsType = Hs

  module _  i : HasHsType A  where
    HsType : Set
    HsType = i .HasHsType.HsType