equal
deleted
inserted
replaced
1563 |
1563 |
1564 Lemmas involving predicates on relations can also be registered |
1564 Lemmas involving predicates on relations can also be registered |
1565 using the same attribute. For example: |
1565 using the same attribute. For example: |
1566 |
1566 |
1567 @{text "bi_unique A \<Longrightarrow> (list_all2 A ===> op =) distinct distinct"}\\ |
1567 @{text "bi_unique A \<Longrightarrow> (list_all2 A ===> op =) distinct distinct"}\\ |
1568 @{text "\<lbrakk>bi_unique A; bi_unique B\<rbrakk> \<Longrightarrow> bi_unique (prod_rel A B)"} |
1568 @{text "\<lbrakk>bi_unique A; bi_unique B\<rbrakk> \<Longrightarrow> bi_unique (rel_prod A B)"} |
1569 |
1569 |
1570 \item @{attribute (HOL) "transfer_domain_rule"} attribute maintains a collection |
1570 \item @{attribute (HOL) "transfer_domain_rule"} attribute maintains a collection |
1571 of rules, which specify a domain of a transfer relation by a predicate. |
1571 of rules, which specify a domain of a transfer relation by a predicate. |
1572 E.g., given the transfer relation @{text "ZN x n \<equiv> (x = int n)"}, |
1572 E.g., given the transfer relation @{text "ZN x n \<equiv> (x = int n)"}, |
1573 one can register the following transfer domain rule: |
1573 one can register the following transfer domain rule: |