Codota Logo
TItemDefinition.<init>
Code IndexAdd Codota to your IDE (free)

How to use
org.kie.dmn.model.v1_1.TItemDefinition
constructor

Best Java code snippets using org.kie.dmn.model.v1_1.TItemDefinition.<init> (Showing top 4 results out of 315)

  • Add the Codota plugin to your IDE and get smart completions
private void myMethod () {
List l =
  • Codota Iconnew LinkedList()
  • Codota IconCollections.emptyList()
  • Codota Iconnew ArrayList()
  • Smart code suggestions by Codota
}
origin: org.kie/kie-dmn-core

private static List<ItemDefinition> getBaseListOfItemDefinitions(final int nameIndexFrom) {
  final List<ItemDefinition> itemDefinitions = new ArrayList<>();
  for (int i = nameIndexFrom; i < NUMBER_OF_BASE_ITEM_DEFINITIONS + nameIndexFrom; i++) {
    final ItemDefinition it = new TItemDefinition();
    it.setName(ITEM_DEFINITION_NAME_BASE + i);
    itemDefinitions.add(it);
  }
  return itemDefinitions;
}
origin: org.kie/kie-dmn-core

private static ItemDefinition createItemDefinitionWithDeps(final ItemDefinition itemDefinitionTemplate,
                                 final List<ItemDefinition> dependencies,
                                 final int maxNumberOfDepsPerItemDefinition,
                                 final Set<String> usedNames) {
  // New ItemDefinition is created, so the original one stays untouched.
  final ItemDefinition it = new TItemDefinition();
  it.setName(itemDefinitionTemplate.getName());
  final List<ItemDefinition> possibleDependencies =
      dependencies.stream().filter(item -> !item.getName().equals(it.getName())).collect(Collectors.toList());
  addDepsToItemDefinition(it, possibleDependencies, maxNumberOfDepsPerItemDefinition, usedNames);
  return it;
}
origin: org.kie/kie-dmn-core

private ItemDefinition build(final String name, final ItemDefinition... components) {
  final ItemDefinition res = new TItemDefinition();
  res.setName(name);
  for ( final ItemDefinition ic : components ) {
    final ItemDefinition c = new TItemDefinition();
    c.setName("_" + name + "-" + ic.getName());
    c.setTypeRef(new QName(TEST_NS, ic.getName()));
    res.getItemComponent().add(c);
  }
  return res;
}

origin: org.kie/kie-dmn-core

private static void createAndAddDependency(final ItemDefinition itemDefinition, final ItemDefinition dependency) {
  final ItemDefinition newDependency = new TItemDefinition();
  newDependency.setName("_" + itemDefinition.getName() + "-" + dependency.getName());
  newDependency.setTypeRef(new QName(TEST_NS, dependency.getName()));
  itemDefinition.getItemComponent().add(newDependency);
}
org.kie.dmn.model.v1_1TItemDefinition<init>

Popular methods of TItemDefinition

  • getName

Popular in Java

  • Updating database using SQL prepared statement
  • putExtra (Intent)
  • compareTo (BigDecimal)
    Compares this BigDecimal with the specified BigDecimal. Two BigDecimal objects that are equal in val
  • getSharedPreferences (Context)
  • Table (com.google.common.collect)
    A collection that associates an ordered pair of keys, called a row key and a column key, with a sing
  • Font (java.awt)
    The Font class represents fonts, which are used to render text in a visible way. A font provides the
  • KeyStore (java.security)
    This class represents an in-memory collection of keys and certificates. It manages two types of entr
  • TimerTask (java.util)
    A task that can be scheduled for one-time or repeated execution by a Timer.
  • JarFile (java.util.jar)
    JarFile is used to read jar entries and their associated data from jar files.
  • Pattern (java.util.regex)
    A compiled representation of a regular expression. A regular expression, specified as a string, must
Codota Logo
  • Products

    Search for Java codeSearch for JavaScript codeEnterprise
  • IDE Plugins

    IntelliJ IDEAWebStormAndroid StudioEclipseVisual Studio CodePyCharmSublime TextPhpStormVimAtomGoLandRubyMineEmacsJupyter
  • Company

    About UsContact UsCareers
  • Resources

    FAQBlogCodota Academy Plugin user guide Terms of usePrivacy policyJava Code IndexJavascript Code Index
Get Codota for your IDE now