author | wenzelm |
Wed, 04 Oct 2017 12:00:53 +0200 | |
changeset 66787 | 64b47495676d |
parent 66453 | cc19f7ca2ed6 |
child 67406 | 23307fd33906 |
permissions | -rw-r--r-- |
47613 | 1 |
theory Abs_Int_init |
66453
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
53013
diff
changeset
|
2 |
imports "HOL-Library.While_Combinator" |
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
wenzelm
parents:
53013
diff
changeset
|
3 |
"HOL-Library.Extended" |
47613 | 4 |
Vars Collecting Abs_Int_Tests |
5 |
begin |
|
6 |
||
51390 | 7 |
hide_const (open) top bot dom --"to avoid qualified names" |
47613 | 8 |
|
9 |
end |