Packages

o

gql

dsl

object dsl

A collection of smart-constructors and syntactic extensions for building GraphQL schemas.

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. type AbstractFields[F[_]] = NonEmptyList[(String, AbstractField[F, _])]
  2. final class FieldBuilder[F[_], I] extends AnyVal
  3. type Fields[F[_], -A] = NonEmptyList[(String, Field[F, A, _])]
  4. final case class FieldsSyntax[F[_], A](fields: Fields[F, A]) extends AnyVal with Product with Serializable
  5. final case class InterfaceSyntax[F[_], A](tpe: Interface[F, A]) extends AnyVal with Product with Serializable
  6. final case class PartiallyAppliedArgFull[A](dummy: Boolean = false) extends AnyVal with Product with Serializable
  7. final class PartiallyAppliedEff[I] extends AnyVal
  8. final class PartiallyAppliedFieldBuilder[F[_], I] extends AnyVal
  9. final class PartiallyAppliedLift[F[_], I] extends AnyVal
  10. final case class PartiallyAppliedUnion0[F[_], A](name: String) extends AnyVal with Product with Serializable
  11. final case class PartiallyAppliedUnion1[F[_], A](name: String, hd: Variant[F, A, _]) extends Product with Serializable
  12. trait ShowMissingKeys[A] extends AnyRef
  13. final case class SyntaxForBatchResolverSignature[F[_], K, V](r: Resolver[F, Set[K], Map[K, V]]) extends AnyVal with Product with Serializable
  14. final case class TypeSyntax[F[_], A](tpe: Type[F, A]) extends AnyVal with Product with Serializable
  15. final case class UnionSyntax[F[_], A](tpe: Union[F, A]) extends AnyVal with Product with Serializable

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, _])*): AbstractFields[F]
  6. def abstWith[F[_], T, A](arg: Arg[A])(implicit tpe: => Out[F, T]): AbstractField[F, T]
  7. def addPosition[F[_], A, Pos <: Position[F, A]](pos: Pos): State[SchemaState[F], Pos]
    Attributes
    protected
  8. def arg[A](name: String, default: Value[Const, Unit], description: String)(implicit tpe: => In[A]): Arg[A]
  9. def arg[A](name: String, default: Value[Const, Unit])(implicit tpe: => In[A]): Arg[A]
  10. def arg[A](name: String, description: String)(implicit tpe: => In[A]): Arg[A]
  11. def arg[A](name: String)(implicit tpe: => In[A]): Arg[A]
  12. def argFull[A]: PartiallyAppliedArgFull[A]
  13. def arged[F[_], I, A](a: Arg[A]): Resolver[F, I, A]
  14. def arrType[A](implicit tpe: => In[A]): In[Seq[A]]
  15. 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]
  16. 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]
  17. final def asInstanceOf[T0]: T0
    Definition Classes
    Any
  18. def build[F[_], I]: FieldBuilder[F, I]
  19. def builder[F[_], I]: PartiallyAppliedFieldBuilder[F, I]
  20. def clone(): AnyRef
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.CloneNotSupportedException]) @native()
  21. def directive[A](name: String, arg: Arg[A]): Directive[A]
  22. def directive(name: String): Directive[Unit]
  23. def eff[I]: PartiallyAppliedEff[I]
  24. def enumType[A](name: String, hd: (String, EnumValue[_ <: A]), tl: (String, EnumValue[_ <: A])*): Enum[A]
  25. def enumVal[A](value: A): EnumValue[A]
  26. final def eq(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  27. def equals(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef → Any
  28. def fields[F[_], A](hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): Fields[F, A]
  29. def finalize(): Unit
    Attributes
    protected[lang]
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.Throwable])
  30. final def getClass(): Class[_ <: AnyRef]
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  31. def hashCode(): Int
    Definition Classes
    AnyRef → Any
    Annotations
    @native()
  32. def input[A](name: String, fields: Arg[A]): Input[A]
  33. def interface[F[_], A](name: String, hd: (String, AbstractField[F, _]), tl: (String, AbstractField[F, _])*): Interface[F, A]
  34. def interfaceFrom[F[_], A](name: String, hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): Interface[F, A]
  35. def interfaceFromNel[F[_], A](name: String, fields: Fields[F, A]): Interface[F, A]
  36. def interfaceNel[F[_], A](name: String, fields: AbstractFields[F]): Interface[F, A]
  37. final def isInstanceOf[T0]: Boolean
    Definition Classes
    Any
  38. def lift[F[_], I]: PartiallyAppliedLift[F, I]
  39. final def ne(arg0: AnyRef): Boolean
    Definition Classes
    AnyRef
  40. final def notify(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  41. final def notifyAll(): Unit
    Definition Classes
    AnyRef
    Annotations
    @native()
  42. def onField[F[_], A](directive: Directive[A], handler: FieldHandler[F, A]): State[SchemaState[F], Field[F, A]]
  43. def onFragmentSpread[F[_], A](directive: Directive[A], handler: QueryHandler[FragmentSpread, A]): State[SchemaState[F], FragmentSpread[A]]
  44. def onInlineFragmentSpread[F[_], A](directive: Directive[A], handler: QueryHandler[InlineFragment, A]): State[SchemaState[F], InlineFragmentSpread[A]]
  45. def optType[A](implicit tpe: => In[A]): In[Option[A]]
  46. def optType[F[_], A, B](resolver: Resolver[F, A, B])(implicit tpe: => Out[F, B]): Out[F, Option[A]]
  47. final def synchronized[T0](arg0: => T0): T0
    Definition Classes
    AnyRef
  48. implicit def syntaxForBatchResolverSignature[F[_], K, V](resolver: Resolver[F, Set[K], Map[K, V]]): SyntaxForBatchResolverSignature[F, K, V]
  49. implicit def syntaxForFields[F[_], A](fields: Fields[F, A]): FieldsSyntax[F, A]
  50. implicit def syntaxForInterface[F[_], A](tpe: Interface[F, A]): InterfaceSyntax[F, A]
  51. implicit def syntaxForType[F[_], A](tpe: Type[F, A]): TypeSyntax[F, A]
  52. implicit def syntaxForUnion[F[_], A](tpe: Union[F, A]): UnionSyntax[F, A]
  53. def toString(): String
    Definition Classes
    AnyRef → Any
  54. def tpe[F[_], A](name: String, hd: (String, Field[F, A, _]), tl: (String, Field[F, A, _])*): Type[F, A]
  55. def tpeNel[F[_], A](name: String, entries: Fields[F, A]): Type[F, A]
  56. def union[F[_], A](name: String): PartiallyAppliedUnion0[F, A]
  57. final def wait(): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  58. final def wait(arg0: Long, arg1: Int): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException])
  59. final def wait(arg0: Long): Unit
    Definition Classes
    AnyRef
    Annotations
    @throws(classOf[java.lang.InterruptedException]) @native()
  60. object ShowMissingKeys
  61. object value

Inherited from AnyRef

Inherited from Any

Ungrouped