Library Pip.Proof.Isolation

Summary

This file contains the formalization of interesting properties that we need to prove
Require Import Pip.Model.ADT Pip.Model.Hardware Pip.Model.Lib Pip.Model.MAL.
Require Import Pip.Proof.StateLib Pip.Proof.Lib.
Require Import List.
Import List.ListNotations.
THE VERTICAL SHARING PROPERTY: All child used pages (configuration tables and mapped pages) are mapped into the parent partition
THE ISOLATION PROPERTY BETWEEN PARTITIONS, If we take two different children of a given parent, so all their used pages are different
THE ISOLATION PROPERTY BETWEEN THE KERNEL DATA AND PARTITIONS kernel data is the configuration pages of partitions. All configuration tables of a given partition are inaccessible by all partitions