Added 'ambiguity_is_error' flag, which, if set, makes the parser fail,
rather than just issue a warning, when the input parsed is ambiguous.
(* Title: HOLCF/One.thy
ID: $Id$
Author: Oscar Slotosch
License: GPL (GNU GENERAL PUBLIC LICENSE)
*)
One = Lift +
types one = unit lift
constdefs
ONE :: "one"
"ONE == Def ()"
translations
"one" <= (type) "unit lift"
end