class SGDQN
Definition at line 34 of file SGDQN.h.
Public Member Functions |
| CSGDQN () |
| CSGDQN (float64_t C) |
| CSGDQN (float64_t C, CDotFeatures *traindat, CLabels *trainlab) |
virtual | ~CSGDQN () |
virtual EClassifierType | get_classifier_type () |
virtual bool | train (CFeatures *data=NULL) |
void | set_C (float64_t c_neg, float64_t c_pos) |
float64_t | get_C1 () |
float64_t | get_C2 () |
void | set_epochs (int32_t e) |
int32_t | get_epochs () |
void | compute_ratio (float64_t *W, float64_t *W_1, float64_t *B, float64_t *dst, int32_t dim, float64_t regularizer_lambda, float64_t loss) |
void | combine_and_clip (float64_t *Bc, float64_t *B, int32_t dim, float64_t c1, float64_t c2, float64_t v1, float64_t v2) |
void | set_loss_function (CLossFunction *loss_func) |
CLossFunction * | get_loss_function () |
virtual const char * | get_name () const |
| CLinearMachine () |
virtual | ~CLinearMachine () |
void | get_w (float64_t *&dst_w, int32_t &dst_dims) |
SGVector< float64_t > | get_w () |
void | set_w (SGVector< float64_t > src_w) |
void | set_bias (float64_t b) |
float64_t | get_bias () |
virtual bool | load (FILE *srcfile) |
virtual bool | save (FILE *dstfile) |
virtual void | set_features (CDotFeatures *feat) |
virtual CLabels * | apply () |
virtual CLabels * | apply (CFeatures *data) |
virtual float64_t | apply (int32_t vec_idx) |
| get output for example "vec_idx"
|
virtual CDotFeatures * | get_features () |
| CMachine () |
virtual | ~CMachine () |
virtual void | set_labels (CLabels *lab) |
virtual CLabels * | get_labels () |
virtual float64_t | get_label (int32_t i) |
void | set_max_train_time (float64_t t) |
float64_t | get_max_train_time () |
void | set_solver_type (ESolverType st) |
ESolverType | get_solver_type () |
virtual void | set_store_model_features (bool store_model) |
| CSGObject () |
| CSGObject (const CSGObject &orig) |
virtual | ~CSGObject () |
virtual bool | is_generic (EPrimitiveType *generic) const |
template<class T > |
void | set_generic () |
void | unset_generic () |
virtual void | print_serializable (const char *prefix="") |
virtual bool | save_serializable (CSerializableFile *file, const char *prefix="") |
virtual bool | load_serializable (CSerializableFile *file, const char *prefix="") |
void | set_global_io (SGIO *io) |
SGIO * | get_global_io () |
void | set_global_parallel (Parallel *parallel) |
Parallel * | get_global_parallel () |
void | set_global_version (Version *version) |
Version * | get_global_version () |
SGVector< char * > | get_modelsel_names () |
char * | get_modsel_param_descr (const char *param_name) |
index_t | get_modsel_param_index (const char *param_name) |