Codebase list coq / run/7ee233ae-feee-4286-8d93-3c2a58e14708/main gramlib / gramext.ml
run/7ee233ae-feee-4286-8d93-3c2a58e14708/main

Tree @run/7ee233ae-feee-4286-8d93-3c2a58e14708/main (Download .tar.gz)

gramext.ml @run/7ee233ae-feee-4286-8d93-3c2a58e14708/mainraw · history · blame

(* camlp5r *)
(* gramext.ml,v *)
(* Copyright (c) INRIA 2007-2017 *)

type position =
  | First
  | Last
  | Before of string
  | After of string

type g_assoc = NonA | RightA | LeftA

let pr_assoc = function
  | LeftA -> Pp.str "left associativity"
  | RightA -> Pp.str "right associativity"
  | NonA -> Pp.str "no associativity"