changeset 58372 | bfd497f2f4c2 |
parent 58353 | c9f374b64d99 |
child 58377 | c6f93b8d2d8e |
1.1 --- a/src/HOL/Main.thy Thu Sep 18 16:47:40 2014 +0200 1.2 +++ b/src/HOL/Main.thy Thu Sep 18 16:47:40 2014 +0200 1.3 @@ -2,7 +2,7 @@ 1.4 1.5 theory Main 1.6 imports Predicate_Compile Quickcheck_Narrowing Extraction Lifting_Sum Coinduction Nitpick 1.7 - Basic_BNF_Least_Fixpoints BNF_Greatest_Fixpoint Old_Datatype 1.8 + Basic_BNF_Least_Fixpoints BNF_Greatest_Fixpoint 1.9 begin 1.10 1.11 text {*