History log of /seL4-l4v-master/l4v/lib/sep_algebra/MonadSep.thy
Revision Date Author Comments
# a424d55e 09-Mar-2020 Gerwin Klein <gerwin.klein@data61.csiro.au>

licenses: convert license tags to SPDX


# 436eae28 10-Jan-2019 Callum Bannister <callum.bannister@data61.csiro.au>

lib: automation for separation logic & folds


# b5cdf470 13-Jun-2018 Gerwin Klein <gerwin.klein@data61.csiro.au>

globally use session-qualified imports; add Lib session

Session-qualified imports will be required for Isabelle2018 and help clarify
the structure of sessions in the build tree.

This commit mainly adds a new set of sessions for lib/, including a Lib
session that includes most theories in lib/ and a few separate sessions for
parts that have dependencies beyond CParser or are separate AFP sessions.
The group "lib" collects all lib/ sessions.

As a consequence, other theories should use lib/ theories by session name,
not by path, which in turns means spec and proof sessions should also refer
to each other by session name, not path, to avoid duplicate theory errors in
theory merges later.


# 47119bf4 13-Jan-2017 Gerwin Klein <gerwin.klein@nicta.com.au>

wp_cleanup: update proofs for new wp behaviour

The things that usually go wrong:
- wp fall through: add +, e.g.
apply (wp select_wp) -> apply (wp select_wp)+

- precondition: you can remove most hoare_pre, but wpc still needs it, and
sometimes the wp instance relies on being able to fit a rule to the
current non-schematic precondition. In that case, use "including no_pre"
to switch off the automatic hoare_pre application.

- very rarely there is a schematic postcondition that interferes with the
new trivial cleanup rules, because the rest of the script assumes some
specific state afterwards (shouldn't happen in a reasonable proof, but
not all proofs are reasonable..). In that case, (wp_once ...)+ should
emulate the old behaviour precisely.


# 41d4aa4f 25-Oct-2016 Matthew Brecknell <Matthew.Brecknell@data61.csiro.au>

Isabelle2016-1: update references to renamed constants and facts


# 5f0bf39c 27-Mar-2016 Gerwin Klein <gerwin.klein@nicta.com.au>

sep_algebra: cleanup

- fixed legacy warnings
- fixed almost all other warnings as well
- clarified some monoid lemmas that had misleading mixed notation
- improved layout style compliance (seriously, people..)
- comment typo fixes etc


# 7072c8e4 14-May-2015 Gerwin Klein <gerwin.klein@nicta.com.au>

lib/sep_algebra: 2015 update


# 7167ea42 08-Sep-2014 Andrew Boyton <andrew.boyton@nicta.com.au>

CapDL: Made IRQ Nodes a new object type, not a small CNode.

IRQ Nodes are now their own object type in capDL. This makes it much easier
to distinguish between "real" CNodes and IRQ Nodes.

Updated:
* the capDL refinement,
* the access proofs, and
* the system initialiser.


# 2a03e81d 14-Jul-2014 Gerwin Klein <gerwin.klein@nicta.com.au>

Import release snapshot.