Packages

o

gql

dsl

object dsl

Source
dsl.scala
Linear Supertypes
Ordering
  1. Alphabetic
  2. By Inheritance
Inherited
  1. dsl
  2. AnyRef
  3. Any
  1. Hide All
  2. Show All
Visibility
  1. Public
  2. Protected

Type Members

  1. final class FieldBuilder[F[_], I] extends AnyVal
  2. implicit final class InterfaceSyntax[F[_], A] extends AnyVal
  3. final case class PartiallyAppliedArgFull[A](dummy: Boolean = false) extends AnyVal with Product with Serializable
  4. final class PartiallyAppliedEff[I] extends AnyVal
  5. final class PartiallyAppliedField[I] extends AnyVal
  6. final class PartiallyAppliedFieldBuilder[F[_], I] extends AnyVal
  7. final class PartiallyAppliedLift[F[_], I] extends AnyVal
  8. final case class PartiallyAppliedUnion0[F[_], A](name: String) extends AnyVal with Product with Serializable
  9. final case class PartiallyAppliedUnion1[F[_], A](name: String, hd: Variant[F, A, _]) extends Product with Serializable
  10. implicit final class TypeSyntax[F[_], A] extends AnyVal
  11. implicit final class UnionSyntax[F[_], A] extends AnyVal

Value Members

  1. final def !=(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  2. final def ##: Int
    Definition Classes
    AnyRef → Any
  3. final def ==(arg0: Any): Boolean
    Definition Classes
    AnyRef → Any
  4. def abst[F[_], T](implicit tpe: => Out[F, T]): AbstractField[F, T]
  5. def abstGroup[F[_]](hd: (String, AbstractField[F, _]), tl: (String, AbstractField[F, _])*): NonEmptyList[(String, AbstractField[F, _])]
  6. def abstWith[F[_], T, A](arg: Arg[A])(implicit tpe: => Out[F, T]): AbstractField[F, T]
  7. def arg[A](name: String, default: Value, description: String)(implicit tpe: => In[A]): Arg[A]
  8. def arg[A](name: String, default: Value)(implicit tpe: => In[A]): Arg[A]
  9. def arg[A](name: String, description: String)(implicit tpe: => In[A]): Arg[A]
  10. def arg[A](name: String)(implicit tpe: => In[A]): Arg[A]
  11. def argFull[A]: PartiallyAppliedArgFull[A]
  12. def arrType[A](implicit tpe: => In[A]): In[Seq[A]]
  13. def arrType[F[_], A, G[x] <: Seq[x], B](resolver: Resolver[F, A, B])(implicit tpe: => Out[F, B]): OutArr[F, A, G[A], B]
  14. def arrType[F[_], A, C, B](toSeq: (C) => Seq[A])(resolver: Resolver[F, A, B])(implicit tpe: => Out[F, B]): OutArr[F, A, C, B]
  15. final def asInstanceOf[T0]: T0
    Definition Classes
    Any
  16. def build[F[_], I]: PartiallyAppliedFieldBuilder[F, I]
  17. def builder[F[_], I]: FieldBuilder[F, I]
  18. def clone(): AnyRef
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.CloneNotSupportedException]) @native()
  19. def eff[I]: PartiallyAppliedEff[I]
  20. def enumType[F[_], A](name: String, hd: (String, EnumValue[_ <: A]), tl: (String, EnumValue[_ <: A])*): Enum[F, A]
  21. def enumVal[A](value: A): EnumValue[A]
  22. final def eq(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  23. def equals(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef → Any
  24. def field[I]: PartiallyAppliedField[I]
  25. def fields[F[_], A](hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): NonEmptyList[(String, Field[F, A, _])]
  26. def fields[F[_], A, B](f: (B) => A)(hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): NonEmptyList[(String, Field[F, B, _])]
  27. def finalize(): Unit
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.Throwable])
  28. final def getClass(): Class[_ <: AnyRef]
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  29. def hashCode(): Int
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  30. def input[A](name: String, fields: Arg[A]): Input[A]
  31. def interface[F[_], A](name: String, hd: (String, AbstractField[F, _]), tl: (String, AbstractField[F, _])*): Interface[F, A]
  32. def interfaceFrom[F[_], A](name: String, hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): Interface[F, A]
  33. def interfaceFromNel[F[_], A](name: String, fields: NonEmptyList[(String, Field[F, A, _])]): Interface[F, A]
  34. def interfaceNel[F[_], A](name: String, fields: NonEmptyList[(String, AbstractField[F, _])]): Interface[F, A]
  35. final def isInstanceOf[T0]: Boolean
    Definition Classes
    Any
  36. def lift[F[_], I]: PartiallyAppliedLift[F, I]
  37. final def ne(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  38. final def notify(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  39. final def notifyAll(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  40. def optType[A](implicit tpe: => In[A]): In[Option[A]]
  41. def optType[F[_], A, B](resolver: Resolver[F, A, B])(implicit tpe: => Out[F, B]): Out[F, Option[A]]
  42. final def synchronized[T0](arg0: => T0): T0
    Definition Classes
    AnyRef
  43. def toString(): String
    Definition Classes
    AnyRef → Any
  44. def tpe[F[_], A](name: String, hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): Type[F, A]
  45. def tpeNel[F[_], A](name: String, entries: NonEmptyList[(String, Field[F, A, _])]): Type[F, A]
  46. def union[F[_], A](name: String): PartiallyAppliedUnion0[F, A]
  47. final def wait(): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  48. final def wait(arg0: Long, arg1: Int): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  49. final def wait(arg0: Long): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException]) @native()
  50. object value

Inherited from AnyRef

Inherited from Any

Ungrouped