Codebase list coq / upstream/8.2.beta4+dfsg ide / config_parser.mly
upstream/8.2.beta4+dfsg

Tree @upstream/8.2.beta4+dfsg (Download .tar.gz)

config_parser.mly @upstream/8.2.beta4+dfsgraw · history · blame

/***********************************************************************)
(*  v      *   The Coq Proof Assistant  /  The Coq Development Team     *)
(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
(*   \VV/  **************************************************************)
(*    //   *      This file is distributed under the terms of the       *)
(*         *       GNU Lesser General Public License Version 2.1        *)
(***********************************************************************/

/* $Id: config_parser.mly 5920 2004-07-16 20:01:26Z herbelin $ */

%{

  open Parsing
  open Util

%}

%token <string> IDENT STRING
%token EQUAL EOF

%type <(string list) Util.Stringmap.t> prefs
%start prefs

%%

prefs:
  pref_list EOF { $1 }
;

pref_list:
   pref_list pref { let (k,d) = $2 in Stringmap.add k d $1 }
 | /* epsilon */  { Stringmap.empty }
;

pref:
  IDENT EQUAL string_list { ($1, List.rev $3) }
;

string_list:
   string_list STRING { $2 :: $1 }
 | /* epsilon */      { [] }
;