GeneratorCli

gql.client.codegen.GeneratorCli$
object GeneratorCli extends CommandIOApp

Attributes

Source
GeneratorCli.scala
Graph
Supertypes
class CommandIOApp
trait IOApp
class Object
trait Matchable
class Any
Self type

Members list

Type members

Classlikes

final case class Input(schema: Path, shared: Path, queries: NonEmptyList[Query])

Attributes

Source
GeneratorCli.scala
Supertypes
trait Serializable
trait Product
trait Equals
class Object
trait Matchable
class Any
Show all
final case class Query(query: Path, output: Option[Path])

Attributes

Source
GeneratorCli.scala
Supertypes
trait Serializable
trait Product
trait Equals
class Object
trait Matchable
class Any
Show all

Value members

Concrete methods

override def main: Opts[IO[ExitCode]]

Attributes

Definition Classes
CommandIOApp
Source
GeneratorCli.scala

Inherited methods

final def main(args: Array[String]): Unit

Attributes

Inherited from:
_$2.toLowerCase())).filterNot(((_$3:String)=>_$3.contains("windows"))).flatMap[String](((_$4:String)=>List.apply[String]("USR1","INFO"))) liveFiberSnapshotSignal.foreach[Unit](((name:String)=>Signal.handle(name,((_$5: )=>IOApp.this.runtime.fiberMonitor.liveFiberSnapshot(((_$6:String)=>System.err.print(_$6))))))) }else() valrt:Runtime=Runtime.getRuntime() valcounter:AtomicInteger=newAtomicInteger(1) valioa:IO[ExitCode]=IOApp.this.run(wrapRefArray[String](args).toList) valqueue:ArrayBlockingQueue[AnyRef]=this.queue valfiber:IOFiber[ExitCode]={ val$3$:IO[ExitCode]=JvmCpuStarvationMetrics.apply().flatMap[IO[OutcomeIO[Nothing]]](((cpuStarvationMetrics:CpuStarvationMetrics)=>CpuStarvationCheck.run(IOApp.this.runtimeConfig,cpuStarvationMetrics,((metrics:CpuStarvationWarningMetrics)=>IOApp.this.onCpuStarvationWarn(metrics))).background)).surround[ExitCode](ioa)(asyncForIO) $3$.unsafeRunFiber({ if(counter.decrementAndGet().==(0))queue.clear()else() queue.put(newCancellationException("IOAppmainfiberwascanceled")) },((`t₂`:Throwable)=>{ if(counter.decrementAndGet().==(0))queue.clear()else() queue.put(`t₂`) }),((a:ExitCode)=>{ if(counter.decrementAndGet().==(0))queue.clear()else() queue.put(a) }),$3$.unsafeRunFiber$default$4)(IOApp.this.runtime) } if(isStackTracing){ IOApp.this.runtime.fiberMonitor.monitorSuspended(fiber) () }else() defhandleShutdown():Unit={ if(counter.compareAndSet(1,0)){ valcancelLatch:CountDownLatch=newCountDownLatch(1) fiber.cancel.unsafeRunAsync(((_$7:Either[Throwable,Unit])=>cancelLatch.countDown()))(IOApp.this.runtime) valtimeout:Duration=IOApp.this.runtimeConfig.shutdownHookTimeout if(timeout.isFinite){ blocking[Boolean](cancelLatch.await(timeout.length,timeout.unit)) () }elseblocking[Unit](cancelLatch.await()) }else() IOApp.this.runtime.shutdown.apply() } valhook:Thread=newThread((()=>handleShutdown())) hook.setName("io-cancel-hook") tryrt.addShutdownHook(hook)catch{ case_:IllegalStateException=> handleShutdown() } try{ vardone:Boolean=false while(done.unary_!){ valresult:Object=blocking[Object](queue.take()) resultmatch{ caseec:ExitCode=> IOApp.this.runtime.shutdown.apply() if(ec.==(ExitCode.Success))if(isForked.&&(IOApp.this.logNonDaemonThreadsEnabled))newNonDaemonThreadLogger(IOApp.this.logNonDaemonThreadsInterval).start()else()elseif(isForked)System.exit(ec.code)else() done=true casee:CancellationException=> if(isForked)System.exit(1)elsethrowe caset:Throwable=> if(NonFatal.apply(`t₃`))if(isForked){ `t₃`.printStackTrace() System.exit(1) }elsethrow`t₃`else{ `t₃`.printStackTrace() rt.halt(1) } caser:Runnable=> tryr.run()catch{ casetifNonFatal.apply(`t₄`)=> if(isForked){ `t₄`.printStackTrace() System.exit(1) }elsethrow`t₄` caset:Throwable=> `t₅`.printStackTrace() rt.halt(1) } case_=> thrownewIllegalStateException(_root_.scala.StringContext.apply("","inMainThreadqueue").s(result.getClass[Object]().getName())) } } }catch{ case_:InterruptedException=> hook.start() rt.removeShutdownHook(hook) Thread.currentThread().interrupt() } }">IOApp
Source
IOApp.scala
final override def run(args: List[String]): IO[ExitCode]

The entry point for your application. Will be called by the runtime when the process is started. If the underlying runtime supports it, any arguments passed to the process will be made available in the args parameter. The numeric value within the resulting ExitCode will be used as the exit code when the process terminates unless terminated exceptionally or by interrupt.

The entry point for your application. Will be called by the runtime when the process is started. If the underlying runtime supports it, any arguments passed to the process will be made available in the args parameter. The numeric value within the resulting ExitCode will be used as the exit code when the process terminates unless terminated exceptionally or by interrupt.

Value parameters

args

The arguments passed to the process, if supported by the underlying runtime. For example, java com.company.MyApp --foo --bar baz or node com-mycompany-fastopt.js --foo --bar baz would each result in List("--foo", "--bar", "baz").

Attributes

See also

IOApp.Simple!.run:cats\.effect\.IO[Unit]*

Definition Classes
CommandIOApp -> IOApp
Inherited from:
CommandIOApp
Source
CommandIOApp.scala

Concrete fields

val kvPairs: Opts[NonEmptyList[Input]]

Attributes

Source
GeneratorCli.scala
val validateOpt: Opts[Boolean]

Attributes

Source
GeneratorCli.scala