made "mk_case_eq_tac" work in the case where the first constructor is an "alternate" constructor (in which case its discriminator paradoxically starts with a negation)
(* Author: Florian Haftmann, TU Muenchen *)
header {* Generating code using pretty literals and natural number literals  *}
theory Candidates_Pretty
imports Candidates Code_Char_ord Efficient_Nat
begin
end