History log of /seL4-l4v-master/isabelle/src/HOL/ex/Coercion_Examples.thy
Revision Date Author Comments
# a7ccdf43 10-Jan-2018 nipkow <none@none>

ran isabelle update_op on all sources


# 8f53ef93 06-Mar-2014 blanchet <none@none>

renamed 'map_pair' to 'map_prod'


# b517a6ea 15-Nov-2013 haftmann <none@none>

dropped duplicate of of_bool

--HG--
extra : rebase_source : 92e27f8d7a09e9ba086ec4a2cdf2876b327b9c28


# 1e5939eb 05-Mar-2013 traytel <none@none>

allow more general coercion maps; tuned;


# a0e73230 01-Mar-2013 traytel <none@none>

coercion-invariant arguments at work


# 5f6496e5 22-Feb-2013 traytel <none@none>

Coercion_Examples defines required coercions itself (no Complex_Main needed)


# 6f80896a 01-Dec-2010 wenzelm <none@none>

activate subtyping/coercions in theory Complex_Main;


# dfd9c5cb 01-Nov-2010 traytel <none@none>

Attribute map_function -> coercion_map;
tuned;


# 2c880186 29-Oct-2010 wenzelm <none@none>

proper signature constraint for ML structure;
explicit theory setup, which is customary outside Pure;
formal @{binding} instead of Binding.name;


# 8ad05042 29-Oct-2010 wenzelm <none@none>

proper header;
tuned whitespace;


# 6c1f2425 29-Oct-2010 wenzelm <none@none>

Coercive subtyping via subtype constraints, by Dmitriy Traytel (21-Oct-2010).