History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Bali/DeclConcepts.thy
Revision Date Author Comments
# 977ba149 13-Mar-2020 wenzelm <none@none>

proper escape for literal single quotes;


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# d4c96e26 15-Jun-2018 nipkow <none@none>

empty -> Map.empty


# f5796e6d 14-Feb-2018 wenzelm <none@none>

more symbols;


# 5385dbfa 16-Jan-2018 wenzelm <none@none>

standardized towards new-style formal comments: isabelle update_comments;


# d9ef7419 02-Jan-2016 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 18551fee 13-Oct-2015 haftmann <none@none>

prod_case as canonical name for product type eliminator


# a2c9fcbe 12-Mar-2015 wenzelm <none@none>

quote "method" to allow Eisbach using this keyword;


# c6877bda 02-Nov-2014 wenzelm <none@none>

modernized header;


# e91e0c03 16-Feb-2014 blanchet <none@none>

folded 'Option.set' into BNF-generated 'set_option'


# a64a7b69 27-Feb-2012 wenzelm <none@none>

tuned proofs;


# f55a6ddf 12-Nov-2011 wenzelm <none@none>

tuned specifications and proofs;


# 3ec8ee77 18-Feb-2011 wenzelm <none@none>

modernized specifications;


# 23accfa8 18-Aug-2010 haftmann <none@none>

adjusted to changed naming convention of logical record types


# 9d68725b 26-Jul-2010 wenzelm <none@none>

modernized/unified some specifications;


# 53a0b22e 01-Jul-2010 haftmann <none@none>

"prod" and "sum" replace "*" and "+" respectively


# b05afef4 11-Jun-2010 haftmann <none@none>

modernized specifications


# 1a1e1c5f 26-Apr-2010 huffman <none@none>

fix if-then-else parse error


# 6bc0017f 02-Mar-2010 wenzelm <none@none>

cleanup type translations;


# 90f5724e 01-Mar-2010 krauss <none@none>

killed more recdefs


# baea5702 01-Mar-2010 haftmann <none@none>

replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)


# 7d42ef37 23-Feb-2010 haftmann <none@none>

dropped axclass


# 803f34cc 09-Feb-2010 wenzelm <none@none>

modernized syntax translations, using mostly abbreviation/notation;
minor tuning;


# 4d0c51ec 30-Jan-2010 berghofe <none@none>

Adapted to changes in cases method.


# f94fe110 10-Jan-2010 berghofe <none@none>

Adapted to changes in induct method.


# 079cde2d 17-Oct-2009 wenzelm <none@none>

eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;


# 0561c763 25-Sep-2009 Thomas Sewell <tsewell@nicta.com.au>

Avoid record-inner constants in polymorphic definitions in Bali

The Bali package needs to insert a record extension into a type
class and define an associated polymorphic constant. There is no
elegant way to do this.

The existing approach was to insert every record extension into
the type class, defining the polymorphic constant at each layer
using inner operations created by the record package. Some of
those operations have been removed. They can be replaced by use
of record_name.extend if necessary, but we can also sidestep
this altogether.

The simpler approach here is to use defs(overloaded) once to
provide a single definition for the composition of all the type
constructors, which seems to be permitted. This gets us exactly
the fact we need, with the cost that some types that were
admitted to the type class have no definition for the constant
at all.


# 86665271 22-Jul-2009 haftmann <none@none>

set intersection and union now named inter and union


# b391ac6a 04-Mar-2009 nipkow <none@none>

Made Option a separate theory and renamed option_map to Option.map


# 46ba2765 22-Oct-2007 wenzelm <none@none>

abbrevs within inductive definitions may no longer depend on each other (reflects in internal organization, particularly for output);


# c32053dd 29-Jul-2007 wenzelm <none@none>

replaced make_imp by rev_mp;


# a44b194c 11-Jul-2007 berghofe <none@none>

Renamed inductive2 to inductive.


# 69946907 09-Mar-2007 haftmann <none@none>

resolved name clashes


# fd8a9d0e 11-Dec-2006 berghofe <none@none>

Adapted to new inductive definition package.


# 5d9071b0 05-May-2006 krauss <none@none>

First usable version of the new function definition package (HOL/function_packake/...).
Moved Accessible_Part.thy from Library to Main.


# a7060872 17-Jun-2005 haftmann <none@none>

migrated theory headers to new format


# 33b1b845 21-Jun-2004 kleing <none@none>

Merged in license change from Isabelle2004


# dcaa2c51 06-May-2004 schirmer <none@none>

tuned HOL/record package; enabled record_upd_simproc by default.


# 53e6b773 03-May-2004 schirmer <none@none>

reimplementation of HOL records; only one type is created for
each record extension, instead of one type for each field. See NEWS.


# 94091e29 14-May-2003 schirmer <none@none>

Adapted to changes in Map.thy


# efd5dc29 14-May-2003 nipkow <none@none>

*** empty log message ***


# c4a5cd8d 31-Oct-2002 schirmer <none@none>

"Definite Assignment Analysis" included, with proof of correctness. Large adjustments of type safety proof and soundness proof of the axiomatic semantics were necessary. Completeness proof of the loop rule of the axiomatic semantic was altered. So the additional polymorphic variants of some rules could be removed.


# 4803de87 26-Sep-2002 paulson <none@none>

Converted Fun to Isar style.
Moved Pi, funcset, restrict from Fun.thy to Library/FuncSet.thy.
Renamed constant "Fun.op o" to "Fun.comp"


# 647bcb01 27-Aug-2002 wenzelm <none@none>

*** empty log message ***


# c14eef5e 27-Feb-2002 schirmer <none@none>

Cleaning up the definition of static overriding.


# 74fc2075 25-Feb-2002 wenzelm <none@none>

clarified syntax of ``long'' statements: fixes/assumes/shows;


# 55bc1056 22-Feb-2002 schirmer <none@none>

Added check for field/method access to operational semantics and proved the acesses valid.


# f54d2aab 28-Jan-2002 wenzelm <none@none>

tuned;


# 77d49ccc 28-Jan-2002 schirmer <none@none>

Isabelle/Bali sources;