| author | wenzelm | 
| Wed, 11 Oct 2023 11:37:18 +0200 | |
| changeset 78758 | 05da36bc806f | 
| parent 67443 | 3abf6a722518 | 
| 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: 
53013diff
changeset | 2 | imports "HOL-Library.While_Combinator" | 
| 
cc19f7ca2ed6
session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;
 wenzelm parents: 
53013diff
changeset | 3 | "HOL-Library.Extended" | 
| 47613 | 4 | Vars Collecting Abs_Int_Tests | 
| 5 | begin | |
| 6 | ||
| 67443 
3abf6a722518
standardized towards new-style formal comments: isabelle update_comments;
 wenzelm parents: 
67406diff
changeset | 7 | hide_const (open) top bot dom \<comment> \<open>to avoid qualified names\<close> | 
| 47613 | 8 | |
| 9 | end |