@@ -649,192 +649,192 @@ class KernelImpl(val rootContext: core.Contexts.Context, val rootPosition: util.
649
649
def TypeTree_symbol (self : TypeTree )(implicit ctx : Context ): Symbol = self.symbol
650
650
def TypeTree_tpe (self : TypeTree )(implicit ctx : Context ): Type = self.tpe.stripTypeVar
651
651
652
- type TypeTree_Inferred = tpd.TypeTree
652
+ type Inferred = tpd.TypeTree
653
653
654
- def matchTypeTree_Inferred (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_Inferred ] = tpt match {
654
+ def matchInferred (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [Inferred ] = tpt match {
655
655
case tpt : tpd.TypeTree if ! tpt.tpe.isInstanceOf [Types .TypeBounds ] => Some (tpt)
656
656
case _ => None
657
657
}
658
658
659
- def TypeTree_Inferred_apply (tpe : Type )(implicit ctx : Context ): TypeTree_Inferred = withDefaultPos(ctx => tpd.TypeTree (tpe)(ctx))
659
+ def Inferred_apply (tpe : Type )(implicit ctx : Context ): Inferred = withDefaultPos(ctx => tpd.TypeTree (tpe)(ctx))
660
660
661
- type TypeTree_TypeIdent = tpd.Ident
661
+ type TypeIdent = tpd.Ident
662
662
663
- def matchTypeTree_TypeIdent (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_TypeIdent ] = tpt match {
663
+ def matchTypeIdent (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeIdent ] = tpt match {
664
664
case tpt : tpd.Ident if tpt.isType => Some (tpt)
665
665
case _ => None
666
666
}
667
667
668
- def TypeTree_TypeIdent_name (self : TypeTree_TypeIdent )(implicit ctx : Context ): String = self.name.toString
668
+ def TypeIdent_name (self : TypeIdent )(implicit ctx : Context ): String = self.name.toString
669
669
670
- def TypeTree_TypeIdent_copy (original : TypeTree_TypeIdent )(name : String )(implicit ctx : Context ): TypeTree_TypeIdent =
670
+ def TypeIdent_copy (original : TypeIdent )(name : String )(implicit ctx : Context ): TypeIdent =
671
671
tpd.cpy.Ident (original)(name.toTypeName)
672
672
673
- type TypeTree_TypeSelect = tpd.Select
673
+ type TypeSelect = tpd.Select
674
674
675
- def matchTypeTree_TypeSelect (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_TypeSelect ] = tpt match {
675
+ def matchTypeSelect (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeSelect ] = tpt match {
676
676
case tpt : tpd.Select if tpt.isType && tpt.qualifier.isTerm => Some (tpt)
677
677
case _ => None
678
678
}
679
679
680
- def TypeTree_TypeSelect_qualifier (self : TypeTree_TypeSelect )(implicit ctx : Context ): Term = self.qualifier
681
- def TypeTree_TypeSelect_name (self : TypeTree_TypeSelect )(implicit ctx : Context ): String = self.name.toString
680
+ def TypeSelect_qualifier (self : TypeSelect )(implicit ctx : Context ): Term = self.qualifier
681
+ def TypeSelect_name (self : TypeSelect )(implicit ctx : Context ): String = self.name.toString
682
682
683
- def TypeTree_TypeSelect_apply (qualifier : Term , name : String )(implicit ctx : Context ): TypeTree_TypeSelect =
683
+ def TypeSelect_apply (qualifier : Term , name : String )(implicit ctx : Context ): TypeSelect =
684
684
withDefaultPos(ctx => tpd.Select (qualifier, name.toTypeName)(ctx))
685
685
686
- def TypeTree_TypeSelect_copy (original : TypeTree_TypeSelect )(qualifier : Term , name : String )(implicit ctx : Context ): TypeTree_TypeSelect =
686
+ def TypeSelect_copy (original : TypeSelect )(qualifier : Term , name : String )(implicit ctx : Context ): TypeSelect =
687
687
tpd.cpy.Select (original)(qualifier, name.toTypeName)
688
688
689
689
690
- type TypeTree_Projection = tpd.Select
690
+ type Projection = tpd.Select
691
691
692
- def matchTypeTree_Projection (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_Projection ] = tpt match {
692
+ def matchProjection (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [Projection ] = tpt match {
693
693
case tpt : tpd.Select if tpt.isType && tpt.qualifier.isType => Some (tpt)
694
694
case _ => None
695
695
}
696
696
697
- def TypeTree_Projection_qualifier (self : TypeTree_Projection )(implicit ctx : Context ): TypeTree = self.qualifier
698
- def TypeTree_Projection_name (self : TypeTree_Projection )(implicit ctx : Context ): String = self.name.toString
697
+ def Projection_qualifier (self : Projection )(implicit ctx : Context ): TypeTree = self.qualifier
698
+ def Projection_name (self : Projection )(implicit ctx : Context ): String = self.name.toString
699
699
700
- def TypeTree_Projection_copy (original : TypeTree_Projection )(qualifier : TypeTree , name : String )(implicit ctx : Context ): TypeTree_Projection =
700
+ def Projection_copy (original : Projection )(qualifier : TypeTree , name : String )(implicit ctx : Context ): Projection =
701
701
tpd.cpy.Select (original)(qualifier, name.toTypeName)
702
702
703
- type TypeTree_Singleton = tpd.SingletonTypeTree
703
+ type Singleton = tpd.SingletonTypeTree
704
704
705
- def matchTypeTree_Singleton (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_Singleton ] = tpt match {
705
+ def matchSingleton (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [Singleton ] = tpt match {
706
706
case tpt : tpd.SingletonTypeTree => Some (tpt)
707
707
case _ => None
708
708
}
709
709
710
- def TypeTree_Singleton_ref (self : TypeTree_Singleton )(implicit ctx : Context ): Term = self.ref
710
+ def Singleton_ref (self : Singleton )(implicit ctx : Context ): Term = self.ref
711
711
712
- def TypeTree_Singleton_apply (ref : Term )(implicit ctx : Context ): TypeTree_Singleton =
712
+ def Singleton_apply (ref : Term )(implicit ctx : Context ): Singleton =
713
713
withDefaultPos(ctx => tpd.SingletonTypeTree (ref)(ctx))
714
714
715
- def TypeTree_Singleton_copy (original : TypeTree_Singleton )(ref : Term )(implicit ctx : Context ): TypeTree_Singleton =
715
+ def Singleton_copy (original : Singleton )(ref : Term )(implicit ctx : Context ): Singleton =
716
716
tpd.cpy.SingletonTypeTree (original)(ref)
717
717
718
- type TypeTree_Refined = tpd.RefinedTypeTree
718
+ type Refined = tpd.RefinedTypeTree
719
719
720
- def matchTypeTree_Refined (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_Refined ] = tpt match {
720
+ def matchRefined (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [Refined ] = tpt match {
721
721
case tpt : tpd.RefinedTypeTree => Some (tpt)
722
722
case _ => None
723
723
}
724
724
725
- def TypeTree_Refined_tpt (self : TypeTree_Refined )(implicit ctx : Context ): TypeTree = self.tpt
726
- def TypeTree_Refined_refinements (self : TypeTree_Refined )(implicit ctx : Context ): List [Definition ] = self.refinements
725
+ def Refined_tpt (self : Refined )(implicit ctx : Context ): TypeTree = self.tpt
726
+ def Refined_refinements (self : Refined )(implicit ctx : Context ): List [Definition ] = self.refinements
727
727
728
- def TypeTree_Refined_copy (original : TypeTree_Refined )(tpt : TypeTree , refinements : List [Definition ])(implicit ctx : Context ): TypeTree_Refined =
728
+ def Refined_copy (original : Refined )(tpt : TypeTree , refinements : List [Definition ])(implicit ctx : Context ): Refined =
729
729
tpd.cpy.RefinedTypeTree (original)(tpt, refinements)
730
730
731
- type TypeTree_Applied = tpd.AppliedTypeTree
731
+ type Applied = tpd.AppliedTypeTree
732
732
733
- def matchTypeTree_Applied (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_Applied ] = tpt match {
733
+ def matchApplied (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [Applied ] = tpt match {
734
734
case tpt : tpd.AppliedTypeTree => Some (tpt)
735
735
case _ => None
736
736
}
737
737
738
- def TypeTree_Applied_tpt (self : TypeTree_Applied )(implicit ctx : Context ): TypeTree = self.tpt
739
- def TypeTree_Applied_args (self : TypeTree_Applied )(implicit ctx : Context ): List [Tree /* TypeTree | TypeBoundsTree*/ ] = self.args
738
+ def Applied_tpt (self : Applied )(implicit ctx : Context ): TypeTree = self.tpt
739
+ def Applied_args (self : Applied )(implicit ctx : Context ): List [Tree /* TypeTree | TypeBoundsTree*/ ] = self.args
740
740
741
- def TypeTree_Applied_apply (tpt : TypeTree , args : List [Tree /* TypeTree | TypeBoundsTree*/ ])(implicit ctx : Context ): TypeTree_Applied =
741
+ def Applied_apply (tpt : TypeTree , args : List [Tree /* TypeTree | TypeBoundsTree*/ ])(implicit ctx : Context ): Applied =
742
742
withDefaultPos(ctx => tpd.AppliedTypeTree (tpt, args)(ctx))
743
743
744
- def TypeTree_Applied_copy (original : TypeTree_Applied )(tpt : TypeTree , args : List [Tree /* TypeTree | TypeBoundsTree*/ ])(implicit ctx : Context ): TypeTree_Applied =
744
+ def Applied_copy (original : Applied )(tpt : TypeTree , args : List [Tree /* TypeTree | TypeBoundsTree*/ ])(implicit ctx : Context ): Applied =
745
745
tpd.cpy.AppliedTypeTree (original)(tpt, args)
746
746
747
- type TypeTree_Annotated = tpd.Annotated
747
+ type Annotated = tpd.Annotated
748
748
749
- def matchTypeTree_Annotated (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_Annotated ] = tpt match {
749
+ def matchAnnotated (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [Annotated ] = tpt match {
750
750
case tpt : tpd.Annotated => Some (tpt)
751
751
case _ => None
752
752
}
753
753
754
- def TypeTree_Annotated_arg (self : TypeTree_Annotated )(implicit ctx : Context ): TypeTree = self.arg
755
- def TypeTree_Annotated_annotation (self : TypeTree_Annotated )(implicit ctx : Context ): Term = self.annot
754
+ def Annotated_arg (self : Annotated )(implicit ctx : Context ): TypeTree = self.arg
755
+ def Annotated_annotation (self : Annotated )(implicit ctx : Context ): Term = self.annot
756
756
757
- def TypeTree_Annotated_apply (arg : TypeTree , annotation : Term )(implicit ctx : Context ): TypeTree_Annotated =
757
+ def Annotated_apply (arg : TypeTree , annotation : Term )(implicit ctx : Context ): Annotated =
758
758
withDefaultPos(ctx => tpd.Annotated (arg, annotation)(ctx))
759
759
760
- def TypeTree_Annotated_copy (original : TypeTree_Annotated )(arg : TypeTree , annotation : Term )(implicit ctx : Context ): TypeTree_Annotated =
760
+ def Annotated_copy (original : Annotated )(arg : TypeTree , annotation : Term )(implicit ctx : Context ): Annotated =
761
761
tpd.cpy.Annotated (original)(arg, annotation)
762
762
763
- type TypeTree_MatchTypeTree = tpd.MatchTypeTree
763
+ type MatchTypeTree = tpd.MatchTypeTree
764
764
765
- def matchTypeTree_MatchTypeTree (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_MatchTypeTree ] = tpt match {
765
+ def matchMatchTypeTree (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [MatchTypeTree ] = tpt match {
766
766
case tpt : tpd.MatchTypeTree => Some (tpt)
767
767
case _ => None
768
768
}
769
769
770
- def TypeTree_MatchTypeTree_bound (self : TypeTree_MatchTypeTree )(implicit ctx : Context ): Option [TypeTree ] = if (self.bound == tpd.EmptyTree ) None else Some (self.bound)
771
- def TypeTree_MatchTypeTree_selector (self : TypeTree_MatchTypeTree )(implicit ctx : Context ): TypeTree = self.selector
772
- def TypeTree_MatchTypeTree_cases (self : TypeTree_MatchTypeTree )(implicit ctx : Context ): List [CaseDef ] = self.cases
770
+ def MatchTypeTree_bound (self : MatchTypeTree )(implicit ctx : Context ): Option [TypeTree ] = if (self.bound == tpd.EmptyTree ) None else Some (self.bound)
771
+ def MatchTypeTree_selector (self : MatchTypeTree )(implicit ctx : Context ): TypeTree = self.selector
772
+ def MatchTypeTree_cases (self : MatchTypeTree )(implicit ctx : Context ): List [CaseDef ] = self.cases
773
773
774
- def TypeTree_MatchTypeTree_apply (bound : Option [TypeTree ], selector : TypeTree , cases : List [TypeCaseDef ])(implicit ctx : Context ): TypeTree_MatchTypeTree =
774
+ def MatchTypeTree_apply (bound : Option [TypeTree ], selector : TypeTree , cases : List [TypeCaseDef ])(implicit ctx : Context ): MatchTypeTree =
775
775
withDefaultPos(ctx => tpd.MatchTypeTree (bound.getOrElse(tpd.EmptyTree ), selector, cases)(ctx))
776
776
777
- def TypeTree_MatchTypeTree_copy (original : TypeTree_MatchTypeTree )(bound : Option [TypeTree ], selector : TypeTree , cases : List [TypeCaseDef ])(implicit ctx : Context ): TypeTree_MatchTypeTree =
777
+ def MatchTypeTree_copy (original : MatchTypeTree )(bound : Option [TypeTree ], selector : TypeTree , cases : List [TypeCaseDef ])(implicit ctx : Context ): MatchTypeTree =
778
778
tpd.cpy.MatchTypeTree (original)(bound.getOrElse(tpd.EmptyTree ), selector, cases)
779
779
780
- type TypeTree_ByName = tpd.ByNameTypeTree
780
+ type ByName = tpd.ByNameTypeTree
781
781
782
- def matchTypeTree_ByName (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_ByName ] = tpt match {
782
+ def matchByName (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [ByName ] = tpt match {
783
783
case tpt : tpd.ByNameTypeTree => Some (tpt)
784
784
case _ => None
785
785
}
786
786
787
- def TypeTree_ByName_result (self : TypeTree_ByName )(implicit ctx : Context ): TypeTree = self.result
787
+ def ByName_result (self : ByName )(implicit ctx : Context ): TypeTree = self.result
788
788
789
- def TypeTree_ByName_apply (result : TypeTree )(implicit ctx : Context ): TypeTree_ByName =
789
+ def ByName_apply (result : TypeTree )(implicit ctx : Context ): ByName =
790
790
withDefaultPos(ctx => tpd.ByNameTypeTree (result)(ctx))
791
791
792
- def TypeTree_ByName_copy (original : TypeTree_ByName )(result : TypeTree )(implicit ctx : Context ): TypeTree_ByName =
792
+ def ByName_copy (original : ByName )(result : TypeTree )(implicit ctx : Context ): ByName =
793
793
tpd.cpy.ByNameTypeTree (original)(result)
794
794
795
- type TypeTree_LambdaTypeTree = tpd.LambdaTypeTree
795
+ type LambdaTypeTree = tpd.LambdaTypeTree
796
796
797
- def matchTypeTree_LambdaTypeTree (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_LambdaTypeTree ] = tpt match {
797
+ def matchLambdaTypeTree (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [LambdaTypeTree ] = tpt match {
798
798
case tpt : tpd.LambdaTypeTree => Some (tpt)
799
799
case _ => None
800
800
}
801
801
802
- def TypeTree_LambdaTypeTree_tparams (self : TypeTree_LambdaTypeTree )(implicit ctx : Context ): List [TypeDef ] = self.tparams
803
- def TypeTree_LambdaTypeTree_body (self : TypeTree_LambdaTypeTree )(implicit ctx : Context ): Tree /* TypeTree | TypeBoundsTree*/ = self.body
802
+ def Lambdatparams (self : LambdaTypeTree )(implicit ctx : Context ): List [TypeDef ] = self.tparams
803
+ def Lambdabody (self : LambdaTypeTree )(implicit ctx : Context ): Tree /* TypeTree | TypeBoundsTree*/ = self.body
804
804
805
- def TypeTree_LambdaTypeTree_apply (tparams : List [TypeDef ], body : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): TypeTree_LambdaTypeTree =
805
+ def Lambdaapply (tparams : List [TypeDef ], body : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): LambdaTypeTree =
806
806
withDefaultPos(ctx => tpd.LambdaTypeTree (tparams, body)(ctx))
807
807
808
- def TypeTree_LambdaTypeTree_copy (original : TypeTree_LambdaTypeTree )(tparams : List [TypeDef ], body : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): TypeTree_LambdaTypeTree =
808
+ def Lambdacopy (original : LambdaTypeTree )(tparams : List [TypeDef ], body : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): LambdaTypeTree =
809
809
tpd.cpy.LambdaTypeTree (original)(tparams, body)
810
810
811
- type TypeTree_TypeBind = tpd.Bind
811
+ type TypeBind = tpd.Bind
812
812
813
- def matchTypeTree_TypeBind (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_TypeBind ] = tpt match {
813
+ def matchTypeBind (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeBind ] = tpt match {
814
814
case tpt : tpd.Bind if tpt.name.isTypeName => Some (tpt)
815
815
case _ => None
816
816
}
817
817
818
- def TypeTree_TypeBind_name (self : TypeTree_TypeBind )(implicit ctx : Context ): String = self.name.toString
819
- def TypeTree_TypeBind_body (self : TypeTree_TypeBind )(implicit ctx : Context ): Tree /* TypeTree | TypeBoundsTree*/ = self.body
818
+ def TypeBind_name (self : TypeBind )(implicit ctx : Context ): String = self.name.toString
819
+ def TypeBind_body (self : TypeBind )(implicit ctx : Context ): Tree /* TypeTree | TypeBoundsTree*/ = self.body
820
820
821
- def TypeTree_TypeBind_copy (original : TypeTree_TypeBind )(name : String , tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): TypeTree_TypeBind =
821
+ def TypeBind_copy (original : TypeBind )(name : String , tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): TypeBind =
822
822
tpd.cpy.Bind (original)(name.toTypeName, tpt)
823
823
824
- type TypeTree_TypeBlock = tpd.Block
824
+ type TypeBlock = tpd.Block
825
825
826
- def matchTypeTree_TypeBlock (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeTree_TypeBlock ] = tpt match {
826
+ def matchTypeBlock (tpt : Tree /* TypeTree | TypeBoundsTree*/ )(implicit ctx : Context ): Option [TypeBlock ] = tpt match {
827
827
case tpt : tpd.Block => Some (tpt)
828
828
case _ => None
829
829
}
830
830
831
- def TypeTree_TypeBlock_aliases (self : TypeTree_TypeBlock )(implicit ctx : Context ): List [TypeDef ] = self.stats.map { case alias : TypeDef => alias }
832
- def TypeTree_TypeBlock_tpt (self : TypeTree_TypeBlock )(implicit ctx : Context ): TypeTree = self.expr
831
+ def TypeBlock_aliases (self : TypeBlock )(implicit ctx : Context ): List [TypeDef ] = self.stats.map { case alias : TypeDef => alias }
832
+ def TypeBlock_tpt (self : TypeBlock )(implicit ctx : Context ): TypeTree = self.expr
833
833
834
- def TypeTree_TypeBlock_apply (aliases : List [TypeDef ], tpt : TypeTree )(implicit ctx : Context ): TypeTree_TypeBlock =
834
+ def TypeBlock_apply (aliases : List [TypeDef ], tpt : TypeTree )(implicit ctx : Context ): TypeBlock =
835
835
withDefaultPos(ctx => tpd.Block (aliases, tpt)(ctx))
836
836
837
- def TypeTree_TypeBlock_copy (original : TypeTree_TypeBlock )(aliases : List [TypeDef ], tpt : TypeTree )(implicit ctx : Context ): TypeTree_TypeBlock =
837
+ def TypeBlock_copy (original : TypeBlock )(aliases : List [TypeDef ], tpt : TypeTree )(implicit ctx : Context ): TypeBlock =
838
838
tpd.cpy.Block (original)(aliases, tpt)
839
839
840
840
type TypeBoundsTree = tpd.TypeBoundsTree
@@ -1578,7 +1578,7 @@ class KernelImpl(val rootContext: core.Contexts.Context, val rootPosition: util.
1578
1578
def matchTypeBindSymbol (symbol : Symbol )(implicit ctx : Context ): Option [TypeBindSymbol ] =
1579
1579
if (symbol.isType && symbol.is(core.Flags .Case )) Some (symbol.asType) else None
1580
1580
1581
- def TypeBindSymbol_tree (self : TypeBindSymbol )(implicit ctx : Context ): TypeTree_TypeBind =
1581
+ def TypeBindSymbol_tree (self : TypeBindSymbol )(implicit ctx : Context ): TypeBind =
1582
1582
FromSymbol .typeBindFromSym(self)
1583
1583
1584
1584
type TermSymbol = core.Symbols .TermSymbol
0 commit comments