use of org.apache.atlas.v1.model.typedef.AttributeDefinition in project atlas by apache.
the class AtlasStructDefStoreV1 method toAttributeDefinition.
public static AttributeDefinition toAttributeDefinition(AtlasAttribute attribute) {
final AtlasAttributeDef attrDef = attribute.getAttributeDef();
AttributeDefinition ret = new AttributeDefinition();
ret.setName(attrDef.getName());
ret.setDataTypeName(attrDef.getTypeName());
ret.setMultiplicity(getMultiplicity(attrDef));
ret.setIsComposite(attribute.isOwnedRef());
ret.setIsUnique(attrDef.getIsUnique());
ret.setIsIndexable(attrDef.getIsIndexable());
ret.setReverseAttributeName(attribute.getInverseRefAttributeName());
ret.setDescription(attrDef.getDescription());
ret.setDefaultValue(attrDef.getDefaultValue());
return ret;
}
use of org.apache.atlas.v1.model.typedef.AttributeDefinition in project atlas by apache.
the class TypeConverterUtil method toAtlasClassificationDefs.
private static List<AtlasClassificationDef> toAtlasClassificationDefs(List<TraitTypeDefinition> traitTypeDefinitions) {
List<AtlasClassificationDef> ret = new ArrayList<>();
for (TraitTypeDefinition traitType : traitTypeDefinitions) {
List<AtlasAttributeDef> attrDefs = new ArrayList<AtlasAttributeDef>();
if (CollectionUtils.isNotEmpty(traitType.getAttributeDefinitions())) {
for (AttributeDefinition attrDefinition : traitType.getAttributeDefinitions()) {
attrDefs.add(toAtlasAttributeDef(attrDefinition));
}
}
AtlasClassificationDef classifDef = new AtlasClassificationDef(traitType.getTypeName(), traitType.getTypeDescription(), traitType.getTypeVersion(), attrDefs, traitType.getSuperTypes());
ret.add(classifDef);
}
return ret;
}
use of org.apache.atlas.v1.model.typedef.AttributeDefinition in project atlas by apache.
the class TypeConverterUtil method toAtlasEntityDefs.
private static List<AtlasEntityDef> toAtlasEntityDefs(List<ClassTypeDefinition> classTypeDefinitions, AtlasTypeRegistry registry) {
List<AtlasEntityDef> ret = new ArrayList<>();
for (ClassTypeDefinition classType : classTypeDefinitions) {
List<AtlasAttributeDef> attrDefs = new ArrayList<AtlasAttributeDef>();
if (CollectionUtils.isNotEmpty(classType.getAttributeDefinitions())) {
for (AttributeDefinition oldAttr : classType.getAttributeDefinitions()) {
AtlasAttributeDef newAttr = toAtlasAttributeDef(oldAttr);
attrDefs.add(newAttr);
}
}
AtlasEntityDef entityDef = new AtlasEntityDef(classType.getTypeName(), classType.getTypeDescription(), classType.getTypeVersion(), attrDefs, classType.getSuperTypes());
ret.add(entityDef);
}
return ret;
}
use of org.apache.atlas.v1.model.typedef.AttributeDefinition in project atlas by apache.
the class TypeConverterUtil method classificationToTypesDef.
private static TypesDef classificationToTypesDef(AtlasClassificationType classificationType, AtlasTypeRegistry registry) {
String typeName = classificationType.getClassificationDef().getName();
String typeDesc = classificationType.getClassificationDef().getDescription();
String typeVersion = classificationType.getClassificationDef().getTypeVersion();
Set<String> superTypes = new HashSet<>(classificationType.getClassificationDef().getSuperTypes());
List<AttributeDefinition> attributes = getAttributes(classificationType, registry);
TraitTypeDefinition traitTypeDef = new TraitTypeDefinition(typeName, typeDesc, typeVersion, attributes, superTypes);
TypesDef ret = new TypesDef(null, null, Arrays.asList(traitTypeDef), null);
return ret;
}
use of org.apache.atlas.v1.model.typedef.AttributeDefinition in project atlas by apache.
the class AtlasClient method createTraitType.
/**
* Creates trait type with specifiedName, superTraits and attributes
* @param traitName the name of the trait type
* @param superTraits the list of super traits from which this trait type inherits attributes
* @param attributeDefinitions the list of attributes of the trait type
* @return the list of types created
* @throws AtlasServiceException
*/
public List<String> createTraitType(String traitName, Set<String> superTraits, AttributeDefinition... attributeDefinitions) throws AtlasServiceException {
TraitTypeDefinition piiTrait = TypesUtil.createTraitTypeDef(traitName, null, superTraits, Arrays.asList(attributeDefinitions));
TypesDef typesDef = new TypesDef(Collections.emptyList(), Collections.emptyList(), Collections.singletonList(piiTrait), Collections.emptyList());
LOG.debug("Creating trait type {} {}", traitName, AtlasType.toV1Json(piiTrait));
return createType(AtlasType.toV1Json(typesDef));
}
Aggregations