SHOGUN
v1.1.0
|
LinearLocalTangentSpaceAlignment converter used to construct embeddings as described in:
Zhang, T., Yang, J., Zhao, D., & Ge, X. (2007). Linear local tangent space alignment and application to face recognition. Neurocomputing, 70(7-9), 1547-1553. Retrieved from http://linkinghub.elsevier.com/retrieve/pii/S0925231206004577
This method is hardly applicable to very high-dimensional data due to necessity to solve eigenproblem involving matrix of size (dim x dim).
Definition at line 38 of file LinearLocalTangentSpaceAlignment.h.
Public Member Functions | |
CLinearLocalTangentSpaceAlignment () | |
virtual | ~CLinearLocalTangentSpaceAlignment () |
virtual const char * | get_name () const |
![]() | |
CLocalTangentSpaceAlignment () | |
virtual | ~CLocalTangentSpaceAlignment () |
![]() | |
CLocallyLinearEmbedding () | |
virtual | ~CLocallyLinearEmbedding () |
virtual CFeatures * | apply (CFeatures *features) |
void | set_k (int32_t k) |
int32_t | get_k () const |
void | set_max_k (int32_t max_k) |
int32_t | get_max_k () const |
void | set_auto_k (bool auto_k) |
bool | get_auto_k () const |
void | set_reconstruction_shift (float64_t reconstruction_shift) |
float64_t | get_reconstruction_shift () const |
void | set_nullspace_shift (float64_t nullspace_shift) |
float64_t | get_nullspace_shift () const |
void | set_use_arpack (bool use_arpack) |
bool | get_use_arpack () const |
![]() | |
CEmbeddingConverter () | |
virtual | ~CEmbeddingConverter () |
virtual CSimpleFeatures < float64_t > * | embed (CFeatures *features) |
void | set_target_dim (int32_t dim) |
int32_t | get_target_dim () const |
void | set_distance (CDistance *distance) |
CDistance * | get_distance () const |
void | set_kernel (CKernel *kernel) |
CKernel * | get_kernel () const |
![]() | |
CConverter () | |
virtual | ~CConverter () |
![]() | |
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) |
Protected Member Functions | |
virtual SGMatrix< float64_t > | construct_embedding (CFeatures *features, SGMatrix< float64_t > matrix, int dimension) |
![]() | |
virtual SGMatrix< float64_t > | construct_weight_matrix (CSimpleFeatures< float64_t > *simple_features, float64_t *W_matrix, SGMatrix< int32_t > neighborhood_matrix) |
HELPER. | |
![]() | |
void | init () |
HELPERS. | |
virtual SGMatrix< float64_t > | construct_embedding (SGMatrix< float64_t > matrix, int dimension) |
virtual SGMatrix< int32_t > | get_neighborhood_matrix (SGMatrix< float64_t > distance_matrix, int32_t k) |
int32_t | estimate_k (CSimpleFeatures< float64_t > *simple_features, SGMatrix< int32_t > neighborhood_matrix) |
float64_t | compute_reconstruction_error (int32_t k, int dim, int N, float64_t *feature_matrix, float64_t *z_matrix, float64_t *covariance_matrix, float64_t *resid_vector, float64_t *id_vector, SGMatrix< int32_t > neighborhood_matrix) |
Additional Inherited Members | |
![]() | |
SGIO * | io |
Parallel * | parallel |
Version * | version |
Parameter * | m_parameters |
Parameter * | m_model_selection_parameters |
![]() | |
static void * | run_ltsa_thread (void *p) |
THREAD. | |
![]() | |
int32_t | m_k |
FIELDS. | |
int32_t | m_max_k |
float64_t | m_reconstruction_shift |
float64_t | m_nullspace_shift |
bool | m_use_arpack |
bool | m_auto_k |
constructor
Definition at line 23 of file LinearLocalTangentSpaceAlignment.cpp.
|
virtual |
destructor
Definition at line 28 of file LinearLocalTangentSpaceAlignment.cpp.
|
protectedvirtual |
constructs embedding
simple | features to be used |
matrix | weight matrix |
dimension | dimension of embedding |
Definition at line 37 of file LinearLocalTangentSpaceAlignment.cpp.
|
virtual |
get name
Reimplemented from CLocalTangentSpaceAlignment.
Definition at line 32 of file LinearLocalTangentSpaceAlignment.cpp.