Scalar

final case class Scalar[F[_], A](name: String, encoder: A => Value, decoder: Value => Either[String, A], description: Option[String]) extends OutToplevel[F, A] with InLeaf[A] with InToplevel[A]
Companion:
object
Source:
ast.scala
trait Product
trait Equals
trait InToplevel[A]
trait InLeaf[A]
trait In[A]
trait OutToplevel[F, A]
trait Toplevel[A]
trait Out[F, A]
class Object
trait Matchable
class Any

Value members

Concrete methods

def document(description: String): Scalar[F, A]
Source:
ast.scala
def eimap[B](f: A => Either[String, B])(g: B => A): Scalar[F, B]
Source:
ast.scala
override def mapK[G[_] : Functor](fk: FunctionK[F, G]): Scalar[G, A]
Definition Classes
Source:
ast.scala
def rename(newName: String): Scalar[F, A]
Source:
ast.scala

Inherited methods

Inherited from:
Product