2001-02-19 21:15:25 +00:00
|
|
|
/*
|
|
|
|
mathlib.c
|
|
|
|
|
|
|
|
math primitives
|
|
|
|
|
|
|
|
Copyright (C) 1996-1997 Id Software, Inc.
|
|
|
|
|
|
|
|
This program is free software; you can redistribute it and/or
|
|
|
|
modify it under the terms of the GNU General Public License
|
|
|
|
as published by the Free Software Foundation; either version 2
|
|
|
|
of the License, or (at your option) any later version.
|
|
|
|
|
|
|
|
This program is distributed in the hope that it will be useful,
|
|
|
|
but WITHOUT ANY WARRANTY; without even the implied warranty of
|
|
|
|
MERCHANTABILITY or FITNESS FOR A PARTICULAR PURPOSE.
|
|
|
|
|
|
|
|
See the GNU General Public License for more details.
|
|
|
|
|
|
|
|
You should have received a copy of the GNU General Public License
|
|
|
|
along with this program; if not, write to:
|
|
|
|
|
|
|
|
Free Software Foundation, Inc.
|
|
|
|
59 Temple Place - Suite 330
|
|
|
|
Boston, MA 02111-1307, USA
|
|
|
|
|
|
|
|
*/
|
|
|
|
#ifdef HAVE_CONFIG_H
|
|
|
|
# include "config.h"
|
|
|
|
#endif
|
2003-01-15 15:31:36 +00:00
|
|
|
|
2001-02-19 21:15:25 +00:00
|
|
|
#ifdef HAVE_STRING_H
|
|
|
|
# include <string.h>
|
|
|
|
#endif
|
|
|
|
#ifdef HAVE_STRINGS_H
|
|
|
|
# include <strings.h>
|
|
|
|
#endif
|
|
|
|
|
|
|
|
#include <math.h>
|
|
|
|
|
2002-08-23 20:46:19 +00:00
|
|
|
#define IMPLEMENT_R_Cull
|
2003-08-11 06:05:07 +00:00
|
|
|
#define IMPLEMENT_VectorNormalize
|
2001-05-07 04:08:34 +00:00
|
|
|
|
2001-03-27 20:33:07 +00:00
|
|
|
#include "QF/mathlib.h"
|
|
|
|
#include "QF/qtypes.h"
|
|
|
|
#include "QF/sys.h"
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE int nanmask = 255 << 23;
|
2011-11-14 02:18:22 +00:00
|
|
|
static plane_t _frustum[4];
|
|
|
|
VISIBLE plane_t *const frustum = _frustum;
|
2004-01-21 00:15:35 +00:00
|
|
|
static vec3_t _vec3_origin = { 0, 0, 0 };
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE const vec_t * const vec3_origin = _vec3_origin;
|
2011-01-10 23:41:40 +00:00
|
|
|
static vec3_t _quat_origin = { 0, 0, 0 };
|
|
|
|
VISIBLE const vec_t * const quat_origin = _quat_origin;
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2001-09-10 04:20:27 +00:00
|
|
|
#define DEG2RAD(a) (a * (M_PI / 180.0))
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2012-04-26 11:55:11 +00:00
|
|
|
#define FMANTBITS 23
|
|
|
|
#define FMANTMASK ((1 << FMANTBITS) - 1)
|
|
|
|
#define FEXPBITS 8
|
|
|
|
#define FEXPMASK ((1 << FEXPBITS) - 1)
|
|
|
|
#define FBIAS (1 << (FEXPBITS - 1))
|
|
|
|
#define FEXPMAX ((1 << FEXPBITS) - 1)
|
|
|
|
|
|
|
|
#define HMANTBITS 10
|
|
|
|
#define HMANTMASK ((1 << HMANTBITS) - 1)
|
|
|
|
#define HEXPBITS 5
|
|
|
|
#define HEXPMASK ((1 << HEXPBITS) - 1)
|
|
|
|
#define HBIAS (1 << (HEXPBITS - 1))
|
|
|
|
#define HEXPMAX ((1 << HEXPBITS) - 1)
|
|
|
|
|
|
|
|
int16_t
|
|
|
|
FloatToHalf (float x)
|
|
|
|
{
|
|
|
|
union {
|
|
|
|
float f;
|
|
|
|
uint32_t u;
|
|
|
|
} uf;
|
|
|
|
unsigned sign;
|
|
|
|
int exp;
|
|
|
|
unsigned mant;
|
|
|
|
int16_t half;
|
|
|
|
|
|
|
|
uf.f = x;
|
|
|
|
sign = (uf.u >> (FEXPBITS + FMANTBITS)) & 1;
|
|
|
|
exp = ((uf.u >> FMANTBITS) & FEXPMASK) - FBIAS + HBIAS;
|
|
|
|
mant = (uf.u & FMANTMASK) >> (FMANTBITS - HMANTBITS);
|
|
|
|
if (exp <= 0) {
|
|
|
|
mant |= 1 << HMANTBITS;
|
|
|
|
mant >>= min (1 - exp, HMANTBITS + 1);
|
|
|
|
exp = 0;
|
|
|
|
} else if (exp >= HEXPMAX) {
|
|
|
|
mant = 0;
|
|
|
|
exp = HEXPMAX;
|
|
|
|
}
|
|
|
|
half = (sign << (HEXPBITS + HMANTBITS)) | (exp << HMANTBITS) | mant;
|
|
|
|
return half;
|
|
|
|
}
|
|
|
|
|
|
|
|
float
|
|
|
|
HalfToFloat (int16_t x)
|
|
|
|
{
|
|
|
|
union {
|
|
|
|
float f;
|
|
|
|
uint32_t u;
|
|
|
|
} uf;
|
|
|
|
unsigned sign;
|
|
|
|
int exp;
|
|
|
|
unsigned mant;
|
|
|
|
|
|
|
|
sign = (x >> (HEXPBITS + HMANTBITS)) & 1;
|
|
|
|
exp = ((x >> HMANTBITS) & HEXPMASK);
|
|
|
|
mant = (x & HMANTMASK) << (FMANTBITS - HMANTBITS);
|
|
|
|
|
|
|
|
if (exp == 0) {
|
|
|
|
if (mant) {
|
|
|
|
while (mant < (1 << FMANTBITS)) {
|
|
|
|
mant <<= 1;
|
|
|
|
exp--;
|
|
|
|
}
|
|
|
|
mant &= (1 << FMANTBITS) - 1;
|
|
|
|
exp += FBIAS - HBIAS + 1;
|
|
|
|
}
|
|
|
|
} else if (exp == HEXPMAX) {
|
|
|
|
exp = FEXPMAX;
|
|
|
|
} else {
|
|
|
|
exp += FBIAS - HBIAS;
|
|
|
|
}
|
|
|
|
uf.u = (sign << (FEXPBITS + FMANTBITS)) | (exp << FMANTBITS) | mant;
|
|
|
|
return uf.f;
|
|
|
|
}
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2003-01-06 18:28:13 +00:00
|
|
|
static void
|
2001-02-19 21:15:25 +00:00
|
|
|
ProjectPointOnPlane (vec3_t dst, const vec3_t p, const vec3_t normal)
|
|
|
|
{
|
2001-09-10 04:20:27 +00:00
|
|
|
float inv_denom, d;
|
|
|
|
vec3_t n;
|
2001-02-19 21:15:25 +00:00
|
|
|
|
|
|
|
inv_denom = 1.0F / DotProduct (normal, normal);
|
|
|
|
|
|
|
|
d = DotProduct (normal, p) * inv_denom;
|
|
|
|
|
2002-01-12 04:34:53 +00:00
|
|
|
VectorScale (normal, inv_denom * d, n);
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2002-01-12 04:34:53 +00:00
|
|
|
VectorSubtract (p, n, dst);
|
2001-02-19 21:15:25 +00:00
|
|
|
}
|
|
|
|
|
2001-10-30 19:55:34 +00:00
|
|
|
// assumes "src" is normalized
|
2003-01-06 18:28:13 +00:00
|
|
|
static void
|
2001-02-19 21:15:25 +00:00
|
|
|
PerpendicularVector (vec3_t dst, const vec3_t src)
|
|
|
|
{
|
2001-09-10 04:20:27 +00:00
|
|
|
int pos, i;
|
|
|
|
float minelem = 1.0F;
|
|
|
|
vec3_t tempvec;
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
/* find the smallest magnitude axially aligned vector */
|
2001-02-19 21:15:25 +00:00
|
|
|
for (pos = 0, i = 0; i < 3; i++) {
|
|
|
|
if (fabs (src[i]) < minelem) {
|
|
|
|
pos = i;
|
|
|
|
minelem = fabs (src[i]);
|
|
|
|
}
|
|
|
|
}
|
2002-01-12 04:34:53 +00:00
|
|
|
VectorZero (tempvec);
|
2001-02-19 21:15:25 +00:00
|
|
|
tempvec[pos] = 1.0F;
|
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
/* project the point onto the plane defined by src */
|
2001-02-19 21:15:25 +00:00
|
|
|
ProjectPointOnPlane (dst, tempvec, src);
|
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
/* normalize the result */
|
2001-02-19 21:15:25 +00:00
|
|
|
VectorNormalize (dst);
|
|
|
|
}
|
|
|
|
|
|
|
|
#if defined(_WIN32) && !defined(__GNUC__)
|
2001-08-22 22:03:16 +00:00
|
|
|
# pragma optimize( "", off )
|
2001-02-19 21:15:25 +00:00
|
|
|
#endif
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2001-10-30 19:55:34 +00:00
|
|
|
VectorVectors(const vec3_t forward, vec3_t right, vec3_t up)
|
2001-04-06 18:37:23 +00:00
|
|
|
{
|
|
|
|
float d;
|
|
|
|
|
|
|
|
right[0] = forward[2];
|
|
|
|
right[1] = -forward[0];
|
|
|
|
right[2] = forward[1];
|
|
|
|
|
2003-08-08 15:25:53 +00:00
|
|
|
d = DotProduct(forward, right);
|
|
|
|
VectorMultSub (right, d, forward, right);
|
2001-10-30 19:55:34 +00:00
|
|
|
VectorNormalize (right);
|
2001-04-06 18:37:23 +00:00
|
|
|
CrossProduct(right, forward, up);
|
|
|
|
}
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-06-26 22:20:12 +00:00
|
|
|
RotatePointAroundVector (vec3_t dst, const vec3_t axis, const vec3_t point,
|
2001-02-19 21:15:25 +00:00
|
|
|
float degrees)
|
|
|
|
{
|
|
|
|
float m[3][3];
|
|
|
|
float im[3][3];
|
|
|
|
float zrot[3][3];
|
|
|
|
float tmpmat[3][3];
|
|
|
|
float rot[3][3];
|
|
|
|
int i;
|
|
|
|
vec3_t vr, vup, vf;
|
|
|
|
|
2002-06-26 22:20:12 +00:00
|
|
|
VectorCopy (axis, vf);
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2002-06-26 22:20:12 +00:00
|
|
|
PerpendicularVector (vr, axis);
|
2001-02-19 21:15:25 +00:00
|
|
|
CrossProduct (vr, vf, vup);
|
|
|
|
|
|
|
|
m[0][0] = vr[0];
|
|
|
|
m[1][0] = vr[1];
|
|
|
|
m[2][0] = vr[2];
|
|
|
|
|
|
|
|
m[0][1] = vup[0];
|
|
|
|
m[1][1] = vup[1];
|
|
|
|
m[2][1] = vup[2];
|
|
|
|
|
|
|
|
m[0][2] = vf[0];
|
|
|
|
m[1][2] = vf[1];
|
|
|
|
m[2][2] = vf[2];
|
|
|
|
|
|
|
|
memcpy (im, m, sizeof (im));
|
|
|
|
|
|
|
|
im[0][1] = m[1][0];
|
|
|
|
im[0][2] = m[2][0];
|
|
|
|
im[1][0] = m[0][1];
|
|
|
|
im[1][2] = m[2][1];
|
|
|
|
im[2][0] = m[0][2];
|
|
|
|
im[2][1] = m[1][2];
|
|
|
|
|
|
|
|
memset (zrot, 0, sizeof (zrot));
|
|
|
|
zrot[0][0] = zrot[1][1] = zrot[2][2] = 1.0F;
|
|
|
|
|
|
|
|
zrot[0][0] = cos (DEG2RAD (degrees));
|
|
|
|
zrot[0][1] = sin (DEG2RAD (degrees));
|
|
|
|
zrot[1][0] = -sin (DEG2RAD (degrees));
|
|
|
|
zrot[1][1] = cos (DEG2RAD (degrees));
|
|
|
|
|
|
|
|
R_ConcatRotations (m, zrot, tmpmat);
|
|
|
|
R_ConcatRotations (tmpmat, im, rot);
|
|
|
|
|
|
|
|
for (i = 0; i < 3; i++) {
|
2002-01-12 04:34:53 +00:00
|
|
|
dst[i] = DotProduct (rot[i], point);
|
2001-02-19 21:15:25 +00:00
|
|
|
}
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2011-01-18 13:22:18 +00:00
|
|
|
QuatMult (const quat_t q1, const quat_t q2, quat_t out)
|
2004-04-07 18:01:45 +00:00
|
|
|
{
|
|
|
|
vec_t s;
|
|
|
|
vec3_t v;
|
|
|
|
|
2011-01-18 13:22:18 +00:00
|
|
|
s = q1[0] * q2[0] - DotProduct (q1 + 1, q2 + 1);
|
|
|
|
CrossProduct (q1 + 1, q2 + 1, v);
|
|
|
|
VectorMultAdd (v, q1[0], q2 + 1, v);
|
|
|
|
VectorMultAdd (v, q2[0], q1 + 1, out + 1);
|
2004-04-08 05:13:24 +00:00
|
|
|
out[0] = s;
|
2004-04-07 18:01:45 +00:00
|
|
|
}
|
|
|
|
|
2012-04-26 00:24:05 +00:00
|
|
|
VISIBLE void
|
|
|
|
QuatMultVec (const quat_t q, const vec3_t v, vec3_t out)
|
|
|
|
{
|
|
|
|
vec_t s;
|
|
|
|
vec3_t tv;
|
|
|
|
|
|
|
|
s = -DotProduct (q + 1, v);
|
|
|
|
CrossProduct (q + 1, v, tv);
|
|
|
|
VectorMultAdd (tv, q[0], v, tv);
|
|
|
|
CrossProduct (q + 1, tv, out);
|
|
|
|
VectorMultSub (out, s, q + 1, out);
|
|
|
|
VectorMultAdd (out, q[0], tv, out);
|
|
|
|
}
|
|
|
|
|
2011-01-18 13:22:18 +00:00
|
|
|
VISIBLE void
|
|
|
|
QuatInverse (const quat_t in, quat_t out)
|
|
|
|
{
|
|
|
|
quat_t q;
|
|
|
|
vec_t m;
|
|
|
|
|
|
|
|
m = QDotProduct (in, in); // in * in*
|
|
|
|
QuatConj (in, q);
|
|
|
|
QuatScale (q, 1 / m, out);
|
|
|
|
}
|
|
|
|
|
2012-01-12 12:22:06 +00:00
|
|
|
VISIBLE void
|
|
|
|
QuatExp (const quat_t a, quat_t b)
|
|
|
|
{
|
|
|
|
vec3_t n;
|
|
|
|
vec_t th;
|
|
|
|
vec_t r;
|
|
|
|
vec_t c, s;
|
|
|
|
|
|
|
|
VectorCopy (a + 1, n);
|
|
|
|
th = VectorNormalize (n);
|
|
|
|
r = expf (a[0]);
|
|
|
|
c = cosf (th);
|
|
|
|
s = sinf (th);
|
|
|
|
VectorScale (n, r * s, b + 1);
|
|
|
|
b[0] = r * c;
|
|
|
|
}
|
|
|
|
|
2010-10-18 14:27:42 +00:00
|
|
|
VISIBLE void
|
|
|
|
QuatToMatrix (const quat_t q, vec_t *m, int homogenous, int vertical)
|
|
|
|
{
|
|
|
|
vec_t aa, ab, ac, ad, bb, bc, bd, cc, cd, dd;
|
|
|
|
vec_t *_m[4] = {
|
2010-10-19 14:41:57 +00:00
|
|
|
m + (homogenous ? 0 : 0),
|
|
|
|
m + (homogenous ? 4 : 3),
|
|
|
|
m + (homogenous ? 8 : 6),
|
|
|
|
m + (homogenous ? 12 : 9),
|
2010-10-18 14:27:42 +00:00
|
|
|
};
|
|
|
|
|
|
|
|
aa = q[0] * q[0];
|
|
|
|
ab = q[0] * q[1];
|
|
|
|
ac = q[0] * q[2];
|
|
|
|
ad = q[0] * q[3];
|
|
|
|
|
|
|
|
bb = q[1] * q[1];
|
|
|
|
bc = q[1] * q[2];
|
|
|
|
bd = q[1] * q[3];
|
|
|
|
|
|
|
|
cc = q[2] * q[2];
|
|
|
|
cd = q[2] * q[3];
|
|
|
|
|
|
|
|
dd = q[3] * q[3];
|
|
|
|
|
|
|
|
if (vertical) {
|
|
|
|
VectorSet (aa + bb - cc - dd, 2 * (bc + ad), 2 * (bd - ac), _m[0]);
|
|
|
|
VectorSet (2 * (bc - ad), aa - bb + cc - dd, 2 * (cd + ab), _m[1]);
|
|
|
|
VectorSet (2 * (bd + ac), 2 * (cd - ab), aa - bb - cc + dd, _m[2]);
|
|
|
|
} else {
|
|
|
|
VectorSet (aa + bb - cc - dd, 2 * (bc - ad), 2 * (bd + ac), _m[0]);
|
|
|
|
VectorSet (2 * (bc + ad), aa - bb + cc - dd, 2 * (cd - ab), _m[1]);
|
|
|
|
VectorSet (2 * (bd - ac), 2 * (cd + ab), aa - bb - cc + dd, _m[2]);
|
|
|
|
}
|
|
|
|
if (homogenous) {
|
|
|
|
_m[0][3] = 0;
|
|
|
|
_m[1][3] = 0;
|
|
|
|
_m[2][3] = 0;
|
|
|
|
VectorZero (_m[3]);
|
|
|
|
_m[3][3] = 1;
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
2001-02-19 21:15:25 +00:00
|
|
|
#if defined(_WIN32) && !defined(__GNUC__)
|
2001-08-22 22:03:16 +00:00
|
|
|
# pragma optimize( "", on )
|
2001-02-19 21:15:25 +00:00
|
|
|
#endif
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE float
|
2001-02-19 21:15:25 +00:00
|
|
|
anglemod (float a)
|
|
|
|
{
|
|
|
|
a = (360.0 / 65536) * ((int) (a * (65536 / 360.0)) & 65535);
|
|
|
|
return a;
|
|
|
|
}
|
|
|
|
|
|
|
|
/*
|
|
|
|
BOPS_Error
|
|
|
|
|
|
|
|
Split out like this for ASM to call.
|
|
|
|
*/
|
2003-01-06 18:28:13 +00:00
|
|
|
void __attribute__ ((noreturn)) BOPS_Error (void);
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void __attribute__ ((noreturn))
|
2001-02-19 21:15:25 +00:00
|
|
|
BOPS_Error (void)
|
|
|
|
{
|
|
|
|
Sys_Error ("BoxOnPlaneSide: Bad signbits");
|
|
|
|
}
|
|
|
|
|
|
|
|
#ifndef USE_INTEL_ASM
|
|
|
|
|
|
|
|
/*
|
|
|
|
BoxOnPlaneSide
|
|
|
|
|
|
|
|
Returns 1, 2, or 1 + 2
|
|
|
|
*/
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE int
|
2011-11-14 02:18:22 +00:00
|
|
|
BoxOnPlaneSide (const vec3_t emins, const vec3_t emaxs, plane_t *p)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
float dist1, dist2;
|
|
|
|
int sides;
|
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
#if 0
|
|
|
|
// this is done by the BOX_ON_PLANE_SIDE macro before
|
|
|
|
// calling this function
|
2001-04-10 02:36:50 +00:00
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
// fast axial cases
|
2001-02-19 21:15:25 +00:00
|
|
|
if (p->type < 3) {
|
|
|
|
if (p->dist <= emins[p->type])
|
|
|
|
return 1;
|
|
|
|
if (p->dist >= emaxs[p->type])
|
|
|
|
return 2;
|
|
|
|
return 3;
|
|
|
|
}
|
|
|
|
#endif
|
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
// general case
|
2001-02-19 21:15:25 +00:00
|
|
|
switch (p->signbits) {
|
|
|
|
case 0:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emaxs[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emins[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
|
|
|
break;
|
|
|
|
case 1:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emins[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emaxs[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
|
|
|
break;
|
|
|
|
case 2:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emaxs[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emins[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
|
|
|
break;
|
|
|
|
case 3:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emins[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emaxs[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
|
|
|
break;
|
|
|
|
case 4:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emaxs[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emins[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
|
|
|
break;
|
|
|
|
case 5:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emins[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emaxs[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
|
|
|
break;
|
|
|
|
case 6:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emaxs[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emins[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
|
|
|
break;
|
|
|
|
case 7:
|
2001-09-10 04:20:27 +00:00
|
|
|
dist1 = p->normal[0] * emins[0] + p->normal[1] * emins[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emins[2];
|
2001-09-10 04:20:27 +00:00
|
|
|
dist2 = p->normal[0] * emaxs[0] + p->normal[1] * emaxs[1] +
|
2001-02-19 21:15:25 +00:00
|
|
|
p->normal[2] * emaxs[2];
|
|
|
|
break;
|
|
|
|
default:
|
|
|
|
BOPS_Error ();
|
|
|
|
}
|
|
|
|
|
|
|
|
#if 0
|
|
|
|
int i;
|
|
|
|
vec3_t corners[2];
|
|
|
|
|
|
|
|
for (i = 0; i < 3; i++) {
|
|
|
|
if (plane->normal[i] < 0) {
|
|
|
|
corners[0][i] = emins[i];
|
|
|
|
corners[1][i] = emaxs[i];
|
|
|
|
} else {
|
|
|
|
corners[1][i] = emins[i];
|
|
|
|
corners[0][i] = emaxs[i];
|
|
|
|
}
|
|
|
|
}
|
|
|
|
dist = DotProduct (plane->normal, corners[0]) - plane->dist;
|
|
|
|
dist2 = DotProduct (plane->normal, corners[1]) - plane->dist;
|
|
|
|
sides = 0;
|
|
|
|
if (dist1 >= 0)
|
|
|
|
sides = 1;
|
|
|
|
if (dist2 < 0)
|
|
|
|
sides |= 2;
|
|
|
|
#endif
|
|
|
|
|
|
|
|
sides = 0;
|
|
|
|
if (dist1 >= p->dist)
|
|
|
|
sides = 1;
|
|
|
|
if (dist2 < p->dist)
|
|
|
|
sides |= 2;
|
|
|
|
|
|
|
|
#ifdef PARANOID
|
|
|
|
if (sides == 0)
|
|
|
|
Sys_Error ("BoxOnPlaneSide: sides==0");
|
|
|
|
#endif
|
|
|
|
|
|
|
|
return sides;
|
|
|
|
}
|
|
|
|
#endif
|
|
|
|
|
2003-03-10 20:44:50 +00:00
|
|
|
/*
|
|
|
|
angles is a left(?) handed system: 'pitch yaw roll' with x (pitch) axis to
|
|
|
|
the right, y (yaw) axis up and z (roll) axis forward.
|
|
|
|
|
|
|
|
the math in AngleVectors has the entity frame as left handed with x
|
|
|
|
(forward) axis forward, y (right) axis to the right and z (up) up. However,
|
2011-08-27 05:38:33 +00:00
|
|
|
the world is a right handed system with x to the right, y forward and
|
2003-03-10 20:44:50 +00:00
|
|
|
z up.
|
|
|
|
|
|
|
|
pitch =
|
|
|
|
cp 0 -sp
|
|
|
|
0 1 0
|
|
|
|
sp 0 cp
|
|
|
|
|
|
|
|
yaw =
|
|
|
|
cy sy 0
|
|
|
|
-sy cy 0
|
|
|
|
0 0 1
|
|
|
|
|
|
|
|
roll =
|
|
|
|
1 0 0
|
|
|
|
0 cr sr
|
|
|
|
0 -sr cr
|
|
|
|
|
|
|
|
final = roll * (pitch * yaw)
|
|
|
|
final =
|
|
|
|
[forward]
|
|
|
|
[-right] -ve due to left handed to right handed conversion
|
|
|
|
[up]
|
|
|
|
*/
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-01-03 05:29:38 +00:00
|
|
|
AngleVectors (const vec3_t angles, vec3_t forward, vec3_t right, vec3_t up)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
2001-09-10 04:20:27 +00:00
|
|
|
float angle, sr, sp, sy, cr, cp, cy;
|
2001-02-19 21:15:25 +00:00
|
|
|
|
|
|
|
angle = angles[YAW] * (M_PI * 2 / 360);
|
|
|
|
sy = sin (angle);
|
|
|
|
cy = cos (angle);
|
|
|
|
angle = angles[PITCH] * (M_PI * 2 / 360);
|
|
|
|
sp = sin (angle);
|
|
|
|
cp = cos (angle);
|
|
|
|
angle = angles[ROLL] * (M_PI * 2 / 360);
|
|
|
|
sr = sin (angle);
|
|
|
|
cr = cos (angle);
|
|
|
|
|
|
|
|
forward[0] = cp * cy;
|
|
|
|
forward[1] = cp * sy;
|
|
|
|
forward[2] = -sp;
|
2003-03-10 20:44:50 +00:00
|
|
|
// need to flip right because it's a left handed system in a right handed
|
|
|
|
// world
|
|
|
|
right[0] = -1 * (sr * sp * cy + cr * -sy);
|
|
|
|
right[1] = -1 * (sr * sp * sy + cr * cy);
|
|
|
|
right[2] = -1 * (sr * cp);
|
2001-02-19 21:15:25 +00:00
|
|
|
up[0] = (cr * sp * cy + -sr * -sy);
|
|
|
|
up[1] = (cr * sp * sy + -sr * cy);
|
|
|
|
up[2] = cr * cp;
|
|
|
|
}
|
|
|
|
|
2011-08-27 05:38:33 +00:00
|
|
|
VISIBLE void
|
|
|
|
AngleQuat (const vec3_t angles, quat_t q)
|
|
|
|
{
|
|
|
|
float alpha, sr, sp, sy, cr, cp, cy;
|
|
|
|
|
|
|
|
// alpha is half the angle
|
|
|
|
alpha = angles[YAW] * (M_PI / 360);
|
|
|
|
sy = sin (alpha);
|
|
|
|
cy = cos (alpha);
|
|
|
|
alpha = angles[PITCH] * (M_PI / 360);
|
|
|
|
sp = sin (alpha);
|
|
|
|
cp = cos (alpha);
|
|
|
|
alpha = angles[ROLL] * (M_PI / 360);
|
|
|
|
sr = sin (alpha);
|
|
|
|
cr = cos (alpha);
|
|
|
|
|
|
|
|
QuatSet (cy * cp * cr + sy * sp * sr,
|
|
|
|
cy * cp * sr - sy * sp * cr,
|
|
|
|
cy * sp * cr + sy * cp * sr,
|
|
|
|
sy * cp * cr - cy * sp * sr,
|
|
|
|
q);
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE int
|
2002-01-03 05:29:38 +00:00
|
|
|
_VectorCompare (const vec3_t v1, const vec3_t v2)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
int i;
|
|
|
|
|
|
|
|
for (i = 0; i < 3; i++)
|
2002-09-20 17:02:53 +00:00
|
|
|
if (fabs (v1[i] - v2[i]) > EQUAL_EPSILON)
|
2001-02-19 21:15:25 +00:00
|
|
|
return 0;
|
|
|
|
|
|
|
|
return 1;
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-01-03 05:29:38 +00:00
|
|
|
_VectorMA (const vec3_t veca, float scale, const vec3_t vecb, vec3_t vecc)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
vecc[0] = veca[0] + scale * vecb[0];
|
|
|
|
vecc[1] = veca[1] + scale * vecb[1];
|
|
|
|
vecc[2] = veca[2] + scale * vecb[2];
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE vec_t
|
2002-01-03 05:29:38 +00:00
|
|
|
_DotProduct (const vec3_t v1, const vec3_t v2)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
return v1[0] * v2[0] + v1[1] * v2[1] + v1[2] * v2[2];
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-01-03 05:29:38 +00:00
|
|
|
_VectorSubtract (const vec3_t veca, const vec3_t vecb, vec3_t out)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
out[0] = veca[0] - vecb[0];
|
|
|
|
out[1] = veca[1] - vecb[1];
|
|
|
|
out[2] = veca[2] - vecb[2];
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-01-03 05:29:38 +00:00
|
|
|
_VectorAdd (const vec3_t veca, const vec3_t vecb, vec3_t out)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
out[0] = veca[0] + vecb[0];
|
|
|
|
out[1] = veca[1] + vecb[1];
|
|
|
|
out[2] = veca[2] + vecb[2];
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-01-03 05:29:38 +00:00
|
|
|
_VectorCopy (const vec3_t in, vec3_t out)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
out[0] = in[0];
|
|
|
|
out[1] = in[1];
|
|
|
|
out[2] = in[2];
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2001-04-06 18:37:23 +00:00
|
|
|
CrossProduct (const vec3_t v1, const vec3_t v2, vec3_t cross)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
2002-01-04 06:13:50 +00:00
|
|
|
float v10 = v1[0];
|
|
|
|
float v11 = v1[1];
|
|
|
|
float v12 = v1[2];
|
|
|
|
float v20 = v2[0];
|
|
|
|
float v21 = v2[1];
|
|
|
|
float v22 = v2[2];
|
|
|
|
|
|
|
|
cross[0] = v11 * v22 - v12 * v21;
|
|
|
|
cross[1] = v12 * v20 - v10 * v22;
|
|
|
|
cross[2] = v10 * v21 - v11 * v20;
|
2001-02-19 21:15:25 +00:00
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE vec_t
|
2002-08-20 02:22:40 +00:00
|
|
|
_VectorLength (const vec3_t v)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
2001-09-10 04:20:27 +00:00
|
|
|
float length;
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2001-10-30 19:55:34 +00:00
|
|
|
length = sqrt (DotProduct (v, v));
|
2001-02-19 21:15:25 +00:00
|
|
|
return length;
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE vec_t
|
2002-09-25 21:35:49 +00:00
|
|
|
_VectorNormalize (vec3_t v)
|
|
|
|
{
|
|
|
|
int i;
|
|
|
|
double length;
|
|
|
|
|
|
|
|
length = 0;
|
2003-03-21 00:51:57 +00:00
|
|
|
for (i = 0; i < 3; i++)
|
2002-09-25 21:35:49 +00:00
|
|
|
length += v[i] * v[i];
|
|
|
|
length = sqrt (length);
|
|
|
|
if (length == 0)
|
|
|
|
return 0;
|
|
|
|
|
2003-03-21 00:51:57 +00:00
|
|
|
for (i = 0; i < 3; i++)
|
2002-09-25 21:35:49 +00:00
|
|
|
v[i] /= length;
|
|
|
|
|
|
|
|
return length;
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2002-01-03 05:29:38 +00:00
|
|
|
_VectorScale (const vec3_t in, vec_t scale, vec3_t out)
|
2001-02-19 21:15:25 +00:00
|
|
|
{
|
|
|
|
out[0] = in[0] * scale;
|
|
|
|
out[1] = in[1] * scale;
|
|
|
|
out[2] = in[2] * scale;
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE int
|
2001-02-19 21:15:25 +00:00
|
|
|
Q_log2 (int val)
|
|
|
|
{
|
|
|
|
int answer = 0;
|
|
|
|
|
|
|
|
while ((val >>= 1) != 0)
|
|
|
|
answer++;
|
|
|
|
return answer;
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2001-02-19 21:15:25 +00:00
|
|
|
R_ConcatRotations (float in1[3][3], float in2[3][3], float out[3][3])
|
|
|
|
{
|
|
|
|
out[0][0] = in1[0][0] * in2[0][0] + in1[0][1] * in2[1][0] +
|
|
|
|
in1[0][2] * in2[2][0];
|
|
|
|
out[0][1] = in1[0][0] * in2[0][1] + in1[0][1] * in2[1][1] +
|
|
|
|
in1[0][2] * in2[2][1];
|
|
|
|
out[0][2] = in1[0][0] * in2[0][2] + in1[0][1] * in2[1][2] +
|
|
|
|
in1[0][2] * in2[2][2];
|
|
|
|
out[1][0] = in1[1][0] * in2[0][0] + in1[1][1] * in2[1][0] +
|
|
|
|
in1[1][2] * in2[2][0];
|
|
|
|
out[1][1] = in1[1][0] * in2[0][1] + in1[1][1] * in2[1][1] +
|
|
|
|
in1[1][2] * in2[2][1];
|
|
|
|
out[1][2] = in1[1][0] * in2[0][2] + in1[1][1] * in2[1][2] +
|
|
|
|
in1[1][2] * in2[2][2];
|
|
|
|
out[2][0] = in1[2][0] * in2[0][0] + in1[2][1] * in2[1][0] +
|
|
|
|
in1[2][2] * in2[2][0];
|
|
|
|
out[2][1] = in1[2][0] * in2[0][1] + in1[2][1] * in2[1][1] +
|
|
|
|
in1[2][2] * in2[2][1];
|
|
|
|
out[2][2] = in1[2][0] * in2[0][2] + in1[2][1] * in2[1][2] +
|
|
|
|
in1[2][2] * in2[2][2];
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2001-02-19 21:15:25 +00:00
|
|
|
R_ConcatTransforms (float in1[3][4], float in2[3][4], float out[3][4])
|
|
|
|
{
|
|
|
|
out[0][0] = in1[0][0] * in2[0][0] + in1[0][1] * in2[1][0] +
|
|
|
|
in1[0][2] * in2[2][0];
|
|
|
|
out[0][1] = in1[0][0] * in2[0][1] + in1[0][1] * in2[1][1] +
|
|
|
|
in1[0][2] * in2[2][1];
|
|
|
|
out[0][2] = in1[0][0] * in2[0][2] + in1[0][1] * in2[1][2] +
|
|
|
|
in1[0][2] * in2[2][2];
|
|
|
|
out[0][3] = in1[0][0] * in2[0][3] + in1[0][1] * in2[1][3] +
|
|
|
|
in1[0][2] * in2[2][3] + in1[0][3];
|
|
|
|
out[1][0] = in1[1][0] * in2[0][0] + in1[1][1] * in2[1][0] +
|
|
|
|
in1[1][2] * in2[2][0];
|
|
|
|
out[1][1] = in1[1][0] * in2[0][1] + in1[1][1] * in2[1][1] +
|
|
|
|
in1[1][2] * in2[2][1];
|
|
|
|
out[1][2] = in1[1][0] * in2[0][2] + in1[1][1] * in2[1][2] +
|
|
|
|
in1[1][2] * in2[2][2];
|
|
|
|
out[1][3] = in1[1][0] * in2[0][3] + in1[1][1] * in2[1][3] +
|
|
|
|
in1[1][2] * in2[2][3] + in1[1][3];
|
|
|
|
out[2][0] = in1[2][0] * in2[0][0] + in1[2][1] * in2[1][0] +
|
|
|
|
in1[2][2] * in2[2][0];
|
|
|
|
out[2][1] = in1[2][0] * in2[0][1] + in1[2][1] * in2[1][1] +
|
|
|
|
in1[2][2] * in2[2][1];
|
|
|
|
out[2][2] = in1[2][0] * in2[0][2] + in1[2][1] * in2[1][2] +
|
|
|
|
in1[2][2] * in2[2][2];
|
|
|
|
out[2][3] = in1[2][0] * in2[0][3] + in1[2][1] * in2[1][3] +
|
|
|
|
in1[2][2] * in2[2][3] + in1[2][3];
|
|
|
|
}
|
|
|
|
|
|
|
|
/*
|
|
|
|
FloorDivMod
|
|
|
|
|
|
|
|
Returns mathematically correct (floor-based) quotient and remainder for
|
|
|
|
numer and denom, both of which should contain no fractional part. The
|
|
|
|
quotient must fit in 32 bits.
|
|
|
|
*/
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE void
|
2001-02-19 21:15:25 +00:00
|
|
|
FloorDivMod (double numer, double denom, int *quotient, int *rem)
|
|
|
|
{
|
2001-09-10 04:20:27 +00:00
|
|
|
double x;
|
|
|
|
int q, r;
|
2001-02-19 21:15:25 +00:00
|
|
|
|
|
|
|
#ifndef PARANOID
|
|
|
|
if (denom <= 0.0)
|
2002-05-14 06:12:29 +00:00
|
|
|
Sys_Error ("FloorDivMod: bad denominator %f", denom);
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
// if ((floor(numer) != numer) || (floor(denom) != denom))
|
2002-05-14 06:12:29 +00:00
|
|
|
// Sys_Error ("FloorDivMod: non-integer numer or denom %f %f",
|
2001-08-22 22:03:16 +00:00
|
|
|
// numer, denom);
|
2001-02-19 21:15:25 +00:00
|
|
|
#endif
|
|
|
|
|
|
|
|
if (numer >= 0.0) {
|
|
|
|
x = floor (numer / denom);
|
|
|
|
q = (int) x;
|
|
|
|
r = (int) floor (numer - (x * denom));
|
|
|
|
} else {
|
|
|
|
// perform operations with positive values, and fix mod to make
|
|
|
|
// floor-based
|
|
|
|
x = floor (-numer / denom);
|
|
|
|
q = -(int) x;
|
|
|
|
r = (int) floor (-numer - (x * denom));
|
|
|
|
if (r != 0) {
|
|
|
|
q--;
|
|
|
|
r = (int) denom - r;
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
*quotient = q;
|
|
|
|
*rem = r;
|
|
|
|
}
|
|
|
|
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE int
|
2001-02-19 21:15:25 +00:00
|
|
|
GreatestCommonDivisor (int i1, int i2)
|
|
|
|
{
|
|
|
|
if (i1 > i2) {
|
|
|
|
if (i2 == 0)
|
|
|
|
return (i1);
|
|
|
|
return GreatestCommonDivisor (i2, i1 % i2);
|
|
|
|
} else {
|
|
|
|
if (i1 == 0)
|
|
|
|
return (i2);
|
|
|
|
return GreatestCommonDivisor (i1, i2 % i1);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
#ifndef USE_INTEL_ASM
|
|
|
|
/*
|
2001-08-22 22:03:16 +00:00
|
|
|
Invert24To16
|
2001-02-19 21:15:25 +00:00
|
|
|
|
2001-08-22 22:03:16 +00:00
|
|
|
Inverts an 8.24 value to a 16.16 value
|
2001-02-19 21:15:25 +00:00
|
|
|
*/
|
2007-03-10 12:00:59 +00:00
|
|
|
VISIBLE fixed16_t
|
2001-02-19 21:15:25 +00:00
|
|
|
Invert24To16 (fixed16_t val)
|
|
|
|
{
|
|
|
|
if (val < 256)
|
|
|
|
return (0xFFFFFFFF);
|
|
|
|
|
|
|
|
return (fixed16_t)
|
|
|
|
(((double) 0x10000 * (double) 0x1000000 / (double) val) + 0.5);
|
|
|
|
}
|
|
|
|
#endif
|
2011-12-30 11:05:56 +00:00
|
|
|
|
|
|
|
void
|
|
|
|
Mat4Transpose (const mat4_t a, mat4_t b)
|
|
|
|
{
|
|
|
|
vec_t t;
|
|
|
|
int i, j;
|
|
|
|
|
|
|
|
for (i = 0; i < 3; i++) {
|
2011-12-31 04:20:31 +00:00
|
|
|
b[i * 4 + i] = a[i * 4 + i]; // in case b != a
|
2011-12-30 11:05:56 +00:00
|
|
|
for (j = i + 1; j < 4; j++) {
|
|
|
|
t = a[i * 4 + j]; // in case b == a
|
|
|
|
b[i * 4 + j] = a[j * 4 + i];
|
|
|
|
b[j * 4 + i] = t;
|
|
|
|
}
|
|
|
|
}
|
2011-12-31 04:20:31 +00:00
|
|
|
b[i * 4 + i] = a[i * 4 + i]; // in case b != a
|
2011-12-30 11:05:56 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
void
|
|
|
|
Mat4Mult (const mat4_t a, const mat4_t b, mat4_t c)
|
|
|
|
{
|
|
|
|
mat4_t ta, tb; // in case c == b or c == a
|
|
|
|
int i, j, k;
|
|
|
|
|
|
|
|
Mat4Transpose (a, ta); // transpose so we can use dot
|
|
|
|
Mat4Copy (b, tb);
|
|
|
|
|
|
|
|
k = 0;
|
|
|
|
for (i = 0; i < 4; i++) {
|
|
|
|
for (j = 0; j < 4; j++) {
|
|
|
|
c[k++] = QDotProduct (ta + 4 * j, tb + 4 * i);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|