doom3-gpl
Doom 3 GPL source release
 All Classes Namespaces Files Functions Variables Typedefs Enumerations Enumerator Friends Macros Pages
Classes | Macros | Typedefs | Functions
jdhuff.c File Reference
#include "jinclude.h"
#include "jpeglib.h"
#include "jdhuff.h"

Go to the source code of this file.

Classes

struct  savable_state
 
struct  huff_entropy_decoder
 

Macros

#define JPEG_INTERNALS
 
#define ASSIGN_STATE(dest, src)   ((dest) = (src))
 
#define MIN_GET_BITS   (BIT_BUF_SIZE-7)
 
#define HUFF_EXTEND(x, s)   ((x) < extend_test[s] ? (x) + extend_offset[s] : (x))
 

Typedefs

typedef huff_entropy_decoderhuff_entropy_ptr
 

Functions

METHODDEF void start_pass_huff_decoder (j_decompress_ptr cinfo)
 
GLOBAL void jpeg_make_d_derived_tbl (j_decompress_ptr cinfo, JHUFF_TBL *htbl, d_derived_tbl **pdtbl)
 
GLOBAL boolean jpeg_fill_bit_buffer (bitread_working_state *state, register bit_buf_type get_buffer, register int bits_left, int nbits)
 
GLOBAL int jpeg_huff_decode (bitread_working_state *state, register bit_buf_type get_buffer, register int bits_left, d_derived_tbl *htbl, int min_bits)
 
LOCAL boolean process_restart (j_decompress_ptr cinfo)
 
METHODDEF boolean decode_mcu (j_decompress_ptr cinfo, JBLOCKROW *MCU_data)
 
GLOBAL void jinit_huff_decoder (j_decompress_ptr cinfo)
 

Macro Definition Documentation

#define ASSIGN_STATE (   dest,
  src 
)    ((dest) = (src))

Definition at line 40 of file jdhuff.c.

#define HUFF_EXTEND (   x,
  s 
)    ((x) < extend_test[s] ? (x) + extend_offset[s] : (x))

Definition at line 372 of file jdhuff.c.

#define JPEG_INTERNALS

Definition at line 17 of file jdhuff.c.

#define MIN_GET_BITS   (BIT_BUF_SIZE-7)

Definition at line 229 of file jdhuff.c.

Typedef Documentation

Definition at line 69 of file jdhuff.c.

Function Documentation

METHODDEF boolean decode_mcu ( j_decompress_ptr  cinfo,
JBLOCKROW MCU_data 
)

Definition at line 437 of file jdhuff.c.

GLOBAL void jinit_huff_decoder ( j_decompress_ptr  cinfo)

Definition at line 558 of file jdhuff.c.

GLOBAL boolean jpeg_fill_bit_buffer ( bitread_working_state state,
register bit_buf_type  get_buffer,
register int  bits_left,
int  nbits 
)

Definition at line 234 of file jdhuff.c.

GLOBAL int jpeg_huff_decode ( bitread_working_state state,
register bit_buf_type  get_buffer,
register int  bits_left,
d_derived_tbl htbl,
int  min_bits 
)

Definition at line 322 of file jdhuff.c.

GLOBAL void jpeg_make_d_derived_tbl ( j_decompress_ptr  cinfo,
JHUFF_TBL htbl,
d_derived_tbl **  pdtbl 
)

Definition at line 128 of file jdhuff.c.

LOCAL boolean process_restart ( j_decompress_ptr  cinfo)

Definition at line 393 of file jdhuff.c.

METHODDEF void start_pass_huff_decoder ( j_decompress_ptr  cinfo)

Definition at line 77 of file jdhuff.c.