src/HOL/Option.thy
2012-09-07 haftmann combinator Option.these
2012-02-18 krauss added congruence rules for Option.{map|bind}
2011-01-11 haftmann "enriched_type" replaces less specific "type_lifting"
2010-12-21 haftmann tuned type_lifting declarations
2010-12-06 haftmann replace `type_mapper` by the more adequate `type_lifting`
2010-11-18 haftmann mapper for option type
2010-09-10 haftmann Haskell == is infix, not infixl
2010-09-06 wenzelm more antiquotations;
2010-09-05 krauss removed duplicate lemma
2010-09-05 krauss added Option.bind
2010-08-27 haftmann renamed class/constant eq to equal; tuned some instantiations
2010-07-19 haftmann Scala: subtle difference in printing strings vs. complex mixfix syntax
2010-04-16 wenzelm replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
2010-03-10 haftmann split off theory Big_Operators from theory Finite_Set
2010-01-13 haftmann some syntax setup for Scala
2009-07-14 haftmann prefer code_inline over code_unfold; use code_unfold_post where appropriate
2009-07-14 haftmann code attributes use common underscore convention
2009-05-14 haftmann preprocessing must consider eq
2009-05-09 nipkow lemmas by Andreas Lochbihler
2009-03-06 haftmann moved instance option :: finite to Option.thy
2009-03-04 nipkow Option.thy
2007-08-07 haftmann split off Option theory
2000-05-30 berghofe the is now defined using primrec, avoiding explicit use of arbitrary.
1998-09-09 oheimb AddIffs[not_None_eq];
1998-07-24 berghofe Adapted to new datatype package.
1998-03-24 oheimb added o2s
1997-11-10 oheimb replaced 8bit characters
1997-11-04 oheimb added the, option_map, and case analysis theorems
1996-09-24 nipkow Moved Option out of IOA into core HOL
less more (0) tip