|
| #define | bound(a, b, c) (max(a, min(b, c))) |
| |
| #define | BOX_ON_PLANE_SIDE(emins, emaxs, p) |
| |
| #define | EQUAL_EPSILON 0.001 |
| |
| #define | IS_NAN(x) (((*(int *) (char *) &x) & nanmask) == nanmask) |
| |
| #define | M_PI 3.14159265358979323846 |
| |
| #define | max(a, b) ((a) > (b) ? (a) : (b)) |
| |
| #define | min(a, b) ((a) < (b) ? (a) : (b)) |
| |
| #define | PITCH 0 |
| |
| #define | PlaneDiff(point, plane) (PlaneDist (point, plane) - (plane)->dist) |
| |
| #define | PlaneDist(point, plane) |
| |
| #define | PlaneFlip(sp, dp) |
| |
| #define | qfrandom(MAX) ((float) MAX * (rand() * (1.0 / (RAND_MAX + 1.0)))) |
| |
| #define | RINT(x) (floor ((x) + 0.5)) |
| |
| #define | ROLL 2 |
| |
| #define | YAW 1 |
| |
|
| float | anglemod (float a) |
| |
| void | AngleQuat (const vec3_t angles, quat_t q) |
| |
| void | AngleVectors (const vec3_t angles, vec3_t forward, vec3_t right, vec3_t up) |
| | Convert quake angles to basis vectors. More...
|
| |
| void | BarycentricCoords (const vec_t **points, int num_points, const vec3_t p, vec_t *lambda) |
| |
| int | BoxOnPlaneSide (const vec3_t emins, const vec3_t emaxs, struct plane_s *plane) |
| |
| int | CircumSphere (const vec3_t points[], int num_points, sphere_t *sphere) |
| |
| void | FloorDivMod (double numer, double denom, int *quotient, int *rem) |
| |
| int | GreatestCommonDivisor (int i1, int i2) |
| |
| fixed16_t | Invert24To16 (fixed16_t val) |
| |
| fixed16_t | Mul16_30 (fixed16_t multiplier, fixed16_t multiplicand) |
| |
| int | Q_log2 (int val) |
| |
| void | R_ConcatRotations (float in1[3][3], float in2[3][3], float out[3][3]) |
| |
| void | R_ConcatTransforms (float in1[3][4], float in2[3][4], float out[3][4]) |
| |
| qboolean | R_CullBox (const vec3_t mins, const vec3_t maxs) |
| |
| qboolean | R_CullSphere (const vec3_t origin, const float radius) |
| |
| void | RotatePointAroundVector (vec3_t dst, const vec3_t axis, const vec3_t point, float degrees) |
| |
| sphere_t | SmallestEnclosingBall (const vec3_t points[], int num_points) |
| |
| void | VectorVectors (const vec3_t forward, vec3_t right, vec3_t up) |
| |